Skip to content

Commit

Permalink
Fix to "preserves" syntax merge
Browse files Browse the repository at this point in the history
  • Loading branch information
simondfoster committed Jul 17, 2024
1 parent 6265785 commit 361be9b
Showing 1 changed file with 0 additions and 10 deletions.
10 changes: 0 additions & 10 deletions Z_Machine.thy
Original file line number Diff line number Diff line change
Expand Up @@ -80,16 +80,6 @@ definition z_machine :: "('s::default) subst \<Rightarrow> ('e, 's) htree list \
[code_unfold]: "z_machine Init Ops = process Init (loop (foldr (\<box>) Ops Stop))"
*)

syntax
"_preserves" :: "logic \<Rightarrow> logic \<Rightarrow> logic" (infix "preserves" 40)
"_preserves_under" :: "logic \<Rightarrow> logic \<Rightarrow> logic \<Rightarrow> logic" ("_ preserves _ under _" [40, 0, 40] 40)
"_establishes" :: "logic \<Rightarrow> logic \<Rightarrow> logic" (infix "establishes" 40)

translations
"_preserves S P" => "H{P} S {P}"
"_preserves_under S P Q" => "H{P \<and> Q} S {P}"
"_establishes \<sigma> P" => "H{CONST True} \<langle>\<sigma>\<rangle>\<^sub>a {P}"

lemma deadlock_free_z_machine:
fixes Inv :: "'s::default \<Rightarrow> bool"
assumes
Expand Down

0 comments on commit 361be9b

Please sign in to comment.