src/HOL/Integ/IntDef.thy
changeset 21113 5b76e541cc0a
parent 21079 747d716e98d0
child 21191 c00161fbf990
--- a/src/HOL/Integ/IntDef.thy	Tue Oct 31 09:28:55 2006 +0100
+++ b/src/HOL/Integ/IntDef.thy	Tue Oct 31 09:28:56 2006 +0100
@@ -909,14 +909,14 @@
 instance int :: eq ..
 
 code_type int
-  (SML target_atom "IntInf.int")
-  (Haskell target_atom "Integer")
+  (SML "IntInf.int")
+  (Haskell "Integer")
 
 code_instance int :: eq
   (Haskell -)
 
 code_const "Code_Generator.eq \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
-  (SML "(op =) (_ : IntInf.int, _)")
+  (SML "!((_ : IntInf.int) = _)")
   (Haskell infixl 4 "==")
 
 code_const "op <= \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
@@ -940,8 +940,8 @@
   (Haskell infixl 7 "*")
 
 code_const "uminus \<Colon> int \<Rightarrow> int"
-  (SML target_atom "IntInf.~")
-  (Haskell target_atom "negate")
+  (SML "IntInf.~")
+  (Haskell "negate")
 
 code_reserved SML IntInf
 code_reserved Haskell Integer negate