begin
theorem Th1:
theorem Th2:
for
n being
Nat holds
n c= n + 1
theorem Th3:
:: deftheorem defines ascending DICKSON:def 1 :
for R being RelStr
for f being sequence of R holds
( f is ascending iff for n being Element of NAT holds
( f . (n + 1) <> f . n & [(f . n),(f . (n + 1))] in the InternalRel of R ) );
:: deftheorem Def2 defines weakly-ascending DICKSON:def 2 :
for R being RelStr
for f being sequence of R holds
( f is weakly-ascending iff for n being Element of NAT holds [(f . n),(f . (n + 1))] in the InternalRel of R );
theorem Th4:
theorem Th5:
theorem
canceled;
theorem Th7:
theorem Th8:
begin
:: deftheorem Def3 defines quasi_ordered DICKSON:def 3 :
for R being RelStr holds
( R is quasi_ordered iff ( R is reflexive & R is transitive ) );
:: deftheorem Def4 defines EqRel DICKSON:def 4 :
for R being RelStr st R is quasi_ordered holds
EqRel R = the InternalRel of R /\ ( the InternalRel of R ~);
theorem Th9:
definition
let R be
RelStr ;
func <=E R -> Relation of
(Class (EqRel R)) means :
Def5:
for
A,
B being
set holds
(
[A,B] in it iff ex
a,
b being
Element of
R st
(
A = Class (
(EqRel R),
a) &
B = Class (
(EqRel R),
b) &
a <= b ) );
existence
ex b1 being Relation of (Class (EqRel R)) st
for A, B being set holds
( [A,B] in b1 iff ex a, b being Element of R st
( A = Class ((EqRel R),a) & B = Class ((EqRel R),b) & a <= b ) )
uniqueness
for b1, b2 being Relation of (Class (EqRel R)) st ( for A, B being set holds
( [A,B] in b1 iff ex a, b being Element of R st
( A = Class ((EqRel R),a) & B = Class ((EqRel R),b) & a <= b ) ) ) & ( for A, B being set holds
( [A,B] in b2 iff ex a, b being Element of R st
( A = Class ((EqRel R),a) & B = Class ((EqRel R),b) & a <= b ) ) ) holds
b1 = b2
end;
:: deftheorem Def5 defines <=E DICKSON:def 5 :
for R being RelStr
for b2 being Relation of (Class (EqRel R)) holds
( b2 = <=E R iff for A, B being set holds
( [A,B] in b2 iff ex a, b being Element of R st
( A = Class ((EqRel R),a) & B = Class ((EqRel R),b) & a <= b ) ) );
theorem Th10:
theorem
:: deftheorem defines \~ DICKSON:def 6 :
for R being Relation holds R \~ = R \ (R ~);
:: deftheorem defines \~ DICKSON:def 7 :
for R being RelStr holds R \~ = RelStr(# the carrier of R,( the InternalRel of R \~) #);
theorem
theorem
theorem
theorem
theorem Th16:
theorem Th17:
begin
theorem Th18:
theorem
:: deftheorem Def8 defines min-classes DICKSON:def 8 :
for R being non empty RelStr
for N being Subset of R
for b3 being Subset-Family of R holds
( b3 = min-classes N iff for x being set holds
( x in b3 iff ex y being Element of (R \~) st
( y is_minimal_wrt N, the InternalRel of (R \~) & x = (Class ((EqRel R),y)) /\ N ) ) );
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
theorem Th24:
theorem
:: deftheorem Def9 defines is_Dickson-basis_of DICKSON:def 9 :
for R being RelStr
for N being Subset of R
for B being set holds
( B is_Dickson-basis_of N,R iff ( B c= N & ( for a being Element of R st a in N holds
ex b being Element of R st
( b in B & b <= a ) ) ) );
theorem Th26:
theorem Th27:
:: deftheorem Def10 defines Dickson DICKSON:def 10 :
for R being RelStr holds
( R is Dickson iff for N being Subset of R ex B being set st
( B is_Dickson-basis_of N,R & B is finite ) );
theorem Th28:
theorem Th29:
:: deftheorem Def11 defines mindex DICKSON:def 11 :
for f being Function
for b being set st dom f = NAT & b in rng f holds
for b3 being Element of NAT holds
( b3 = f mindex b iff ( f . b3 = b & ( for i being Element of NAT st f . i = b holds
b3 <= i ) ) );
:: deftheorem Def12 defines mindex DICKSON:def 12 :
for R being non empty 1-sorted
for f being sequence of R
for b being set
for m being Element of NAT st ex j being Element of NAT st
( m < j & f . j = b ) holds
for b5 being Element of NAT holds
( b5 = f mindex (b,m) iff ( f . b5 = b & m < b5 & ( for i being Element of NAT st m < i & f . i = b holds
b5 <= i ) ) );
theorem Th30:
theorem Th31:
theorem Th32:
theorem Th33:
theorem Th34:
theorem
:: deftheorem Def13 defines Dickson-bases DICKSON:def 13 :
for R being non empty RelStr
for N being Subset of R st R is Dickson holds
for b3 being non empty Subset-Family of R holds
( b3 = Dickson-bases (N,R) iff for B being set holds
( B in b3 iff B is_Dickson-basis_of N,R ) );
theorem Th36:
theorem Th37:
theorem Th38:
theorem Th39:
theorem Th40:
theorem Th41:
theorem Th42:
theorem Th43:
Lm1:
for p being RelStr-yielding ManySortedSet of {} holds
( not product p is empty & product p is quasi_ordered & product p is Dickson & product p is antisymmetric )
:: deftheorem defines NATOrd DICKSON:def 14 :
NATOrd = { [x,y] where x, y is Element of NAT : x <= y } ;
theorem Th44:
theorem Th45:
theorem Th46:
theorem Th47:
:: deftheorem defines OrderedNAT DICKSON:def 15 :
OrderedNAT = RelStr(# NAT,NATOrd #);
theorem
theorem Th49:
theorem