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

29 lines
760 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
*)
chapter "Architecture-specific TCB functions"
theory ArchTcb_A
imports KHeap_A
begin
context Arch begin global_naming RISCV64_A
2018-08-06 09:05:25 +00:00
definition sanitise_register :: "bool \<Rightarrow> register \<Rightarrow> machine_word \<Rightarrow> machine_word"
where
"sanitise_register t r v \<equiv> v"
2018-08-06 09:05:25 +00:00
definition arch_get_sanitise_register_info :: "obj_ref \<Rightarrow> (bool, 'a::state_ext) s_monad"
where
"arch_get_sanitise_register_info t \<equiv> return False"
2018-08-06 09:05:25 +00:00
definition arch_post_modify_registers :: "obj_ref \<Rightarrow> obj_ref \<Rightarrow> (unit, 'a::state_ext) s_monad"
where
"arch_post_modify_registers cur t \<equiv> return ()"
end
end