src/HOL/Integ/IntArith.thy
changeset 21191 c00161fbf990
parent 21113 5b76e541cc0a
child 21820 2f2b6a965ccc
--- a/src/HOL/Integ/IntArith.thy	Mon Nov 06 16:28:30 2006 +0100
+++ b/src/HOL/Integ/IntArith.thy	Mon Nov 06 16:28:31 2006 +0100
@@ -364,20 +364,8 @@
 
 subsection {* code generator setup *}
 
-code_typename
-  "Numeral.bit" "IntDef.bit"
-
-code_constname
-  "number_of \<Colon> int \<Rightarrow> int" "IntDef.number_of"
-  "Numeral.pred" "IntDef.pred"
-  "Numeral.succ" "IntDef.succ"
-  "Numeral.Pls" "IntDef.pls"
-  "Numeral.Min" "IntDef.min"
-  "Numeral.Bit" "IntDef.bit"
-  "Numeral.bit.bit_case" "IntDef.bit_case"
-  "Code_Generator.eq \<Colon> bit \<Rightarrow> bit \<Rightarrow> bool" "IntDef.eq_bit"
-  "Numeral.B0" "IntDef.b0"
-  "Numeral.B1" "IntDef.b1"
+code_modulename SML
+  Numeral Integer
 
 lemma Numeral_Pls_refl [code func]:
   "Numeral.Pls = Numeral.Pls" ..