src/ZF/Integ/Int.thy
changeset 9570 e16e168984e1
parent 9548 15bee2731e43
child 9578 ab26d6c8ebfe
--- a/src/ZF/Integ/Int.thy	Thu Aug 10 00:45:23 2000 +0200
+++ b/src/ZF/Integ/Int.thy	Thu Aug 10 11:27:34 2000 +0200
@@ -30,7 +30,10 @@
 
   znegative   ::      i=>o
     "znegative(z) == EX x y. x<y & y:nat & <x,y>:z"
-  
+
+  iszero      ::      i=>o
+    "iszero(z) == z = $# 0"
+    
   zmagnitude  ::      i=>i
     "zmagnitude(z) ==
      THE m. m : nat & ((~ znegative(z) & z = $# m) |
@@ -62,7 +65,7 @@
      "z1 $< z2 == znegative(z1 $- z2)"
   
   zle          ::      [i,i]=>o      (infixl "$<=" 50)
-     "z1 $<= z2 == z1 $< z2 | z1=z2"
+     "z1 $<= z2 == z1 $< z2 | intify(z1)=intify(z2)"
   
 (*div and mod await definitions!*)
 consts