begin
:: deftheorem Def1 defines uncurrying WAYBEL27:def 1 :
for F being Function holds
( F is uncurrying iff ( ( for x being set st x in dom F holds
x is Function-yielding Function ) & ( for f being Function st f in dom F holds
F . f = uncurry f ) ) );
:: deftheorem Def2 defines currying WAYBEL27:def 2 :
for F being Function holds
( F is currying iff ( ( for x being set st x in dom F holds
( x is Function & proj1 x is Relation ) ) & ( for f being Function st f in dom F holds
F . f = curry f ) ) );
:: deftheorem Def3 defines commuting WAYBEL27:def 3 :
for F being Function holds
( F is commuting iff ( ( for x being set st x in dom F holds
x is Function-yielding Function ) & ( for f being Function st f in dom F holds
F . f = commute f ) ) );
theorem Th1:
theorem Th2:
registration
let X,
Y,
Z be
set ;
cluster Relation-like Funcs (
X,
(Funcs (Y,Z)))
-defined Function-like V24(
Funcs (
X,
(Funcs (Y,Z))))
uncurrying set ;
existence
ex b1 being ManySortedSet of Funcs (X,(Funcs (Y,Z))) st b1 is uncurrying
cluster Relation-like Funcs (
[:X,Y:],
Z)
-defined Function-like V24(
Funcs (
[:X,Y:],
Z))
currying set ;
existence
ex b1 being ManySortedSet of Funcs ([:X,Y:],Z) st b1 is currying
end;
theorem Th3:
theorem Th4:
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
theorem Th9:
theorem Th10:
theorem
theorem Th12:
theorem Th13:
begin
theorem Th14:
theorem Th15:
theorem
theorem Th17:
theorem Th18:
theorem Th19:
theorem Th20:
theorem Th21:
begin
:: deftheorem Def4 defines UPS WAYBEL27:def 4 :
for S being non empty RelStr
for T being non empty reflexive antisymmetric RelStr
for b3 being strict RelStr holds
( b3 = UPS (S,T) iff ( b3 is full SubRelStr of T |^ the carrier of S & ( for x being set holds
( x in the carrier of b3 iff x is directed-sups-preserving Function of S,T ) ) ) );
theorem Th22:
theorem Th23:
theorem Th24:
theorem Th25:
theorem Th26:
theorem Th27:
definition
let S1,
S2,
T1,
T2 be non
empty reflexive antisymmetric RelStr ;
let f be
Function of
S1,
S2;
assume A1:
f is
directed-sups-preserving
;
let g be
Function of
T1,
T2;
assume A2:
g is
directed-sups-preserving
;
func UPS (
f,
g)
-> Function of
(UPS (S2,T1)),
(UPS (S1,T2)) means :
Def5:
for
h being
directed-sups-preserving Function of
S2,
T1 holds
it . h = (g * h) * f;
existence
ex b1 being Function of (UPS (S2,T1)),(UPS (S1,T2)) st
for h being directed-sups-preserving Function of S2,T1 holds b1 . h = (g * h) * f
uniqueness
for b1, b2 being Function of (UPS (S2,T1)),(UPS (S1,T2)) st ( for h being directed-sups-preserving Function of S2,T1 holds b1 . h = (g * h) * f ) & ( for h being directed-sups-preserving Function of S2,T1 holds b2 . h = (g * h) * f ) holds
b1 = b2
end;
:: deftheorem Def5 defines UPS WAYBEL27:def 5 :
for S1, S2, T1, T2 being non empty reflexive antisymmetric RelStr
for f being Function of S1,S2 st f is directed-sups-preserving holds
for g being Function of T1,T2 st g is directed-sups-preserving holds
for b7 being Function of (UPS (S2,T1)),(UPS (S1,T2)) holds
( b7 = UPS (f,g) iff for h being directed-sups-preserving Function of S2,T1 holds b7 . h = (g * h) * f );
theorem Th28:
for
S1,
S2,
S3,
T1,
T2,
T3 being non
empty Poset for
f1 being
directed-sups-preserving Function of
S2,
S3 for
f2 being
directed-sups-preserving Function of
S1,
S2 for
g1 being
directed-sups-preserving Function of
T1,
T2 for
g2 being
directed-sups-preserving Function of
T2,
T3 holds
(UPS (f2,g2)) * (UPS (f1,g1)) = UPS (
(f1 * f2),
(g2 * g1))
theorem Th29:
theorem Th30:
theorem Th31:
theorem
theorem Th33:
theorem Th34:
theorem Th35:
theorem Th36:
theorem Th37:
Lm1:
now
let M be non
empty set ;
for X, Y being non empty Poset
for f being directed-sups-preserving Function of X,(Y |^ M) holds
( f in Funcs ( the carrier of X,(Funcs (M, the carrier of Y))) & rng (commute f) c= Funcs ( the carrier of X, the carrier of Y) & dom (commute f) = M )let X,
Y be non
empty Poset;
for f being directed-sups-preserving Function of X,(Y |^ M) holds
( f in Funcs ( the carrier of X,(Funcs (M, the carrier of Y))) & rng (commute f) c= Funcs ( the carrier of X, the carrier of Y) & dom (commute f) = M )let f be
directed-sups-preserving Function of
X,
(Y |^ M);
( f in Funcs ( the carrier of X,(Funcs (M, the carrier of Y))) & rng (commute f) c= Funcs ( the carrier of X, the carrier of Y) & dom (commute f) = M )
the
carrier of
(Y |^ M) = Funcs (
M, the
carrier of
Y)
by YELLOW_1:28;
then A1:
rng f c= Funcs (
M, the
carrier of
Y)
;
dom f = the
carrier of
X
by FUNCT_2:def 1;
hence
f in Funcs ( the
carrier of
X,
(Funcs (M, the carrier of Y)))
by A1, FUNCT_2:def 2;
( rng (commute f) c= Funcs ( the carrier of X, the carrier of Y) & dom (commute f) = M )then
commute f in Funcs (
M,
(Funcs ( the carrier of X, the carrier of Y)))
by FUNCT_6:85;
then
ex
g being
Function st
(
commute f = g &
dom g = M &
rng g c= Funcs ( the
carrier of
X, the
carrier of
Y) )
by FUNCT_2:def 2;
hence
(
rng (commute f) c= Funcs ( the
carrier of
X, the
carrier of
Y) &
dom (commute f) = M )
;
verum
end;
theorem Th38:
theorem Th39:
theorem Th40:
theorem Th41:
theorem Th42:
theorem
theorem
theorem Th45:
theorem Th46:
theorem