diff -r 102f2430cef9 -r fe05af7ec816 src/HOL/MicroJava/BV/StepMono.thy --- a/src/HOL/MicroJava/BV/StepMono.thy Tue Sep 12 19:03:13 2000 +0200 +++ b/src/HOL/MicroJava/BV/StepMono.thy Tue Sep 12 22:13:23 2000 +0200 @@ -13,7 +13,7 @@ by (auto elim: widen.elims) -lemma sup_loc_some [rulified]: +lemma sup_loc_some [rule_format]: "\ y n. (G \ b <=l y) \ n < length y \ y!n = Ok t \ (\t. b!n = Ok t \ (G \ (b!n) <=o (y!n)))" (is "?P b") proof (induct (open) ?P b) @@ -59,7 +59,7 @@ qed -lemma append_length_n [rulified]: +lemma append_length_n [rule_format]: "\n. n \ length x \ (\a b. x = a@b \ length a = n)" (is "?P x") proof (induct (open) ?P x) show "?P []" by simp @@ -78,7 +78,7 @@ fix "n'" assume s: "n = Suc n'" with l have "n' \ length ls" by simp - hence "\a b. ls = a @ b \ length a = n'" by (rule Cons [rulified]) + hence "\a b. ls = a @ b \ length a = n'" by (rule Cons [rule_format]) thus ?thesis proof elim fix a b @@ -254,7 +254,7 @@ have "length list < length (fst s2)" by (simp add: sup_state_length) hence "\a b c. (fst s2) = rev a @ b # c \ length a = length list" - by (rule rev_append_cons [rulified]) + by (rule rev_append_cons [rule_format]) thus ?thesis by - (cases s2, elim exE conjE, simp, rule that) qed