definition
let X,
Y,
Z be
RealLinearSpace;
existence
ex b1 being Subset of (RealVectSpace ( the carrier of [:X,Y:],Z)) st
for x being set holds
( x in b1 iff x is BilinearOperator of X,Y,Z )
uniqueness
for b1, b2 being Subset of (RealVectSpace ( the carrier of [:X,Y:],Z)) st ( for x being set holds
( x in b1 iff x is BilinearOperator of X,Y,Z ) ) & ( for x being set holds
( x in b2 iff x is BilinearOperator of X,Y,Z ) ) holds
b1 = b2
end;
LM14:
for X being RealLinearSpace
for x1, x2, x3, x4 being Point of X holds (x1 + x2) + (x3 + x4) = (x1 + x3) + (x2 + x4)
Th14:
for X, Y, Z being RealLinearSpace holds BilinearOperators (X,Y,Z) is linearly-closed
definition
let X,
Y,
Z be
RealLinearSpace;
func R_VectorSpace_of_BilinearOperators (
X,
Y,
Z)
-> strict RLSStruct equals
RLSStruct(#
(BilinearOperators (X,Y,Z)),
(Zero_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))),
(Add_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))),
(Mult_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))) #);
coherence
RLSStruct(# (BilinearOperators (X,Y,Z)),(Zero_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))),(Add_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))),(Mult_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))) #) is strict RLSStruct
;
end;
::
deftheorem defines
R_VectorSpace_of_BilinearOperators LOPBAN_9:def 2 :
for X, Y, Z being RealLinearSpace holds R_VectorSpace_of_BilinearOperators (X,Y,Z) = RLSStruct(# (BilinearOperators (X,Y,Z)),(Zero_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))),(Add_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))),(Mult_ ((BilinearOperators (X,Y,Z)),(RealVectSpace ( the carrier of [:X,Y:],Z)))) #);
registration
let X,
Y,
Z be
RealLinearSpace;
coherence
( R_VectorSpace_of_BilinearOperators (X,Y,Z) is Abelian & R_VectorSpace_of_BilinearOperators (X,Y,Z) is add-associative & R_VectorSpace_of_BilinearOperators (X,Y,Z) is right_zeroed & R_VectorSpace_of_BilinearOperators (X,Y,Z) is right_complementable & R_VectorSpace_of_BilinearOperators (X,Y,Z) is vector-distributive & R_VectorSpace_of_BilinearOperators (X,Y,Z) is scalar-distributive & R_VectorSpace_of_BilinearOperators (X,Y,Z) is scalar-associative & R_VectorSpace_of_BilinearOperators (X,Y,Z) is scalar-unital )
by RSSPACE:11;
end;
definition
let X,
Y,
Z be
RealNormSpace;
existence
ex b1 being Subset of (R_VectorSpace_of_BilinearOperators (X,Y,Z)) st
for x being set holds
( x in b1 iff x is Lipschitzian BilinearOperator of X,Y,Z )
uniqueness
for b1, b2 being Subset of (R_VectorSpace_of_BilinearOperators (X,Y,Z)) st ( for x being set holds
( x in b1 iff x is Lipschitzian BilinearOperator of X,Y,Z ) ) & ( for x being set holds
( x in b2 iff x is Lipschitzian BilinearOperator of X,Y,Z ) ) holds
b1 = b2
end;
definition
let X,
Y,
Z be
RealNormSpace;
func R_VectorSpace_of_BoundedBilinearOperators (
X,
Y,
Z)
-> strict RLSStruct equals
RLSStruct(#
(BoundedBilinearOperators (X,Y,Z)),
(Zero_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),
(Add_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),
(Mult_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))) #);
coherence
RLSStruct(# (BoundedBilinearOperators (X,Y,Z)),(Zero_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Add_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Mult_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))) #) is strict RLSStruct
;
end;
::
deftheorem defines
R_VectorSpace_of_BoundedBilinearOperators LOPBAN_9:def 5 :
for X, Y, Z being RealNormSpace holds R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) = RLSStruct(# (BoundedBilinearOperators (X,Y,Z)),(Zero_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Add_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Mult_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))) #);
registration
let X,
Y,
Z be
RealNormSpace;
coherence
( R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is Abelian & R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is add-associative & R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is right_zeroed & R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is right_complementable & R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is vector-distributive & R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is scalar-distributive & R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is scalar-associative & R_VectorSpace_of_BoundedBilinearOperators (X,Y,Z) is scalar-unital )
by RSSPACE:11;
end;
definition
let X,
Y,
Z be
RealNormSpace;
func BoundedBilinearOperatorsNorm (
X,
Y,
Z)
-> Function of
(BoundedBilinearOperators (X,Y,Z)),
REAL means :
Def13:
for
x being
object st
x in BoundedBilinearOperators (
X,
Y,
Z) holds
it . x = upper_bound (PreNorms (modetrans (x,X,Y,Z)));
existence
ex b1 being Function of (BoundedBilinearOperators (X,Y,Z)),REAL st
for x being object st x in BoundedBilinearOperators (X,Y,Z) holds
b1 . x = upper_bound (PreNorms (modetrans (x,X,Y,Z)))
uniqueness
for b1, b2 being Function of (BoundedBilinearOperators (X,Y,Z)),REAL st ( for x being object st x in BoundedBilinearOperators (X,Y,Z) holds
b1 . x = upper_bound (PreNorms (modetrans (x,X,Y,Z))) ) & ( for x being object st x in BoundedBilinearOperators (X,Y,Z) holds
b2 . x = upper_bound (PreNorms (modetrans (x,X,Y,Z))) ) holds
b1 = b2
end;
::
deftheorem Def13 defines
BoundedBilinearOperatorsNorm LOPBAN_9:def 8 :
for X, Y, Z being RealNormSpace
for b4 being Function of (BoundedBilinearOperators (X,Y,Z)),REAL holds
( b4 = BoundedBilinearOperatorsNorm (X,Y,Z) iff for x being object st x in BoundedBilinearOperators (X,Y,Z) holds
b4 . x = upper_bound (PreNorms (modetrans (x,X,Y,Z))) );
Th29:
for X, Y, Z being RealNormSpace
for f being Lipschitzian BilinearOperator of X,Y,Z holds modetrans (f,X,Y,Z) = f
definition
let X,
Y,
Z be
RealNormSpace;
func R_NormSpace_of_BoundedBilinearOperators (
X,
Y,
Z)
-> non
empty NORMSTR equals
NORMSTR(#
(BoundedBilinearOperators (X,Y,Z)),
(Zero_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),
(Add_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),
(Mult_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),
(BoundedBilinearOperatorsNorm (X,Y,Z)) #);
coherence
NORMSTR(# (BoundedBilinearOperators (X,Y,Z)),(Zero_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Add_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Mult_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(BoundedBilinearOperatorsNorm (X,Y,Z)) #) is non empty NORMSTR
;
end;
::
deftheorem defines
R_NormSpace_of_BoundedBilinearOperators LOPBAN_9:def 9 :
for X, Y, Z being RealNormSpace holds R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) = NORMSTR(# (BoundedBilinearOperators (X,Y,Z)),(Zero_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Add_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(Mult_ ((BoundedBilinearOperators (X,Y,Z)),(R_VectorSpace_of_BilinearOperators (X,Y,Z)))),(BoundedBilinearOperatorsNorm (X,Y,Z)) #);
Th38:
for X, Y, Z being RealNormSpace holds
( R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is reflexive & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is discerning & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is RealNormSpace-like )
registration
let X,
Y,
Z be
RealNormSpace;
coherence
( R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is vector-distributive & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is scalar-distributive & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is scalar-associative & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is scalar-unital & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is Abelian & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is add-associative & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is right_zeroed & R_NormSpace_of_BoundedBilinearOperators (X,Y,Z) is right_complementable )
by Th39;
end;
Lm3:
for e being Real
for seq being Real_Sequence st seq is convergent & ex k being Nat st
for i being Nat st k <= i holds
seq . i <= e holds
lim seq <= e
theorem
for
X,
Y,
Z being
RealLinearSpace ex
I being
LinearOperator of
(R_VectorSpace_of_LinearOperators (X,(R_VectorSpace_of_LinearOperators (Y,Z)))),
(R_VectorSpace_of_BilinearOperators (X,Y,Z)) st
(
I is
bijective & ( for
u being
Point of
(R_VectorSpace_of_LinearOperators (X,(R_VectorSpace_of_LinearOperators (Y,Z)))) for
x being
Point of
X for
y being
Point of
Y holds
(I . u) . (
x,
y)
= (u . x) . y ) )
theorem
for
X,
Y,
Z being
RealNormSpace ex
I being
LinearOperator of
(R_NormSpace_of_BoundedLinearOperators (X,(R_NormSpace_of_BoundedLinearOperators (Y,Z)))),
(R_NormSpace_of_BoundedBilinearOperators (X,Y,Z)) st
(
I is
bijective & ( for
u being
Point of
(R_NormSpace_of_BoundedLinearOperators (X,(R_NormSpace_of_BoundedLinearOperators (Y,Z)))) holds
(
||.u.|| = ||.(I . u).|| & ( for
x being
Point of
X for
y being
Point of
Y holds
(I . u) . (
x,
y)
= (u . x) . y ) ) ) )