Th1:
for X being RealLinearSpace-Sequence
for i being Element of dom X
for x being Element of (product X)
for r being Element of (X . i) holds (reproj (i,x)) . r = x +* (i,r)
by LOPBAN12:2;
Lm1:
for Y being RealNormSpace
for X being RealNormSpace-Sequence ex I being Lipschitzian LinearOperator of (NestingLB (X,Y)),(R_NormSpace_of_BoundedMultilinearOperators (X,Y)) st
( I is one-to-one & I is onto & I is isometric & ( for u being Element of (NestingLB (X,Y)) holds ||.(I . u).|| = ||.u.|| ) & ( for u being Point of (NestingLB (X,Y))
for x being Point of (product X) ex g being FinSequence st
( len g = len X & g . 1 = u & ( for i being Element of NAT st 1 <= i & i < len X holds
ex Xi being RealNormSpace-Sequence ex h being Point of (NestingLB (Xi,Y)) st
( Xi = X | (((len X) -' i) + 1) & h = g . i & g . (i + 1) = h . (x . (((len X) -' i) + 1)) ) ) & ex X1 being RealNormSpace-Sequence ex h being Point of (NestingLB (X1,Y)) st
( X1 = <*(X . 1)*> & h = g . (len X) & (I . u) . x = h . (x . 1) ) ) ) )
definition
let Y be
RealNormSpace;
let X be
RealNormSpace-Sequence;
existence
ex b1 being Lipschitzian LinearOperator of (NestingLB (X,Y)),(R_NormSpace_of_BoundedMultilinearOperators (X,Y)) st
( b1 is one-to-one & b1 is onto & b1 is isometric & ( for u being Element of (NestingLB (X,Y)) holds ||.(b1 . u).|| = ||.u.|| ) & ( for u being Point of (NestingLB (X,Y))
for x being Point of (product X) ex g being FinSequence st
( len g = len X & g . 1 = u & ( for i being Element of NAT st 1 <= i & i < len X holds
ex Xi being RealNormSpace-Sequence ex h being Point of (NestingLB (Xi,Y)) st
( Xi = X | (((len X) -' i) + 1) & h = g . i & g . (i + 1) = h . (x . (((len X) -' i) + 1)) ) ) & ex X1 being RealNormSpace-Sequence ex h being Point of (NestingLB (X1,Y)) st
( X1 = <*(X . 1)*> & h = g . (len X) & (b1 . u) . x = h . (x . 1) ) ) ) )
by Lm1;
uniqueness
for b1, b2 being Lipschitzian LinearOperator of (NestingLB (X,Y)),(R_NormSpace_of_BoundedMultilinearOperators (X,Y)) st b1 is one-to-one & b1 is onto & b1 is isometric & ( for u being Element of (NestingLB (X,Y)) holds ||.(b1 . u).|| = ||.u.|| ) & ( for u being Point of (NestingLB (X,Y))
for x being Point of (product X) ex g being FinSequence st
( len g = len X & g . 1 = u & ( for i being Element of NAT st 1 <= i & i < len X holds
ex Xi being RealNormSpace-Sequence ex h being Point of (NestingLB (Xi,Y)) st
( Xi = X | (((len X) -' i) + 1) & h = g . i & g . (i + 1) = h . (x . (((len X) -' i) + 1)) ) ) & ex X1 being RealNormSpace-Sequence ex h being Point of (NestingLB (X1,Y)) st
( X1 = <*(X . 1)*> & h = g . (len X) & (b1 . u) . x = h . (x . 1) ) ) ) & b2 is one-to-one & b2 is onto & b2 is isometric & ( for u being Element of (NestingLB (X,Y)) holds ||.(b2 . u).|| = ||.u.|| ) & ( for u being Point of (NestingLB (X,Y))
for x being Point of (product X) ex g being FinSequence st
( len g = len X & g . 1 = u & ( for i being Element of NAT st 1 <= i & i < len X holds
ex Xi being RealNormSpace-Sequence ex h being Point of (NestingLB (Xi,Y)) st
( Xi = X | (((len X) -' i) + 1) & h = g . i & g . (i + 1) = h . (x . (((len X) -' i) + 1)) ) ) & ex X1 being RealNormSpace-Sequence ex h being Point of (NestingLB (X1,Y)) st
( X1 = <*(X . 1)*> & h = g . (len X) & (b2 . u) . x = h . (x . 1) ) ) ) holds
b1 = b2
end;