diff -r a34d89ce6097 -r 6616e6c53d48 src/ZF/Nat.thy --- a/src/ZF/Nat.thy Mon May 26 18:36:15 2003 +0200 +++ b/src/ZF/Nat.thy Tue May 27 11:39:03 2003 +0200 @@ -38,12 +38,13 @@ Gt :: i "Gt == {:nat*nat. y < x}" - less_than :: "i=>i" - "less_than(n) == {i:nat. ii" "greater_than(n) == {i:nat. n < i}" +text{*No need for a less-than operator: a natural number is its list of +predecessors!*} + + lemma nat_bnd_mono: "bnd_mono(Inf, %X. {0} Un {succ(i). i:X})" apply (rule bnd_monoI) apply (cut_tac infinity, blast, blast) @@ -281,6 +282,14 @@ lemma nat_nonempty [simp]: "nat ~= 0" by blast +text{*A natural number is the set of its predecessors*} +lemma nat_eq_Collect_lt: "i \ nat ==> {j\nat. j