Skip to content

Commit

Permalink
[squash] minor adjustments
Browse files Browse the repository at this point in the history
  • Loading branch information
Xaphiosis committed Dec 9, 2024
1 parent 7d8844e commit 973b1e3
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 4 deletions.
5 changes: 2 additions & 3 deletions proof/refine/AARCH64/ArchInvsDefs_H.thy
Original file line number Diff line number Diff line change
Expand Up @@ -6,8 +6,8 @@
*)

(* This theory contains the arch-dependent part of invariant definitions.
Due to the large amount of definitins, we opt for a Pre file rather than fixing constants in
locales. *)
Due to the large amount of definitions, we place it before Invariants_H rather than fixing
constants in locales. *)

theory ArchInvsDefs_H
imports
Expand All @@ -33,7 +33,6 @@ requalify_facts (aliasing)
Retype_H.createObject_def Retype_H.capUntypedPtr_def Retype_H.capUntypedSize_def
Retype_H.performInvocation_def Retype_H.decodeInvocation_def
end

end

context Arch begin arch_global_naming
Expand Down
1 change: 0 additions & 1 deletion proof/refine/Invariants_H.thy
Original file line number Diff line number Diff line change
Expand Up @@ -174,7 +174,6 @@ primrec live0' :: "Structures_H.kernel_object \<Rightarrow> bool" where

(* hyp_refs *)

(* FIXME arch-split: do we want to expose this, or put it in Arch? *)
definition hyp_refs_of' :: "kernel_object \<Rightarrow> (obj_ref \<times> reftype) set" where
"hyp_refs_of' x \<equiv> case x of
(KOTCB tcb) \<Rightarrow> tcb_hyp_refs' (tcbArch tcb)
Expand Down

0 comments on commit 973b1e3

Please sign in to comment.