src/HOL/Integ/IntDef.thy
changeset 5562 02261e6880d1
parent 5540 0f16c3b66ab4
child 5582 a356fb49e69e
--- a/src/HOL/Integ/IntDef.thy	Fri Sep 25 13:18:07 1998 +0200
+++ b/src/HOL/Integ/IntDef.thy	Fri Sep 25 13:57:01 1998 +0200
@@ -23,7 +23,7 @@
 
 constdefs
 
-  nat        :: nat => int                                  ("$# _" [80] 80)
+  int :: nat => int                                  ("$# _" [80] 80)
   "$# m == Abs_Integ(intrel ^^ {(m,0)})"
 
   neg   :: int => bool