src/HOL/Nat.thy
changeset 61531 ab2e862263e7
parent 61378 3e04c9ca001a
child 61649 268d88ec9087
--- a/src/HOL/Nat.thy	Thu Oct 29 15:40:52 2015 +0100
+++ b/src/HOL/Nat.thy	Mon Nov 02 11:56:28 2015 +0100
@@ -1472,6 +1472,9 @@
 lemma of_nat_mult: "of_nat (m * n) = of_nat m * of_nat n"
   by (induct m) (simp_all add: ac_simps distrib_right)
 
+lemma mult_of_nat_commute: "of_nat x * y = y * of_nat x"
+  by (induction x) (simp_all add: algebra_simps)
+
 primrec of_nat_aux :: "('a \<Rightarrow> 'a) \<Rightarrow> nat \<Rightarrow> 'a \<Rightarrow> 'a" where
   "of_nat_aux inc 0 i = i"
 | "of_nat_aux inc (Suc n) i = of_nat_aux inc n (inc i)" -- \<open>tail recursive\<close>