src/HOL/NatBin.thy
changeset 30079 293b896b9c25
parent 29958 6d84e2f9f5cf
child 30081 46b9c8ae3897
--- a/src/HOL/NatBin.thy	Mon Feb 23 13:55:36 2009 -0800
+++ b/src/HOL/NatBin.thy	Mon Feb 23 16:25:52 2009 -0800
@@ -442,19 +442,13 @@
 (* These two can be useful when m = number_of... *)
 
 lemma add_eq_if: "(m::nat) + n = (if m=0 then n else Suc ((m - 1) + n))"
-apply (case_tac "m")
-apply (simp_all add: numerals)
-done
+  unfolding One_nat_def by (cases m) simp_all
 
 lemma mult_eq_if: "(m::nat) * n = (if m=0 then 0 else n + ((m - 1) * n))"
-apply (case_tac "m")
-apply (simp_all add: numerals)
-done
+  unfolding One_nat_def by (cases m) simp_all
 
 lemma power_eq_if: "(p ^ m :: nat) = (if m=0 then 1 else p * (p ^ (m - 1)))"
-apply (case_tac "m")
-apply (simp_all add: numerals)
-done
+  unfolding One_nat_def by (cases m) simp_all
 
 
 subsection{*Comparisons involving (0::nat) *}