begin
:: deftheorem DefComplexAlgebra defines ComplexSubAlgebra CC0SP1:def 1 :
for V, b2 being ComplexAlgebra holds
( b2 is ComplexSubAlgebra of V iff ( the carrier of b2 c= the carrier of V & the addF of b2 = the addF of V || the carrier of b2 & the multF of b2 = the multF of V || the carrier of b2 & the Mult of b2 = the Mult of V | [:COMPLEX, the carrier of b2:] & 1. b2 = 1. V & 0. b2 = 0. V ) );
theorem Th1:
for
X being non
empty set for
V being
ComplexAlgebra for
V1 being non
empty Subset of
V for
d1,
d2 being
Element of
X for
A being
BinOp of
X for
M being
Function of
[:X,X:],
X for
MR being
Function of
[:COMPLEX,X:],
X st
V1 = X &
d1 = 0. V &
d2 = 1. V &
A = the
addF of
V || V1 &
M = the
multF of
V || V1 &
MR = the
Mult of
V | [:COMPLEX,V1:] &
V1 is
having-inverse holds
ComplexAlgebraStr(#
X,
M,
A,
MR,
d2,
d1 #) is
ComplexSubAlgebra of
V
:: deftheorem Def10 defines Cadditively-linearly-closed CC0SP1:def 2 :
for V being ComplexAlgebra
for V1 being Subset of V holds
( V1 is Cadditively-linearly-closed iff ( V1 is add-closed & V1 is having-inverse & ( for a being Complex
for v being Element of V st v in V1 holds
a * v in V1 ) ) );
:: deftheorem Def11 defines Mult_ CC0SP1:def 3 :
for V being ComplexAlgebra
for V1 being Subset of V st V1 is Cadditively-linearly-closed & not V1 is empty holds
Mult_ (V1,V) = the Mult of V | [:COMPLEX,V1:];
:: deftheorem defines ComplexBoundedFunctions CC0SP1:def 4 :
for X being non empty set holds ComplexBoundedFunctions X = { f where f is Function of X,COMPLEX : f | X is bounded } ;
:: deftheorem defines scalar-mult-cancelable CC0SP1:def 5 :
for V being non empty CLSStruct holds
( V is scalar-mult-cancelable iff for a being Complex
for v being Element of V holds
( not a * v = 0. V or a = 0 or v = 0. V ) );
theorem Th2:
for
V being
ComplexAlgebra for
V1 being non
empty multiplicatively-closed Cadditively-linearly-closed Subset of
V holds
ComplexAlgebraStr(#
V1,
(mult_ (V1,V)),
(Add_ (V1,V)),
(Mult_ (V1,V)),
(One_ (V1,V)),
(Zero_ (V1,V)) #) is
ComplexSubAlgebra of
V
theorem Th4:
definition
let X be non
empty set ;
func C_Algebra_of_BoundedFunctions X -> ComplexAlgebra equals
ComplexAlgebraStr(#
(ComplexBoundedFunctions X),
(mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(Add_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(Mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(One_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(Zero_ ((ComplexBoundedFunctions X),(CAlgebra X))) #);
coherence
ComplexAlgebraStr(# (ComplexBoundedFunctions X),(mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Add_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(One_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Zero_ ((ComplexBoundedFunctions X),(CAlgebra X))) #) is ComplexAlgebra
by Th2;
end;
:: deftheorem defines C_Algebra_of_BoundedFunctions CC0SP1:def 6 :
for X being non empty set holds C_Algebra_of_BoundedFunctions X = ComplexAlgebraStr(# (ComplexBoundedFunctions X),(mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Add_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(One_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Zero_ ((ComplexBoundedFunctions X),(CAlgebra X))) #);
theorem
theorem Th8:
theorem Th9:
theorem Th10:
theorem Th11:
theorem Th12:
:: deftheorem DefB7 defines modetrans CC0SP1:def 7 :
for X being non empty set
for F being set st F in ComplexBoundedFunctions X holds
for b3 being Function of X,COMPLEX holds
( b3 = modetrans (F,X) iff ( b3 = F & b3 | X is bounded ) );
:: deftheorem defines PreNorms CC0SP1:def 8 :
for X being non empty set
for f being Function of X,COMPLEX holds PreNorms f = { |.(f . x).| where x is Element of X : verum } ;
Lm1:
for C being non empty set
for f being PartFunc of C,COMPLEX holds
( |.f.| is bounded iff f is bounded )
theorem Th13:
theorem Th14:
theorem Th15:
:: deftheorem DefB9C defines ComplexBoundedFunctionsNorm CC0SP1:def 9 :
for X being non empty set
for b2 being Function of (ComplexBoundedFunctions X),REAL holds
( b2 = ComplexBoundedFunctionsNorm X iff for x being set st x in ComplexBoundedFunctions X holds
b2 . x = upper_bound (PreNorms (modetrans (x,X))) );
theorem Th16:
theorem Th17:
definition
let X be non
empty set ;
func C_Normed_Algebra_of_BoundedFunctions X -> Normed_Complex_AlgebraStr equals
Normed_Complex_AlgebraStr(#
(ComplexBoundedFunctions X),
(mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(Add_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(Mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(One_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(Zero_ ((ComplexBoundedFunctions X),(CAlgebra X))),
(ComplexBoundedFunctionsNorm X) #);
correctness
coherence
Normed_Complex_AlgebraStr(# (ComplexBoundedFunctions X),(mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Add_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(One_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Zero_ ((ComplexBoundedFunctions X),(CAlgebra X))),(ComplexBoundedFunctionsNorm X) #) is Normed_Complex_AlgebraStr ;
;
end;
:: deftheorem defines C_Normed_Algebra_of_BoundedFunctions CC0SP1:def 10 :
for X being non empty set holds C_Normed_Algebra_of_BoundedFunctions X = Normed_Complex_AlgebraStr(# (ComplexBoundedFunctions X),(mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Add_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Mult_ ((ComplexBoundedFunctions X),(CAlgebra X))),(One_ ((ComplexBoundedFunctions X),(CAlgebra X))),(Zero_ ((ComplexBoundedFunctions X),(CAlgebra X))),(ComplexBoundedFunctionsNorm X) #);
Lm2:
now
let X be non
empty set ;
for x, e being Element of (C_Normed_Algebra_of_BoundedFunctions X) st e = One_ ((ComplexBoundedFunctions X),(CAlgebra X)) holds
( x * e = x & e * x = x )set F =
C_Normed_Algebra_of_BoundedFunctions X;
let x,
e be
Element of
(C_Normed_Algebra_of_BoundedFunctions X);
( e = One_ ((ComplexBoundedFunctions X),(CAlgebra X)) implies ( x * e = x & e * x = x ) )set X1 =
ComplexBoundedFunctions X;
reconsider f =
x as
Element of
ComplexBoundedFunctions X ;
assume A1:
e = One_ (
(ComplexBoundedFunctions X),
(CAlgebra X))
;
( x * e = x & e * x = x )then
x * e = (mult_ ((ComplexBoundedFunctions X),(CAlgebra X))) . (
f,
(1_ (CAlgebra X)))
by C0SP1:def 8;
then A2:
x * e = ( the multF of (CAlgebra X) || (ComplexBoundedFunctions X)) . (
f,
(1_ (CAlgebra X)))
by C0SP1:def 6;
e * x = (mult_ ((ComplexBoundedFunctions X),(CAlgebra X))) . (
(1_ (CAlgebra X)),
f)
by A1, C0SP1:def 8;
then A3:
e * x = ( the multF of (CAlgebra X) || (ComplexBoundedFunctions X)) . (
(1_ (CAlgebra X)),
f)
by C0SP1:def 6;
A4:
1_ (CAlgebra X) = 1_ (C_Algebra_of_BoundedFunctions X)
by Th12;
then
[f,(1_ (CAlgebra X))] in [:(ComplexBoundedFunctions X),(ComplexBoundedFunctions X):]
by ZFMISC_1:106;
then
x * e = f * (1_ (CAlgebra X))
by A2, FUNCT_1:72;
hence
x * e = x
by VECTSP_1:def 13;
e * x = x
[(1_ (CAlgebra X)),f] in [:(ComplexBoundedFunctions X),(ComplexBoundedFunctions X):]
by A4, ZFMISC_1:106;
then
e * x = (1_ (CAlgebra X)) * f
by A3, FUNCT_1:72;
hence
e * x = x
by VECTSP_1:def 13;
verum
end;
theorem Th18:
theorem Th19:
theorem
theorem Th21:
theorem Th22:
theorem Th23:
theorem
theorem Th25:
theorem Th26:
theorem Th27:
theorem Th28:
theorem Th29:
Th30:
for X being non empty set holds
( C_Normed_Algebra_of_BoundedFunctions X is reflexive & C_Normed_Algebra_of_BoundedFunctions X is discerning & C_Normed_Algebra_of_BoundedFunctions X is ComplexNormSpace-like )
theorem Th31:
theorem Th32:
theorem