begin
:: deftheorem Def1 defines convex VECTMETR:def 1 :
for V being non empty MetrStruct holds
( V is convex iff for x, y being Element of V
for r being Real st 0 <= r & r <= 1 holds
ex z being Element of V st
( dist (x,z) = r * (dist (x,y)) & dist (z,y) = (1 - r) * (dist (x,y)) ) );
:: deftheorem defines internal VECTMETR:def 2 :
for V being non empty MetrStruct holds
( V is internal iff for x, y being Element of V
for p, q being Real st p > 0 & q > 0 holds
ex f being FinSequence of the carrier of V st
( f /. 1 = x & f /. (len f) = y & ( for i being Element of NAT st 1 <= i & i <= (len f) - 1 holds
dist ((f /. i),(f /. (i + 1))) < p ) & ( for F being FinSequence of REAL st len F = (len f) - 1 & ( for i being Element of NAT st 1 <= i & i <= len F holds
F /. i = dist ((f /. i),(f /. (i + 1))) ) holds
abs ((dist (x,y)) - (Sum F)) < q ) ) );
theorem Th1:
begin
:: deftheorem Def3 defines isometric VECTMETR:def 3 :
for V being non empty MetrStruct
for f being Function of V,V holds
( f is isometric iff for x, y being Element of V holds dist (x,y) = dist ((f . x),(f . y)) );
theorem
:: deftheorem Def4 defines ISOM VECTMETR:def 4 :
for V being non empty MetrStruct
for b2 being set holds
( b2 = ISOM V iff for x being set holds
( x in b2 iff x is onto isometric Function of V,V ) );
theorem
theorem
theorem
begin
registration
let X be non
empty set ;
let F be
Function of
[:X,X:],
REAL;
let O be
Element of
X;
let B be
BinOp of
X;
let G be
Function of
[:REAL,X:],
X;
cluster RLSMetrStruct(#
X,
F,
O,
B,
G #)
-> non
empty ;
coherence
not RLSMetrStruct(# X,F,O,B,G #) is empty
;
end;
:: deftheorem Def5 defines homogeneous VECTMETR:def 5 :
for V being non empty RLSMetrStruct holds
( V is homogeneous iff for r being Real
for v, w being Element of V holds dist ((r * v),(r * w)) = (abs r) * (dist (v,w)) );
:: deftheorem Def6 defines translatible VECTMETR:def 6 :
for V being non empty RLSMetrStruct holds
( V is translatible iff for u, w, v being Element of V holds dist (v,w) = dist ((v + u),(w + u)) );
:: deftheorem defines Norm VECTMETR:def 7 :
for V being non empty RLSMetrStruct
for v being Element of V holds Norm v = dist ((0. V),v);
theorem
theorem
theorem
definition
let n be
Element of
NAT ;
func RLMSpace n -> strict RealLinearMetrSpace means :
Def8:
( the
carrier of
it = REAL n & the
distance of
it = Pitag_dist n &
0. it = 0* n & ( for
x,
y being
Element of
REAL n holds the
addF of
it . (
x,
y)
= x + y ) & ( for
x being
Element of
REAL n for
r being
Element of
REAL holds the
Mult of
it . (
r,
x)
= r * x ) );
existence
ex b1 being strict RealLinearMetrSpace st
( the carrier of b1 = REAL n & the distance of b1 = Pitag_dist n & 0. b1 = 0* n & ( for x, y being Element of REAL n holds the addF of b1 . (x,y) = x + y ) & ( for x being Element of REAL n
for r being Element of REAL holds the Mult of b1 . (r,x) = r * x ) )
uniqueness
for b1, b2 being strict RealLinearMetrSpace st the carrier of b1 = REAL n & the distance of b1 = Pitag_dist n & 0. b1 = 0* n & ( for x, y being Element of REAL n holds the addF of b1 . (x,y) = x + y ) & ( for x being Element of REAL n
for r being Element of REAL holds the Mult of b1 . (r,x) = r * x ) & the carrier of b2 = REAL n & the distance of b2 = Pitag_dist n & 0. b2 = 0* n & ( for x, y being Element of REAL n holds the addF of b2 . (x,y) = x + y ) & ( for x being Element of REAL n
for r being Element of REAL holds the Mult of b2 . (r,x) = r * x ) holds
b1 = b2
end;
:: deftheorem Def8 defines RLMSpace VECTMETR:def 8 :
for n being Element of NAT
for b2 being strict RealLinearMetrSpace holds
( b2 = RLMSpace n iff ( the carrier of b2 = REAL n & the distance of b2 = Pitag_dist n & 0. b2 = 0* n & ( for x, y being Element of REAL n holds the addF of b2 . (x,y) = x + y ) & ( for x being Element of REAL n
for r being Element of REAL holds the Mult of b2 . (r,x) = r * x ) ) );
theorem
begin
:: deftheorem Def9 defines IsomGroup VECTMETR:def 9 :
for n being Element of NAT
for b2 being strict multMagma holds
( b2 = IsomGroup n iff ( the carrier of b2 = ISOM (RLMSpace n) & ( for f, g being Function st f in ISOM (RLMSpace n) & g in ISOM (RLMSpace n) holds
the multF of b2 . (f,g) = f * g ) ) );
theorem Th10:
theorem Th11:
:: deftheorem Def10 defines SubIsomGroupRel VECTMETR:def 10 :
for n being Element of NAT
for G being Subgroup of IsomGroup n
for b3 being Relation of the carrier of (RLMSpace n) holds
( b3 = SubIsomGroupRel G iff for A, B being Element of (RLMSpace n) holds
( [A,B] in b3 iff ex f being Function st
( f in the carrier of G & f . A = B ) ) );