src/HOL/Integ/Integ.thy
changeset 5540 0f16c3b66ab4
parent 5509 c38cc427976c
child 5547 29f09a778037
--- a/src/HOL/Integ/Integ.thy	Wed Sep 23 10:17:11 1998 +0200
+++ b/src/HOL/Integ/Integ.thy	Wed Sep 23 10:25:37 1998 +0200
@@ -12,7 +12,7 @@
 instance int :: linorder (zle_linear)
 
 constdefs
-  zmagnitude  :: int => nat
-  "zmagnitude(Z) == @m. Z = $# m | -Z = $# m"
+  nat_of  :: int => nat
+  "nat_of(Z) == @m. Z = $# m | -Z = $# m"
 
 end