definition
let X,
Y be
RealLinearSpace;
existence
ex b1 being LinearOperator of [:X,Y:],(product <*X,Y*>) st
for x being Point of X
for y being Point of Y holds b1 . (x,y) = <*x,y*>
uniqueness
for b1, b2 being LinearOperator of [:X,Y:],(product <*X,Y*>) st ( for x being Point of X
for y being Point of Y holds b1 . (x,y) = <*x,y*> ) & ( for x being Point of X
for y being Point of Y holds b2 . (x,y) = <*x,y*> ) holds
b1 = b2
end;
registration
let X,
Y be
RealLinearSpace;
cluster Relation-like the
carrier of
[:X,Y:] -defined the
carrier of
(product <*X,Y*>) -valued Function-like V11()
V14( the
carrier of
[:X,Y:])
quasi_total bijective V166(
[:X,Y:],
product <*X,Y*>)
V167(
[:X,Y:],
product <*X,Y*>) for
Element of
K19(
K20( the
carrier of
[:X,Y:], the
carrier of
(product <*X,Y*>)));
correctness
existence
ex b1 being LinearOperator of [:X,Y:],(product <*X,Y*>) st b1 is bijective ;
end;
definition
let X,
Y be
RealLinearSpace;
let f be
bijective LinearOperator of
[:X,Y:],
(product <*X,Y*>);
"redefine func f " -> LinearOperator of
(product <*X,Y*>),
[:X,Y:];
correctness
coherence
f " is LinearOperator of (product <*X,Y*>),[:X,Y:];
end;
registration
let X,
Y be
RealLinearSpace;
cluster Relation-like the
carrier of
(product <*X,Y*>) -defined the
carrier of
[:X,Y:] -valued Function-like V11()
V14( the
carrier of
(product <*X,Y*>))
quasi_total bijective V166(
product <*X,Y*>,
[:X,Y:])
V167(
product <*X,Y*>,
[:X,Y:]) for
Element of
K19(
K20( the
carrier of
(product <*X,Y*>), the
carrier of
[:X,Y:]));
correctness
existence
ex b1 being LinearOperator of (product <*X,Y*>),[:X,Y:] st b1 is bijective ;
end;
theorem IS03:
for
X,
Y,
Z being
RealLinearSpace ex
I being
LinearOperator of
(R_VectorSpace_of_BilinearOperators (X,Y,Z)),
(R_VectorSpace_of_MultilinearOperators (<*X,Y*>,Z)) st
(
I is
bijective & ( for
u being
Point of
(R_VectorSpace_of_BilinearOperators (X,Y,Z)) holds
I . u = u * ((IsoCPRLSP (X,Y)) ") ) )
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_MultilinearOperators (<*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 IS03A:
for
X,
Y,
Z being
RealNormSpace ex
I being
LinearOperator of
(R_NormSpace_of_BoundedBilinearOperators (X,Y,Z)),
(R_NormSpace_of_BoundedMultilinearOperators (<*X,Y*>,Z)) st
(
I is
bijective &
I is
isometric & ( for
u being
Point of
(R_NormSpace_of_BoundedBilinearOperators (X,Y,Z)) holds
I . u = u * ((IsoCPNrSP (X,Y)) ") ) )
theorem IS04A:
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_BoundedMultilinearOperators (<*X,Y*>,Z)) st
(
I is
bijective &
I is
isometric & ( 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 ) ) ) )