src/HOL/MicroJava/BV/LBVCorrect.thy
changeset 12389 23bd419144eb
parent 11085 b830bf10bf71
child 12516 d09d0f160888
--- a/src/HOL/MicroJava/BV/LBVCorrect.thy	Wed Dec 05 13:16:34 2001 +0100
+++ b/src/HOL/MicroJava/BV/LBVCorrect.thy	Wed Dec 05 14:32:10 2001 +0100
@@ -241,18 +241,18 @@
   moreover
   from pc
   obtain x xs where "is = x#xs" 
-    by (simp add: neq_Nil_conv) (elim, rule that)
+    by (auto simp add: neq_Nil_conv)
   with wtl
   obtain s' where
     "wtl_cert x G rT s cert mxs (length is) 0 = OK s'"
-    by simp (elim, rule that, simp)
+    by auto
   hence 
     "!!t. cert!0 = Some t ==> G \<turnstile> s <=' cert!0"
     by (simp add: wtl_cert_def split: if_splits)
 
   ultimately
   show ?thesis
-    by - (cases "cert!0", auto)
+    by (cases "cert!0") auto
 qed