begin
Lm1:
for R being Relation holds
( R is reflexive iff for x being set st x in field R holds
[x,x] in R )
Lm2:
for R being Relation holds
( R is transitive iff for x, y, z being set st [x,y] in R & [y,z] in R holds
[x,z] in R )
Lm3:
for R being Relation holds
( R is antisymmetric iff for x, y being set st [x,y] in R & [y,x] in R holds
x = y )
Lm4:
for R being Relation holds
( R is connected iff for x, y being set st x in field R & y in field R & x <> y & not [x,y] in R holds
[y,x] in R )
:: deftheorem defines -Seg WELLORD1:def 1 :
for R being Relation
for a being set holds R -Seg a = (Coim (R,a)) \ {a};
theorem Th1:
theorem Th2:
:: deftheorem Def2 defines well_founded WELLORD1:def 2 :
for R being Relation holds
( R is well_founded iff for Y being set st Y c= field R & Y <> {} holds
ex a being set st
( a in Y & R -Seg a misses Y ) );
:: deftheorem Def3 defines is_well_founded_in WELLORD1:def 3 :
for R being Relation
for X being set holds
( R is_well_founded_in X iff for Y being set st Y c= X & Y <> {} holds
ex a being set st
( a in Y & R -Seg a misses Y ) );
theorem
canceled;
theorem
canceled;
theorem Th5:
:: deftheorem Def4 defines well-ordering WELLORD1:def 4 :
for R being Relation holds
( R is well-ordering iff ( R is reflexive & R is transitive & R is antisymmetric & R is connected & R is well_founded ) );
:: deftheorem Def5 defines well_orders WELLORD1:def 5 :
for R being Relation
for X being set holds
( R well_orders X iff ( R is_reflexive_in X & R is_transitive_in X & R is_antisymmetric_in X & R is_connected_in X & R is_well_founded_in X ) );
theorem
canceled;
theorem
canceled;
theorem
theorem
theorem Th10:
theorem
theorem
theorem Th13:
:: deftheorem defines |_2 WELLORD1:def 6 :
for R being Relation
for Y being set holds R |_2 Y = R /\ [:Y,Y:];
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th17:
theorem Th18:
Lm5:
for X being set
for R being Relation holds dom (X | R) c= dom R
theorem Th19:
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
theorem Th24:
theorem Th25:
theorem Th26:
theorem
theorem
theorem Th29:
theorem Th30:
theorem Th31:
theorem Th32:
theorem Th33:
theorem
canceled;
theorem Th35:
theorem Th36:
theorem Th37:
theorem Th38:
theorem Th39:
theorem Th40:
theorem Th41:
theorem Th42:
theorem Th43:
:: deftheorem Def7 defines is_isomorphism_of WELLORD1:def 7 :
for R, S being Relation
for F being Function holds
( F is_isomorphism_of R,S iff ( dom F = field R & rng F = field S & F is one-to-one & ( for a, b being set holds
( [a,b] in R iff ( a in field R & b in field R & [(F . a),(F . b)] in S ) ) ) ) );
theorem
canceled;
theorem Th45:
:: deftheorem Def8 defines are_isomorphic WELLORD1:def 8 :
for R, S being Relation holds
( R,S are_isomorphic iff ex F being Function st F is_isomorphism_of R,S );
theorem
canceled;
theorem Th47:
theorem
theorem Th49:
theorem Th50:
theorem Th51:
theorem Th52:
theorem Th53:
theorem Th54:
theorem Th55:
definition
let R,
S be
Relation;
assume that A1:
R is
well-ordering
and A2:
R,
S are_isomorphic
;
func canonical_isomorphism_of (
R,
S)
-> Function means :
Def9:
it is_isomorphism_of R,
S;
existence
ex b1 being Function st b1 is_isomorphism_of R,S
by A2, Def8;
uniqueness
for b1, b2 being Function st b1 is_isomorphism_of R,S & b2 is_isomorphism_of R,S holds
b1 = b2
by A1, Th55;
end;
:: deftheorem Def9 defines canonical_isomorphism_of WELLORD1:def 9 :
for R, S being Relation st R is well-ordering & R,S are_isomorphic holds
for b3 being Function holds
( b3 = canonical_isomorphism_of (R,S) iff b3 is_isomorphism_of R,S );
theorem
canceled;
theorem Th57:
theorem Th58:
theorem Th59:
theorem Th60:
theorem Th61:
theorem Th62:
theorem Th63:
theorem
theorem