diff -r 135fd6f2dadd -r d7c0aa802f0d src/HOL/MicroJava/BV/JVMType.thy --- a/src/HOL/MicroJava/BV/JVMType.thy Thu May 24 22:07:00 2012 +0200 +++ b/src/HOL/MicroJava/BV/JVMType.thy Thu May 24 22:41:27 2012 +0200 @@ -236,7 +236,7 @@ assume "G \ (x # xs) <=l b" "n < length (x # xs)" with IH show "G \ ((x # xs) ! n) <=o (b ! n)" - by - (cases n, auto) + by (cases n) auto qed qed with a @@ -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, rule that) with f have "\n. n < length ls \ (G \ (ls!n) <=o (bs!n))" @@ -289,7 +289,7 @@ assume "length (l#ls) = length (b::ty err list)" with IH show "(G \ ((l#ls)@x) <=l (b@y)) = ((G \ (l#ls) <=l b) \ (G \ x <=l y))" - by - (cases b, auto) + by (cases b) auto qed qed with l @@ -355,7 +355,7 @@ assume "G \a <=o b" "G \ (l # ls) <=l y" "n < length y" with IH show "G \ (l # ls)[n := a] <=l y[n := b]" - by - (cases n, auto simp add: sup_loc_Cons2 list_all2_Cons1) + by (cases n) (auto simp add: sup_loc_Cons2 list_all2_Cons1) qed qed @@ -433,9 +433,9 @@ proof (intro strip) fix n assume n: "n < length a" - with G + with G(1) have "G \ (a!n) <=o (b!n)" - by - (rule sup_loc_nth) + by (rule sup_loc_nth) also from n G have "G \ \ <=o (c!n)"