src/HOL/Nat.thy
changeset 55424 9ab4129a76a3
parent 55423 07dea66779f3
child 55443 3def821deb70
--- a/src/HOL/Nat.thy	Wed Feb 12 08:37:28 2014 +0100
+++ b/src/HOL/Nat.thy	Wed Feb 12 08:37:28 2014 +0100
@@ -119,6 +119,8 @@
 abbreviation rec_nat :: "'a \<Rightarrow> (nat \<Rightarrow> 'a \<Rightarrow> 'a) \<Rightarrow> nat \<Rightarrow> 'a" where
   "rec_nat \<equiv> old.rec_nat"
 
+declare nat.sel[code del]
+
 hide_const Nat.pred -- {* hide everything related to the selector *}
 hide_fact
   nat.case_eq_if
@@ -1943,13 +1945,13 @@
 qed
 
 
-subsection {* aliasses *}
+subsection {* aliases *}
 
 lemma nat_mult_1: "(1::nat) * n = n"
-  by simp
+  by (rule mult_1_left)
  
 lemma nat_mult_1_right: "n * (1::nat) = n"
-  by simp
+  by (rule mult_1_right)
 
 
 subsection {* size of a datatype value *}