src/HOL/IMP/Denotation.thy
changeset 34055 fdf294ee08b2
parent 32235 8f9b8d14fc9f
child 41589 bbd861837ebc
--- a/src/HOL/IMP/Denotation.thy	Thu Dec 10 17:34:09 2009 +0000
+++ b/src/HOL/IMP/Denotation.thy	Thu Dec 10 17:34:18 2009 +0000
@@ -47,22 +47,20 @@
 apply (subst lfp_unfold[OF Gamma_mono, simplified Gamma_def])
 apply fast
 apply (subst lfp_unfold[OF Gamma_mono, simplified Gamma_def])
-apply fast
+apply auto 
 done
 
 (* Denotational Semantics implies Operational Semantics *)
 
 lemma com2: "(s,t) \<in> C(c) \<Longrightarrow> \<langle>c,s\<rangle> \<longrightarrow>\<^sub>c t"
 apply (induct c arbitrary: s t)
-
-apply simp_all
-apply fast
-apply fast
+apply auto 
+apply blast
 
 (* while *)
 apply (erule lfp_induct2 [OF _ Gamma_mono])
 apply (unfold Gamma_def)
-apply fast
+apply auto
 done