begin
:: deftheorem defines InclPoset YELLOW_1:def 1 :
for X being set holds InclPoset X = RelStr(# X,(RelIncl X) #);
theorem
:: deftheorem defines BoolePoset YELLOW_1:def 2 :
for X being set holds BoolePoset X = LattPOSet (BooleLatt X);
theorem Th2:
theorem Th3:
theorem Th4:
theorem
theorem
theorem
theorem Th8:
theorem Th9:
theorem
theorem
theorem
theorem Th13:
theorem Th14:
theorem
theorem
Lm1:
for X being set
for x, y being Element of (BoolePoset X) holds
( x /\ y in bool X & x \/ y in bool X )
theorem
theorem
theorem
theorem
theorem
theorem
theorem
Lm2:
for T being non empty TopSpace holds InclPoset the topology of T is lower-bounded
theorem
Lm3:
for T being non empty TopSpace holds InclPoset the topology of T is complete
Lm4:
for T being non empty TopSpace holds not InclPoset the topology of T is trivial
theorem
begin
:: deftheorem Def3 defines RelStr-yielding YELLOW_1:def 3 :
for R being Relation holds
( R is RelStr-yielding iff for v being set st v in rng R holds
v is RelStr );
definition
let I be
set ;
let J be
RelStr-yielding ManySortedSet of
I;
func product J -> strict RelStr means :
Def4:
( the
carrier of
it = product (Carrier J) & ( for
x,
y being
Element of
it st
x in product (Carrier J) holds
(
x <= y iff ex
f,
g being
Function st
(
f = x &
g = y & ( for
i being
set st
i in I holds
ex
R being
RelStr ex
xi,
yi being
Element of
R st
(
R = J . i &
xi = f . i &
yi = g . i &
xi <= yi ) ) ) ) ) );
existence
ex b1 being strict RelStr st
( the carrier of b1 = product (Carrier J) & ( for x, y being Element of b1 st x in product (Carrier J) holds
( x <= y iff ex f, g being Function st
( f = x & g = y & ( for i being set st i in I holds
ex R being RelStr ex xi, yi being Element of R st
( R = J . i & xi = f . i & yi = g . i & xi <= yi ) ) ) ) ) )
uniqueness
for b1, b2 being strict RelStr st the carrier of b1 = product (Carrier J) & ( for x, y being Element of b1 st x in product (Carrier J) holds
( x <= y iff ex f, g being Function st
( f = x & g = y & ( for i being set st i in I holds
ex R being RelStr ex xi, yi being Element of R st
( R = J . i & xi = f . i & yi = g . i & xi <= yi ) ) ) ) ) & the carrier of b2 = product (Carrier J) & ( for x, y being Element of b2 st x in product (Carrier J) holds
( x <= y iff ex f, g being Function st
( f = x & g = y & ( for i being set st i in I holds
ex R being RelStr ex xi, yi being Element of R st
( R = J . i & xi = f . i & yi = g . i & xi <= yi ) ) ) ) ) holds
b1 = b2
end;
:: deftheorem Def4 defines product YELLOW_1:def 4 :
for I being set
for J being RelStr-yielding ManySortedSet of I
for b3 being strict RelStr holds
( b3 = product J iff ( the carrier of b3 = product (Carrier J) & ( for x, y being Element of b3 st x in product (Carrier J) holds
( x <= y iff ex f, g being Function st
( f = x & g = y & ( for i being set st i in I holds
ex R being RelStr ex xi, yi being Element of R st
( R = J . i & xi = f . i & yi = g . i & xi <= yi ) ) ) ) ) ) );
:: deftheorem defines |^ YELLOW_1:def 5 :
for I being set
for T being RelStr holds T |^ I = product (I --> T);
theorem Th26:
theorem
theorem Th28:
Lm5:
for X being set
for Y being non empty RelStr
for x being Element of (Y |^ X) holds
( x in the carrier of (product (X --> Y)) & x is Function of X, the carrier of Y )
definition
let S,
T be
RelStr ;
func MonMaps (
S,
T)
-> strict full SubRelStr of
T |^ the
carrier of
S means
for
f being
Function of
S,
T holds
(
f in the
carrier of
it iff (
f in Funcs ( the
carrier of
S, the
carrier of
T) &
f is
monotone ) );
existence
ex b1 being strict full SubRelStr of T |^ the carrier of S st
for f being Function of S,T holds
( f in the carrier of b1 iff ( f in Funcs ( the carrier of S, the carrier of T) & f is monotone ) )
uniqueness
for b1, b2 being strict full SubRelStr of T |^ the carrier of S st ( for f being Function of S,T holds
( f in the carrier of b1 iff ( f in Funcs ( the carrier of S, the carrier of T) & f is monotone ) ) ) & ( for f being Function of S,T holds
( f in the carrier of b2 iff ( f in Funcs ( the carrier of S, the carrier of T) & f is monotone ) ) ) holds
b1 = b2
end;
:: deftheorem defines MonMaps YELLOW_1:def 6 :
for S, T being RelStr
for b3 being strict full SubRelStr of T |^ the carrier of S holds
( b3 = MonMaps (S,T) iff for f being Function of S,T holds
( f in the carrier of b3 iff ( f in Funcs ( the carrier of S, the carrier of T) & f is monotone ) ) );