theorem LMINEQ:
for
x,
y,
z being
Real st
0 <= y & ( for
e being
Real st
0 < e holds
x <= z + (y * e) ) holds
x <= z
SUBTH:
for V being RealNormSpace
for V1 being Subset of V
for x, y being Point of V
for x1, y1 being Point of (NLin V1)
for a being Real st x = x1 & y = y1 holds
( ||.x.|| = ||.x1.|| & x + y = x1 + y1 & a * x = a * x1 )
XTh7:
for V being RealNormSpace
for V1 being Subset of V
for x, y being Point of (NLin V1)
for a being Real holds
( ( ||.x.|| = 0 implies x = 0. (NLin V1) ) & ( x = 0. (NLin V1) implies ||.x.|| = 0 ) & 0 <= ||.x.|| & ||.(x + y).|| <= ||.x.|| + ||.y.|| & ||.(a * x).|| = |.a.| * ||.x.|| )
NISOM06:
for X, Y being RealNormSpace
for L being Lipschitzian LinearOperator of X,Y
for V being Subset of X
for W being Subset of Y st L is isomorphism & W = L .: V & W is closed holds
V is closed
definition
let V,
W be
RealLinearSpace;
let L be
LinearOperator of
V,
W;
existence
ex b1 being LinearOperator of (VectQuot (V,(Ker L))),(Im L) st
( b1 is isomorphism & ( for z being Point of (VectQuot (V,(Ker L)))
for v being VECTOR of V st z = v + (Ker L) holds
b1 . z = L . v ) )
by LMQ21;
uniqueness
for b1, b2 being LinearOperator of (VectQuot (V,(Ker L))),(Im L) st b1 is isomorphism & ( for z being Point of (VectQuot (V,(Ker L)))
for v being VECTOR of V st z = v + (Ker L) holds
b1 . z = L . v ) & b2 is isomorphism & ( for z being Point of (VectQuot (V,(Ker L)))
for v being VECTOR of V st z = v + (Ker L) holds
b2 . z = L . v ) holds
b1 = b2
end;
LMQ231:
for V being RealNormSpace
for W being Subspace of V
for v being VECTOR of V holds NormVSets (V,W,v) is bounded_below
definition
let V be
RealNormSpace;
let W be
Subspace of
V;
existence
ex b1 being Function of (CosetSet (V,W)),REAL st
for A being Element of CosetSet (V,W)
for v being VECTOR of V st A = v + W holds
b1 . A = lower_bound (NormVSets (V,W,v))
uniqueness
for b1, b2 being Function of (CosetSet (V,W)),REAL st ( for A being Element of CosetSet (V,W)
for v being VECTOR of V st A = v + W holds
b1 . A = lower_bound (NormVSets (V,W,v)) ) & ( for A being Element of CosetSet (V,W)
for v being VECTOR of V st A = v + W holds
b2 . A = lower_bound (NormVSets (V,W,v)) ) holds
b1 = b2
end;
definition
let X be
RealNormSpace;
let Y be
Subspace of
X;
assume A1:
ex
CY being
Subset of
X st
(
CY = the
carrier of
Y &
CY is
closed )
;
existence
ex b1 being strict RealNormSpace st
( RLSStruct(# the carrier of b1, the ZeroF of b1, the addF of b1, the Mult of b1 #) = VectQuot (X,Y) & the normF of b1 = NormCoset (X,Y) )
uniqueness
for b1, b2 being strict RealNormSpace st RLSStruct(# the carrier of b1, the ZeroF of b1, the addF of b1, the Mult of b1 #) = VectQuot (X,Y) & the normF of b1 = NormCoset (X,Y) & RLSStruct(# the carrier of b2, the ZeroF of b2, the addF of b2, the Mult of b2 #) = VectQuot (X,Y) & the normF of b2 = NormCoset (X,Y) holds
b1 = b2
;
end;
LMCL1:
for X being RealNormSpace
for Y, Z being Subset of X st Z = the carrier of (Lin Y) holds
not Cl Z is empty
definition
let X be
RealNormSpace;
let Y be
Subset of
X;
correctness
existence
ex b1 being non empty NORMSTR ex Z being Subset of X st
( Z = the carrier of (Lin Y) & b1 = NORMSTR(# (Cl Z),(Zero_ ((Cl Z),X)),(Add_ ((Cl Z),X)),(Mult_ ((Cl Z),X)),(Norm_ ((Cl Z),X)) #) );
uniqueness
for b1, b2 being non empty NORMSTR st ex Z being Subset of X st
( Z = the carrier of (Lin Y) & b1 = NORMSTR(# (Cl Z),(Zero_ ((Cl Z),X)),(Add_ ((Cl Z),X)),(Mult_ ((Cl Z),X)),(Norm_ ((Cl Z),X)) #) ) & ex Z being Subset of X st
( Z = the carrier of (Lin Y) & b2 = NORMSTR(# (Cl Z),(Zero_ ((Cl Z),X)),(Add_ ((Cl Z),X)),(Mult_ ((Cl Z),X)),(Norm_ ((Cl Z),X)) #) ) holds
b1 = b2;
end;
SUBTHCL:
for V being RealNormSpace
for V1 being Subset of V
for x, y being Point of V
for x1, y1 being Point of (ClNLin V1)
for a being Real st x = x1 & y = y1 holds
( ||.x.|| = ||.x1.|| & x + y = x1 + y1 & a * x = a * x1 )