src/ZF/IMP/Equiv.thy
changeset 14060 c0c4af41fa3b
parent 13612 55d32e76ef4e
child 16417 9bc16273c2d4
--- a/src/ZF/IMP/Equiv.thy	Thu Jun 19 18:40:39 2003 +0200
+++ b/src/ZF/IMP/Equiv.thy	Fri Jun 20 12:10:45 2003 +0200
@@ -39,8 +39,6 @@
 lemma com1: "<c,sigma> -c-> sigma' ==> <sigma,sigma'> \<in> C(c)"
   apply (erule evalc.induct)
         apply (simp_all (no_asm_simp))
-      txt {* @{text skip} *}
-      apply fast
      txt {* @{text assign} *}
      apply (simp add: update_type)
     txt {* @{text comp} *}
@@ -48,7 +46,6 @@
    txt {* @{text while} *}
    apply (erule Gamma_bnd_mono [THEN lfp_unfold, THEN ssubst, OF C_subset])
    apply (simp add: Gamma_def)
-   apply force
   txt {* recursive case of @{text while} *}
   apply (erule Gamma_bnd_mono [THEN lfp_unfold, THEN ssubst, OF C_subset])
   apply (auto simp add: Gamma_def)