src/HOL/Lambda/WeakNorm.thy
changeset 23399 1766da98eaa9
parent 22925 86b4a7d04d43
child 23464 bc2563c37b1a
--- a/src/HOL/Lambda/WeakNorm.thy	Fri Jun 15 15:10:32 2007 +0200
+++ b/src/HOL/Lambda/WeakNorm.thy	Fri Jun 15 19:19:23 2007 +0200
@@ -575,6 +575,10 @@
   CodegenSerializer.add_undefined "SML" "arbitrary" "(raise Fail \"arbitrary\")"
 *}
 
+definition
+  int :: "nat \<Rightarrow> int" where
+  "int \<equiv> of_nat"
+
 code_gen type_NF nat int in SML
 
 ML {*
@@ -584,7 +588,7 @@
 structure Nat = ROOT.Nat;
 
 val nat_of_int = ROOT.Integer.nat o IntInf.fromInt;
-val int_of_nat = IntInf.toInt o ROOT.Integer.int;
+val int_of_nat = IntInf.toInt o ROOT.WeakNorm.int;
 
 fun dBtype_of_typ (Type ("fun", [T, U])) =
       Type.Fun (dBtype_of_typ T, dBtype_of_typ U)