src/HOL/Hoare_Parallel/Mul_Gar_Coll.thy
changeset 32687 27530efec97a
parent 32621 a073cb249a06
child 32960 69916a850301
equal deleted inserted replaced
32686:a62c8627931b 32687:27530efec97a
   274  apply(rule disjI2, clarify, erule less_SucE, force)
   274  apply(rule disjI2, clarify, erule less_SucE, force)
   275  apply(case_tac "M x!snd(E x! ind x)=Black")
   275  apply(case_tac "M x!snd(E x! ind x)=Black")
   276   apply(force)
   276   apply(force)
   277  apply(force)
   277  apply(force)
   278 apply(rule disjI2, rule disjI1, erule subset_psubset_trans, erule Graph11, force)
   278 apply(rule disjI2, rule disjI1, erule subset_psubset_trans, erule Graph11, force)
   279 --{* 3 subgoals left *}
       
   280 apply force
       
   281 --{* 2 subgoals left *}
   279 --{* 2 subgoals left *}
   282 apply clarify
   280 apply clarify
   283 apply(conjI_tac)
   281 apply(conjI_tac)
   284 apply(disjE_tac)
   282 apply(disjE_tac)
   285  apply (simp_all)
   283  apply (simp_all)
  1233 apply interfree_aux
  1231 apply interfree_aux
  1234 apply(simp_all add:mul_collector_mutator_interfree)
  1232 apply(simp_all add:mul_collector_mutator_interfree)
  1235 apply(unfold mul_modules mul_collector_defs mul_mutator_defs)
  1233 apply(unfold mul_modules mul_collector_defs mul_mutator_defs)
  1236 apply(tactic  {* TRYALL (interfree_aux_tac) *})
  1234 apply(tactic  {* TRYALL (interfree_aux_tac) *})
  1237 --{* 76 subgoals left *}
  1235 --{* 76 subgoals left *}
  1238 apply (clarify,simp add: nth_list_update)+
  1236 apply (clarsimp simp add: nth_list_update)+
  1239 --{* 56 subgoals left *}
  1237 --{* 56 subgoals left *}
  1240 apply(clarify,simp add:Mul_AppendInv_def Append_to_free0 nth_list_update)+
  1238 apply (clarsimp simp add: Mul_AppendInv_def Append_to_free0 nth_list_update)+
  1241 done
  1239 done
  1242 
  1240 
  1243 subsubsection {* The Multi-Mutator Garbage Collection Algorithm *}
  1241 subsubsection {* The Multi-Mutator Garbage Collection Algorithm *}
  1244 
  1242 
  1245 text {* The total number of verification conditions is 328 *}
  1243 text {* The total number of verification conditions is 328 *}