src/HOL/Nat.thy
changeset 20640 05e6042394b9
parent 20588 c847c56edf0c
child 20699 0cc77abb185a
--- a/src/HOL/Nat.thy	Wed Sep 20 12:23:54 2006 +0200
+++ b/src/HOL/Nat.thy	Wed Sep 20 12:24:11 2006 +0200
@@ -1062,4 +1062,18 @@
 lemma [code func]:
   "OperationalEquality.eq 0 (Suc m) = False" unfolding eq_def by auto
 
+code_typename
+  "nat" "IntDef.nat"
+
+code_constname
+  "0 \<Colon> nat" "IntDef.zero_nat"
+  "1 \<Colon> nat" "IntDef.one_nat"
+  Suc "IntDef.succ_nat"
+  "op + \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.plus_nat"
+  "op - \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.minus_nat"
+  "op * \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.times_nat"
+  "op < \<Colon> nat \<Rightarrow> nat \<Rightarrow> bool" "IntDef.less_nat"
+  "op \<le> \<Colon> nat \<Rightarrow> nat \<Rightarrow> bool" "IntDef.less_eq_nat"
+  "OperationalEquality.eq \<Colon> nat \<Rightarrow> nat \<Rightarrow> bool" "IntDef.eq_nat"
+
 end