src/HOL/Hoare_Parallel/Gar_Coll.thy
changeset 58963 26bf09b95dda
parent 58884 be4d203d35b3
child 59189 ad8e0a789af6
equal deleted inserted replaced
58960:4bee6d8c1500 58963:26bf09b95dda
   775 --{* 20 subgoals left *}
   775 --{* 20 subgoals left *}
   776 apply(tactic{* TRYALL (clarify_tac @{context}) *})
   776 apply(tactic{* TRYALL (clarify_tac @{context}) *})
   777 apply(simp_all add:Graph6 Graph7 Graph8 Append_to_free0 Append_to_free1 Graph12)
   777 apply(simp_all add:Graph6 Graph7 Graph8 Append_to_free0 Append_to_free1 Graph12)
   778 apply(tactic {* TRYALL (etac disjE) *})
   778 apply(tactic {* TRYALL (etac disjE) *})
   779 apply simp_all
   779 apply simp_all
   780 apply(tactic {* TRYALL(EVERY'[rtac disjI2,rtac subset_trans,etac @{thm Graph3},force_tac @{context}, assume_tac]) *})
   780 apply(tactic {* TRYALL(EVERY'[rtac disjI2,rtac subset_trans,etac @{thm Graph3},force_tac @{context}, assume_tac @{context}]) *})
   781 apply(tactic {* TRYALL(EVERY'[rtac disjI2,etac subset_trans,rtac @{thm Graph9},force_tac @{context}]) *})
   781 apply(tactic {* TRYALL(EVERY'[rtac disjI2,etac subset_trans,rtac @{thm Graph9},force_tac @{context}]) *})
   782 apply(tactic {* TRYALL(EVERY'[rtac disjI1,etac @{thm psubset_subset_trans},rtac @{thm Graph9},force_tac @{context}]) *})
   782 apply(tactic {* TRYALL(EVERY'[rtac disjI1,etac @{thm psubset_subset_trans},rtac @{thm Graph9},force_tac @{context}]) *})
   783 done
   783 done
   784 
   784 
   785 subsubsection {* Interference freedom Mutator-Collector *}
   785 subsubsection {* Interference freedom Mutator-Collector *}