begin
:: deftheorem Def1 defines directed WAYBEL_0:def 1 :
for L being RelStr
for X being Subset of L holds
( X is directed iff for x, y being Element of L st x in X & y in X holds
ex z being Element of L st
( z in X & x <= z & y <= z ) );
:: deftheorem Def2 defines filtered WAYBEL_0:def 2 :
for L being RelStr
for X being Subset of L holds
( X is filtered iff for x, y being Element of L st x in X & y in X holds
ex z being Element of L st
( z in X & z <= x & z <= y ) );
theorem Th1:
theorem Th2:
theorem Th3:
theorem
theorem Th5:
:: deftheorem Def3 defines filtered-infs-inheriting WAYBEL_0:def 3 :
for L being non empty RelStr
for S being SubRelStr of L holds
( S is filtered-infs-inheriting iff for X being filtered Subset of S st X <> {} & ex_inf_of X,L holds
"/\" (X,L) in the carrier of S );
:: deftheorem Def4 defines directed-sups-inheriting WAYBEL_0:def 4 :
for L being non empty RelStr
for S being SubRelStr of L holds
( S is directed-sups-inheriting iff for X being directed Subset of S st X <> {} & ex_sup_of X,L holds
"\/" (X,L) in the carrier of S );
theorem
theorem
begin
:: deftheorem defines antitone WAYBEL_0:def 5 :
for L1, L2 being RelStr
for f being Function of L1,L2 holds
( f is antitone iff for x, y being Element of L1 st x <= y holds
for a, b being Element of L2 st a = f . x & b = f . y holds
a >= b );
:: deftheorem Def6 defines directed WAYBEL_0:def 6 :
for N being RelStr holds
( N is directed iff [#] N is directed );
:: deftheorem defines netmap WAYBEL_0:def 7 :
for L being non empty 1-sorted
for N being non empty NetStr of L holds netmap (N,L) = the mapping of N;
:: deftheorem defines . WAYBEL_0:def 8 :
for L being non empty 1-sorted
for N being non empty NetStr of L
for i being Element of N holds N . i = the mapping of N . i;
:: deftheorem defines monotone WAYBEL_0:def 9 :
for L being non empty RelStr
for N being non empty NetStr of L holds
( N is monotone iff netmap (N,L) is monotone );
:: deftheorem defines antitone WAYBEL_0:def 10 :
for L being non empty RelStr
for N being non empty NetStr of L holds
( N is antitone iff netmap (N,L) is antitone );
:: deftheorem Def11 defines is_eventually_in WAYBEL_0:def 11 :
for L being non empty 1-sorted
for N being non empty NetStr of L
for X being set holds
( N is_eventually_in X iff ex i being Element of N st
for j being Element of N st i <= j holds
N . j in X );
:: deftheorem defines is_often_in WAYBEL_0:def 12 :
for L being non empty 1-sorted
for N being non empty NetStr of L
for X being set holds
( N is_often_in X iff for i being Element of N ex j being Element of N st
( i <= j & N . j in X ) );
theorem
theorem
theorem
:: deftheorem Def13 defines eventually-directed WAYBEL_0:def 13 :
for L being non empty RelStr
for N being non empty NetStr of L holds
( N is eventually-directed iff for i being Element of N holds N is_eventually_in { (N . j) where j is Element of N : N . i <= N . j } );
:: deftheorem Def14 defines eventually-filtered WAYBEL_0:def 14 :
for L being non empty RelStr
for N being non empty NetStr of L holds
( N is eventually-filtered iff for i being Element of N holds N is_eventually_in { (N . j) where j is Element of N : N . i >= N . j } );
theorem Th11:
theorem Th12:
begin
:: deftheorem Def15 defines downarrow WAYBEL_0:def 15 :
for L being RelStr
for X, b3 being Subset of L holds
( b3 = downarrow X iff for x being Element of L holds
( x in b3 iff ex y being Element of L st
( y >= x & y in X ) ) );
:: deftheorem Def16 defines uparrow WAYBEL_0:def 16 :
for L being RelStr
for X, b3 being Subset of L holds
( b3 = uparrow X iff for x being Element of L holds
( x in b3 iff ex y being Element of L st
( y <= x & y in X ) ) );
theorem Th13:
theorem Th14:
theorem Th15:
theorem Th16:
:: deftheorem defines downarrow WAYBEL_0:def 17 :
for L being non empty RelStr
for x being Element of L holds downarrow x = downarrow {x};
:: deftheorem defines uparrow WAYBEL_0:def 18 :
for L being non empty RelStr
for x being Element of L holds uparrow x = uparrow {x};
theorem Th17:
theorem Th18:
theorem
theorem
theorem Th21:
theorem Th22:
:: deftheorem Def19 defines lower WAYBEL_0:def 19 :
for L being RelStr
for X being Subset of L holds
( X is lower iff for x, y being Element of L st x in X & y <= x holds
y in X );
:: deftheorem Def20 defines upper WAYBEL_0:def 20 :
for L being RelStr
for X being Subset of L holds
( X is upper iff for x, y being Element of L st x in X & x <= y holds
y in X );
theorem Th23:
theorem Th24:
theorem
theorem
theorem Th27:
theorem
theorem Th29:
theorem Th30:
theorem Th31:
theorem Th32:
theorem Th33:
theorem
theorem Th35:
theorem Th36:
theorem Th37:
theorem Th38:
theorem
begin
theorem Th40:
theorem Th41:
theorem Th42:
theorem Th43:
theorem
theorem
theorem
theorem
:: deftheorem defines principal WAYBEL_0:def 21 :
for L being non empty reflexive transitive RelStr
for I being Ideal of L holds
( I is principal iff ex x being Element of L st
( x in I & x is_>=_than I ) );
:: deftheorem defines principal WAYBEL_0:def 22 :
for L being non empty reflexive transitive RelStr
for F being Filter of L holds
( F is principal iff ex x being Element of L st
( x in F & x is_<=_than F ) );
theorem
theorem
:: deftheorem defines Ids WAYBEL_0:def 23 :
for L being non empty reflexive transitive RelStr holds Ids L = { X where X is Ideal of L : verum } ;
:: deftheorem defines Filt WAYBEL_0:def 24 :
for L being non empty reflexive transitive RelStr holds Filt L = { X where X is Filter of L : verum } ;
:: deftheorem defines Ids_0 WAYBEL_0:def 25 :
for L being non empty reflexive transitive RelStr holds Ids_0 L = (Ids L) \/ {{}};
:: deftheorem defines Filt_0 WAYBEL_0:def 26 :
for L being non empty reflexive transitive RelStr holds Filt_0 L = (Filt L) \/ {{}};
definition
let L be non
empty RelStr ;
let X be
Subset of
L;
set D =
{ ("\/" (Y,L)) where Y is finite Subset of X : ex_sup_of Y,L } ;
A1:
{ ("\/" (Y,L)) where Y is finite Subset of X : ex_sup_of Y,L } c= the
carrier of
L
func finsups X -> Subset of
L equals
{ ("\/" (Y,L)) where Y is finite Subset of X : ex_sup_of Y,L } ;
correctness
coherence
{ ("\/" (Y,L)) where Y is finite Subset of X : ex_sup_of Y,L } is Subset of L;
by A1;
set D =
{ ("/\" (Y,L)) where Y is finite Subset of X : ex_inf_of Y,L } ;
A2:
{ ("/\" (Y,L)) where Y is finite Subset of X : ex_inf_of Y,L } c= the
carrier of
L
func fininfs X -> Subset of
L equals
{ ("/\" (Y,L)) where Y is finite Subset of X : ex_inf_of Y,L } ;
correctness
coherence
{ ("/\" (Y,L)) where Y is finite Subset of X : ex_inf_of Y,L } is Subset of L;
by A2;
end;
:: deftheorem defines finsups WAYBEL_0:def 27 :
for L being non empty RelStr
for X being Subset of L holds finsups X = { ("\/" (Y,L)) where Y is finite Subset of X : ex_sup_of Y,L } ;
:: deftheorem defines fininfs WAYBEL_0:def 28 :
for L being non empty RelStr
for X being Subset of L holds fininfs X = { ("/\" (Y,L)) where Y is finite Subset of X : ex_inf_of Y,L } ;
theorem Th50:
theorem Th51:
theorem Th52:
theorem Th53:
theorem Th54:
theorem
theorem Th56:
theorem Th57:
theorem Th58:
theorem Th59:
theorem
theorem
theorem
begin
:: deftheorem Def29 defines connected WAYBEL_0:def 29 :
for L being non empty RelStr holds
( L is connected iff for x, y being Element of L holds
( x <= y or y <= x ) );
begin
theorem
theorem
begin
:: deftheorem Def30 defines preserves_inf_of WAYBEL_0:def 30 :
for S, T being non empty RelStr
for f being Function of S,T
for X being Subset of S holds
( f preserves_inf_of X iff ( ex_inf_of X,S implies ( ex_inf_of f .: X,T & inf (f .: X) = f . (inf X) ) ) );
:: deftheorem Def31 defines preserves_sup_of WAYBEL_0:def 31 :
for S, T being non empty RelStr
for f being Function of S,T
for X being Subset of S holds
( f preserves_sup_of X iff ( ex_sup_of X,S implies ( ex_sup_of f .: X,T & sup (f .: X) = f . (sup X) ) ) );
theorem
:: deftheorem defines infs-preserving WAYBEL_0:def 32 :
for L1, L2 being non empty RelStr
for f being Function of L1,L2 holds
( f is infs-preserving iff for X being Subset of L1 holds f preserves_inf_of X );
:: deftheorem defines sups-preserving WAYBEL_0:def 33 :
for L1, L2 being non empty RelStr
for f being Function of L1,L2 holds
( f is sups-preserving iff for X being Subset of L1 holds f preserves_sup_of X );
:: deftheorem defines meet-preserving WAYBEL_0:def 34 :
for L1, L2 being non empty RelStr
for f being Function of L1,L2 holds
( f is meet-preserving iff for x, y being Element of L1 holds f preserves_inf_of {x,y} );
:: deftheorem defines join-preserving WAYBEL_0:def 35 :
for L1, L2 being non empty RelStr
for f being Function of L1,L2 holds
( f is join-preserving iff for x, y being Element of L1 holds f preserves_sup_of {x,y} );
:: deftheorem defines filtered-infs-preserving WAYBEL_0:def 36 :
for L1, L2 being non empty RelStr
for f being Function of L1,L2 holds
( f is filtered-infs-preserving iff for X being Subset of L1 st not X is empty & X is filtered holds
f preserves_inf_of X );
:: deftheorem defines directed-sups-preserving WAYBEL_0:def 37 :
for L1, L2 being non empty RelStr
for f being Function of L1,L2 holds
( f is directed-sups-preserving iff for X being Subset of L1 st not X is empty & X is directed holds
f preserves_sup_of X );
:: deftheorem Def38 defines isomorphic WAYBEL_0:def 38 :
for S, T being RelStr
for f being Function of S,T holds
( ( not S is empty & not T is empty implies ( f is isomorphic iff ( f is one-to-one & f is monotone & ex g being Function of T,S st
( g = f " & g is monotone ) ) ) ) & ( ( S is empty or T is empty ) implies ( f is isomorphic iff ( S is empty & T is empty ) ) ) );
theorem Th66:
theorem
theorem
theorem Th69:
theorem
theorem
theorem Th72:
theorem
theorem
begin
:: deftheorem Def39 defines up-complete WAYBEL_0:def 39 :
for L being non empty reflexive RelStr holds
( L is up-complete iff for X being non empty directed Subset of L ex x being Element of L st
( x is_>=_than X & ( for y being Element of L st y is_>=_than X holds
x <= y ) ) );
theorem
:: deftheorem Def40 defines /\-complete WAYBEL_0:def 40 :
for L being non empty reflexive RelStr holds
( L is /\-complete iff for X being non empty Subset of L ex x being Element of L st
( x is_<=_than X & ( for y being Element of L st y is_<=_than X holds
x >= y ) ) );
theorem Th76: