src/HOL/Bali/Eval.thy
changeset 44890 22f665a2e91c
parent 41778 5f79a9e42507
child 51717 9e7d1c139569
--- a/src/HOL/Bali/Eval.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Bali/Eval.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -901,7 +901,7 @@
     then have "False" by induct auto
   }  
   then show ?thesis
-    by (cases s') fastsimp
+    by (cases s') fastforce
 qed
 
 
@@ -914,7 +914,7 @@
     then have "False" by induct auto
   }
   then show ?thesis
-    by (cases s') fastsimp
+    by (cases s') fastforce
 qed
 
 lemma eval_InsInitV: "G\<turnstile>Norm s\<midarrow>InsInitV c w=\<succ>v\<rightarrow> s' = False"
@@ -926,7 +926,7 @@
     then have "False" by induct auto
   }  
   then show ?thesis
-    by (cases s') fastsimp
+    by (cases s') fastforce
 qed
 
 lemma eval_FinA: "G\<turnstile>Norm s\<midarrow>FinA a c\<rightarrow> s' = False"
@@ -938,7 +938,7 @@
     then have "False" by induct auto
   }  
   then show ?thesis
-    by (cases s') fastsimp 
+    by (cases s') fastforce 
 qed
 
 lemma eval_no_abrupt_lemma: