author | berghofe |
Mon, 21 Jan 2002 14:43:38 +0100 | |
changeset 12822 | 073116d65bb9 |
parent 12114 | a8e860c86252 |
child 13155 | dcbf6cb95534 |
permissions | -rw-r--r-- |
1478 | 1 |
(* Title: ZF/Ordinal.thy |
435 | 2 |
ID: $Id$ |
1478 | 3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
435 | 4 |
Copyright 1994 University of Cambridge |
5 |
||
6 |
Ordinals in Zermelo-Fraenkel Set Theory |
|
7 |
*) |
|
8 |
||
2469 | 9 |
Ordinal = WF + Bool + equalities + |
435 | 10 |
consts |
1478 | 11 |
Memrel :: i=>i |
1401 | 12 |
Transset,Ord :: i=>o |
13 |
"<" :: [i,i] => o (infixl 50) (*less than on ordinals*) |
|
2539 | 14 |
Limit :: i=>o |
15 |
||
16 |
syntax |
|
1401 | 17 |
"le" :: [i,i] => o (infixl 50) (*less than or equals*) |
435 | 18 |
|
19 |
translations |
|
20 |
"x le y" == "x < succ(y)" |
|
21 |
||
12114
a8e860c86252
eliminated old "symbols" syntax, use "xsymbols" instead;
wenzelm
parents:
2540
diff
changeset
|
22 |
syntax (xsymbols) |
2540 | 23 |
"op le" :: [i,i] => o (infixl "\\<le>" 50) (*less than or equals*) |
24 |
||
753 | 25 |
defs |
1478 | 26 |
Memrel_def "Memrel(A) == {z: A*A . EX x y. z=<x,y> & x:y }" |
27 |
Transset_def "Transset(i) == ALL x:i. x<=i" |
|
28 |
Ord_def "Ord(i) == Transset(i) & (ALL x:i. Transset(x))" |
|
435 | 29 |
lt_def "i<j == i:j & Ord(j)" |
30 |
Limit_def "Limit(i) == Ord(i) & 0<i & (ALL y. y<i --> succ(y)<i)" |
|
31 |
||
32 |
end |