src/HOL/UNITY/Comp/AllocBase.thy
changeset 46911 6d2a2f0e904e
parent 45827 66c68453455c
child 57418 6ab1c7cb0b8d
--- a/src/HOL/UNITY/Comp/AllocBase.thy	Tue Mar 13 21:17:37 2012 +0100
+++ b/src/HOL/UNITY/Comp/AllocBase.thy	Tue Mar 13 22:49:02 2012 +0100
@@ -27,11 +27,8 @@
 apply (auto simp add: lessThan_Suc)
 done
 
-lemma tokens_mono_prefix [rule_format]:
-     "ALL xs. xs <= ys --> tokens xs <= tokens ys"
-apply (induct_tac "ys")
-apply (auto simp add: prefix_Cons)
-done
+lemma tokens_mono_prefix: "xs <= ys ==> tokens xs <= tokens ys"
+  by (induct ys arbitrary: xs) (auto simp add: prefix_Cons)
 
 lemma mono_tokens: "mono tokens"
 apply (unfold mono_def)
@@ -42,9 +39,7 @@
 (** bag_of **)
 
 lemma bag_of_append [simp]: "bag_of (l@l') = bag_of l + bag_of l'"
-apply (induct_tac "l", simp)
- apply (simp add: add_ac)
-done
+  by (induct l) (simp_all add: add_ac)
 
 lemma mono_bag_of: "mono (bag_of :: 'a list => ('a::order) multiset)"
 apply (rule monoI)