definition
let A be
set ;
existence
ex b1 being BinOp of (Funcs (A,COMPLEX)) st
for f, g being Element of Funcs (A,COMPLEX) holds b1 . (f,g) = addcomplex .: (f,g)
uniqueness
for b1, b2 being BinOp of (Funcs (A,COMPLEX)) st ( for f, g being Element of Funcs (A,COMPLEX) holds b1 . (f,g) = addcomplex .: (f,g) ) & ( for f, g being Element of Funcs (A,COMPLEX) holds b2 . (f,g) = addcomplex .: (f,g) ) holds
b1 = b2
end;
definition
let A be
set ;
existence
ex b1 being BinOp of (Funcs (A,COMPLEX)) st
for f, g being Element of Funcs (A,COMPLEX) holds b1 . (f,g) = multcomplex .: (f,g)
uniqueness
for b1, b2 being BinOp of (Funcs (A,COMPLEX)) st ( for f, g being Element of Funcs (A,COMPLEX) holds b1 . (f,g) = multcomplex .: (f,g) ) & ( for f, g being Element of Funcs (A,COMPLEX) holds b2 . (f,g) = multcomplex .: (f,g) ) holds
b1 = b2
end;
definition
let A be non
empty set ;
existence
ex b1 being Function of [:COMPLEX,(Funcs (A,COMPLEX)):],(Funcs (A,COMPLEX)) st
for z being Complex
for f being Element of Funcs (A,COMPLEX)
for x being Element of A holds (b1 . [z,f]) . x = z * (f . x)
uniqueness
for b1, b2 being Function of [:COMPLEX,(Funcs (A,COMPLEX)):],(Funcs (A,COMPLEX)) st ( for z being Complex
for f being Element of Funcs (A,COMPLEX)
for x being Element of A holds (b1 . [z,f]) . x = z * (f . x) ) & ( for z being Complex
for f being Element of Funcs (A,COMPLEX)
for x being Element of A holds (b2 . [z,f]) . x = z * (f . x) ) holds
b1 = b2
end;
Lm1:
for A, B being non empty set
for x being Element of A
for f being Function of A,B holds x in dom f
Lm2:
for A being non empty set
for f, g being Element of Funcs (A,COMPLEX)
for a being Complex holds (ComplexFuncAdd A) . (((ComplexFuncExtMult A) . [a,f]),((ComplexFuncExtMult A) . [a,g])) = (ComplexFuncExtMult A) . [a,((ComplexFuncAdd A) . (f,g))]
theorem Th22:
for
x1,
x2 being
set for
A being non
empty set st
A = {x1,x2} &
x1 <> x2 holds
ex
f,
g being
Element of
Funcs (
A,
COMPLEX) st
( ( for
a,
b being
Complex st
(ComplexFuncAdd A) . (
((ComplexFuncExtMult A) . [a,f]),
((ComplexFuncExtMult A) . [b,g]))
= ComplexFuncZero A holds
(
a = 0 &
b = 0 ) ) & ( for
h being
Element of
Funcs (
A,
COMPLEX) ex
a,
b being
Complex st
h = (ComplexFuncAdd A) . (
((ComplexFuncExtMult A) . [a,f]),
((ComplexFuncExtMult A) . [b,g])) ) )
Lm3:
ex A being non empty set ex x1, x2 being set st
( A = {x1,x2} & x1 <> x2 )