src/HOL/MicroJava/BV/JVMType.thy
changeset 56073 29e308b56d23
parent 55524 f41ef840f09d
child 58860 fee7cfa69c50
--- a/src/HOL/MicroJava/BV/JVMType.thy	Wed Mar 12 22:57:50 2014 +0100
+++ b/src/HOL/MicroJava/BV/JVMType.thy	Thu Mar 13 07:07:07 2014 +0100
@@ -258,7 +258,7 @@
     assume l: "length (l#ls) = length b"
     
     then obtain b' bs where b: "b = b'#bs"
-      by (cases b) (simp, simp add: neq_Nil_conv, rule that)
+      by (cases b) (simp, simp add: neq_Nil_conv)
 
     with f
     have "\<forall>n. n < length ls \<longrightarrow> (G \<turnstile> (ls!n) <=o (bs!n))"