src/HOLCF/IOA/NTP/Impl.thy
changeset 28265 7e14443f2dd6
parent 27361 24ec32bee347
child 28839 32d498cf7595
equal deleted inserted replaced
28264:e1dae766c108 28265:7e14443f2dd6
   197   apply (simp (no_asm_simp) add: impl_ioas split del: split_if)
   197   apply (simp (no_asm_simp) add: impl_ioas split del: split_if)
   198   apply (induct_tac "a")
   198   apply (induct_tac "a")
   199 
   199 
   200   txt {* 10 cases. First 4 are simple, since state doesn't change *}
   200   txt {* 10 cases. First 4 are simple, since state doesn't change *}
   201 
   201 
   202 ML_command {* val tac2 = asm_full_simp_tac (ss addsimps [@{thm inv2_def}]) *}
   202   ML_prf {* val tac2 = asm_full_simp_tac (ss addsimps [@{thm inv2_def}]) *}
   203 
   203 
   204   txt {* 10 - 7 *}
   204   txt {* 10 - 7 *}
   205   apply (tactic "EVERY1 [tac2,tac2,tac2,tac2]")
   205   apply (tactic "EVERY1 [tac2,tac2,tac2,tac2]")
   206   txt {* 6 *}
   206   txt {* 6 *}
   207   apply (tactic {* forward_tac [rewrite_rule [@{thm Impl.inv1_def}]
   207   apply (tactic {* forward_tac [rewrite_rule [@{thm Impl.inv1_def}]
   253   apply (simp add: Impl.inv3_def receiver_projections sender_projections impl_ioas)
   253   apply (simp add: Impl.inv3_def receiver_projections sender_projections impl_ioas)
   254 
   254 
   255   apply (simp (no_asm_simp) add: impl_ioas split del: split_if)
   255   apply (simp (no_asm_simp) add: impl_ioas split del: split_if)
   256   apply (induct_tac "a")
   256   apply (induct_tac "a")
   257 
   257 
   258 ML_command {* val tac3 = asm_full_simp_tac (ss addsimps [@{thm inv3_def}]) *}
   258   ML_prf {* val tac3 = asm_full_simp_tac (ss addsimps [@{thm inv3_def}]) *}
   259 
   259 
   260   txt {* 10 - 8 *}
   260   txt {* 10 - 8 *}
   261 
   261 
   262   apply (tactic "EVERY1[tac3,tac3,tac3]")
   262   apply (tactic "EVERY1[tac3,tac3,tac3]")
   263 
   263 
   318   apply (simp add: Impl.inv4_def receiver_projections sender_projections impl_ioas)
   318   apply (simp add: Impl.inv4_def receiver_projections sender_projections impl_ioas)
   319 
   319 
   320   apply (simp (no_asm_simp) add: impl_ioas split del: split_if)
   320   apply (simp (no_asm_simp) add: impl_ioas split del: split_if)
   321   apply (induct_tac "a")
   321   apply (induct_tac "a")
   322 
   322 
   323 ML_command {* val tac4 =  asm_full_simp_tac (ss addsimps [@{thm inv4_def}]) *}
   323   ML_prf {* val tac4 =  asm_full_simp_tac (ss addsimps [@{thm inv4_def}]) *}
   324 
   324 
   325   txt {* 10 - 2 *}
   325   txt {* 10 - 2 *}
   326 
   326 
   327   apply (tactic "EVERY1[tac4,tac4,tac4,tac4,tac4,tac4,tac4,tac4,tac4]")
   327   apply (tactic "EVERY1[tac4,tac4,tac4,tac4,tac4,tac4,tac4,tac4,tac4]")
   328 
   328