src/HOL/Integ/IntDef.thy
changeset 20186 56207a6f4cc5
parent 20180 a751bec7cf29
child 20217 25b068a99d2b
--- a/src/HOL/Integ/IntDef.thy	Sun Jul 23 07:20:52 2006 +0200
+++ b/src/HOL/Integ/IntDef.thy	Sun Jul 23 07:21:22 2006 +0200
@@ -914,7 +914,7 @@
     ml ("IntInf.* (_, _)")
     haskell (infixl 7 "*")
   "uminus :: int \<Rightarrow> int"
-    ml (target_atom "~")
+    ml (target_atom "IntInf.~")
     haskell (target_atom "negate")
   "op = :: int \<Rightarrow> int \<Rightarrow> bool"
     ml ("(op =) (_ : IntInf.int, _)")