lh-l4v/spec/abstract/RISCV64/Hypervisor_A.thy

20 lines
439 B
Plaintext
Raw Normal View History

(*
2020-03-09 06:18:30 +00:00
* Copyright 2020, Data61, CSIRO (ABN 41 687 119 230)
*
2020-03-09 06:18:30 +00:00
* SPDX-License-Identifier: GPL-2.0-only
*)
2018-08-06 09:05:25 +00:00
chapter "Handle Hypervisor Fault Events"
theory Hypervisor_A
imports Exceptions_A
begin
context Arch begin global_naming RISCV64_A
fun handle_hypervisor_fault :: "machine_word \<Rightarrow> hyp_fault_type \<Rightarrow> (unit, 'z::state_ext) s_monad"
2018-08-06 09:05:25 +00:00
where
"handle_hypervisor_fault thread RISCVNoHypFaults = return ()"
end
end