changeset 9883 | c1c8647af477 |
parent 9654 | 9754ba005b64 |
child 9964 | 7966a2902266 |
--- a/src/ZF/Integ/Int.thy Thu Sep 07 15:31:09 2000 +0200 +++ b/src/ZF/Integ/Int.thy Thu Sep 07 17:36:37 2000 +0200 @@ -34,6 +34,14 @@ iszero :: i=>o "iszero(z) == z = $# 0" + raw_nat_of :: i => i + "raw_nat_of(z) == if znegative(z) then 0 + else (THE m. m: nat & z = int_of(m))" + + nat_of :: i => i + "nat_of(z) == raw_nat_of (intify(z))" + + (*could be replaced by an absolute value function from int to int?*) zmagnitude :: i=>i "zmagnitude(z) == THE m. m : nat & ((~ znegative(z) & z = $# m) |