src/HOL/HOLCF/IOA/meta_theory/CompoTraces.thy
changeset 44890 22f665a2e91c
parent 42151 4da4fc77664b
child 45625 750c5a47400b
equal deleted inserted replaced
44889:340df9f3491f 44890:22f665a2e91c
   297 apply assumption
   297 apply assumption
   298 (* IH *)
   298 (* IH *)
   299 apply (simp add: not_ext_is_int_or_not_act ForallTL ForallDropwhile)
   299 apply (simp add: not_ext_is_int_or_not_act ForallTL ForallDropwhile)
   300 
   300 
   301 (* a~: act B; a~: act A *)
   301 (* a~: act B; a~: act A *)
   302 apply (fastsimp intro!: ext_is_act simp: externals_of_par)
   302 apply (fastforce intro!: ext_is_act simp: externals_of_par)
   303 done
   303 done
   304 
   304 
   305 declare FiniteConc [simp]
   305 declare FiniteConc [simp]
   306 
   306 
   307 declare FilterConc [simp del]
   307 declare FilterConc [simp del]
   450 back
   450 back
   451 apply assumption
   451 apply assumption
   452 apply (simp add: not_ext_is_int_or_not_act ForallTL ForallDropwhile)
   452 apply (simp add: not_ext_is_int_or_not_act ForallTL ForallDropwhile)
   453 
   453 
   454 (* Case a~:A, a~:B *)
   454 (* Case a~:A, a~:B *)
   455 apply (fastsimp intro!: ext_is_act simp: externals_of_par)
   455 apply (fastforce intro!: ext_is_act simp: externals_of_par)
   456 done
   456 done
   457 
   457 
   458 
   458 
   459 subsection" Filter of mksch(tr,schA,schB) to A is schA -- take lemma proof"
   459 subsection" Filter of mksch(tr,schA,schB) to A is schA -- take lemma proof"
   460 
   460