begin
theorem
for
D,
E,
F,
G being non
empty set ex
I being
Function of
[:[:D,E:],[:F,G:]:],
[:[:D,F:],[:E,G:]:] st
(
I is
one-to-one &
I is
onto & ( for
d,
e,
f,
g being
set st
d in D &
e in E &
f in F &
g in G holds
I . (
[d,e],
[f,g])
= [[d,f],[e,g]] ) )
theorem Th2:
theorem Th3:
theorem Th4:
theorem Th5:
theorem Th6:
Lm1:
for G, F being non empty 1-sorted
for x being set st x in [: the carrier of G, the carrier of F:] holds
ex x1 being Point of G ex x2 being Point of F st x = [x1,x2]
by SUBSET_1:65;
Lm2:
for G, F being non empty addLoopStr ex ADGF being Function of [:[: the carrier of G, the carrier of F:],[: the carrier of G, the carrier of F:]:],[: the carrier of G, the carrier of F:] st
for g1, g2 being Point of G
for f1, f2 being Point of F holds ADGF . ([g1,f1],[g2,f2]) = [(g1 + g2),(f1 + f2)]
definition
let G,
F be non
empty addLoopStr ;
func prod_ADD (
G,
F)
-> BinOp of
[: the carrier of G, the carrier of F:] means :
Def1:
for
g1,
g2 being
Point of
G for
f1,
f2 being
Point of
F holds
it . (
[g1,f1],
[g2,f2])
= [(g1 + g2),(f1 + f2)];
existence
ex b1 being BinOp of [: the carrier of G, the carrier of F:] st
for g1, g2 being Point of G
for f1, f2 being Point of F holds b1 . ([g1,f1],[g2,f2]) = [(g1 + g2),(f1 + f2)]
by Lm2;
uniqueness
for b1, b2 being BinOp of [: the carrier of G, the carrier of F:] st ( for g1, g2 being Point of G
for f1, f2 being Point of F holds b1 . ([g1,f1],[g2,f2]) = [(g1 + g2),(f1 + f2)] ) & ( for g1, g2 being Point of G
for f1, f2 being Point of F holds b2 . ([g1,f1],[g2,f2]) = [(g1 + g2),(f1 + f2)] ) holds
b1 = b2
end;
:: deftheorem Def1 defines prod_ADD PRVECT_3:def 1 :
for G, F being non empty addLoopStr
for b3 being BinOp of [: the carrier of G, the carrier of F:] holds
( b3 = prod_ADD (G,F) iff for g1, g2 being Point of G
for f1, f2 being Point of F holds b3 . ([g1,f1],[g2,f2]) = [(g1 + g2),(f1 + f2)] );
Lm3:
for G, F being non empty RLSStruct ex MLTGF being Function of [:REAL,[: the carrier of G, the carrier of F:]:],[: the carrier of G, the carrier of F:] st
for r being Element of REAL
for g being Point of G
for f being Point of F holds MLTGF . (r,[g,f]) = [(r * g),(r * f)]
definition
let G,
F be non
empty RLSStruct ;
func prod_MLT (
G,
F)
-> Function of
[:REAL,[: the carrier of G, the carrier of F:]:],
[: the carrier of G, the carrier of F:] means :
Def2:
for
r being
Element of
REAL for
g being
Point of
G for
f being
Point of
F holds
it . (
r,
[g,f])
= [(r * g),(r * f)];
existence
ex b1 being Function of [:REAL,[: the carrier of G, the carrier of F:]:],[: the carrier of G, the carrier of F:] st
for r being Element of REAL
for g being Point of G
for f being Point of F holds b1 . (r,[g,f]) = [(r * g),(r * f)]
by Lm3;
uniqueness
for b1, b2 being Function of [:REAL,[: the carrier of G, the carrier of F:]:],[: the carrier of G, the carrier of F:] st ( for r being Element of REAL
for g being Point of G
for f being Point of F holds b1 . (r,[g,f]) = [(r * g),(r * f)] ) & ( for r being Element of REAL
for g being Point of G
for f being Point of F holds b2 . (r,[g,f]) = [(r * g),(r * f)] ) holds
b1 = b2
end;
:: deftheorem Def2 defines prod_MLT PRVECT_3:def 2 :
for G, F being non empty RLSStruct
for b3 being Function of [:REAL,[: the carrier of G, the carrier of F:]:],[: the carrier of G, the carrier of F:] holds
( b3 = prod_MLT (G,F) iff for r being Element of REAL
for g being Point of G
for f being Point of F holds b3 . (r,[g,f]) = [(r * g),(r * f)] );
:: deftheorem defines prod_ZERO PRVECT_3:def 3 :
for G, F being non empty addLoopStr holds prod_ZERO (G,F) = [(0. G),(0. F)];
definition
let G,
F be non
empty addLoopStr ;
func [:G,F:] -> non
empty strict addLoopStr equals
addLoopStr(#
[: the carrier of G, the carrier of F:],
(prod_ADD (G,F)),
(prod_ZERO (G,F)) #);
correctness
coherence
addLoopStr(# [: the carrier of G, the carrier of F:],(prod_ADD (G,F)),(prod_ZERO (G,F)) #) is non empty strict addLoopStr ;
;
end;
:: deftheorem defines [: PRVECT_3:def 4 :
for G, F being non empty addLoopStr holds [:G,F:] = addLoopStr(# [: the carrier of G, the carrier of F:],(prod_ADD (G,F)),(prod_ZERO (G,F)) #);
theorem
for
G,
F being non
empty addLoopStr holds
( ( for
x being
set holds
(
x is
Point of
[:G,F:] iff ex
x1 being
Point of
G ex
x2 being
Point of
F st
x = [x1,x2] ) ) & ( for
x,
y being
Point of
[:G,F:] for
x1,
y1 being
Point of
G for
x2,
y2 being
Point of
F st
x = [x1,x2] &
y = [y1,y2] holds
x + y = [(x1 + y1),(x2 + y2)] ) &
0. [:G,F:] = [(0. G),(0. F)] )
by Lm1, Def1;
theorem
definition
let G,
F be non
empty RLSStruct ;
func [:G,F:] -> non
empty strict RLSStruct equals
RLSStruct(#
[: the carrier of G, the carrier of F:],
(prod_ZERO (G,F)),
(prod_ADD (G,F)),
(prod_MLT (G,F)) #);
correctness
coherence
RLSStruct(# [: the carrier of G, the carrier of F:],(prod_ZERO (G,F)),(prod_ADD (G,F)),(prod_MLT (G,F)) #) is non empty strict RLSStruct ;
;
end;
:: deftheorem defines [: PRVECT_3:def 5 :
for G, F being non empty RLSStruct holds [:G,F:] = RLSStruct(# [: the carrier of G, the carrier of F:],(prod_ZERO (G,F)),(prod_ADD (G,F)),(prod_MLT (G,F)) #);
theorem Th9:
for
G,
F being non
empty RLSStruct holds
( ( for
x being
set holds
(
x is
Point of
[:G,F:] iff ex
x1 being
Point of
G ex
x2 being
Point of
F st
x = [x1,x2] ) ) & ( for
x,
y being
Point of
[:G,F:] for
x1,
y1 being
Point of
G for
x2,
y2 being
Point of
F st
x = [x1,x2] &
y = [y1,y2] holds
x + y = [(x1 + y1),(x2 + y2)] ) &
0. [:G,F:] = [(0. G),(0. F)] & ( for
x being
Point of
[:G,F:] for
x1 being
Point of
G for
x2 being
Point of
F for
a being
real number st
x = [x1,x2] holds
a * x = [(a * x1),(a * x2)] ) )
theorem
begin
theorem Th11:
theorem Th12:
for
X,
Y being
RealLinearSpace ex
I being
Function of
[:X,Y:],
(product <*X,Y*>) st
(
I is
one-to-one &
I is
onto & ( for
x being
Point of
X for
y being
Point of
Y holds
I . (
x,
y)
= <*x,y*> ) & ( for
v,
w being
Point of
[:X,Y:] holds
I . (v + w) = (I . v) + (I . w) ) & ( for
v being
Point of
[:X,Y:] for
r being
Element of
REAL holds
I . (r * v) = r * (I . v) ) &
I . (0. [:X,Y:]) = 0. (product <*X,Y*>) )
Lm4:
for X being non empty non-empty FinSequence
for x being set st x in product X holds
x is FinSequence
theorem Th13:
theorem
for
G,
F being
RealLinearSpace holds
( ( for
x being
set holds
(
x is
Point of
(product <*G,F*>) iff ex
x1 being
Point of
G ex
x2 being
Point of
F st
x = <*x1,x2*> ) ) & ( for
x,
y being
Point of
(product <*G,F*>) for
x1,
y1 being
Point of
G for
x2,
y2 being
Point of
F st
x = <*x1,x2*> &
y = <*y1,y2*> holds
x + y = <*(x1 + y1),(x2 + y2)*> ) &
0. (product <*G,F*>) = <*(0. G),(0. F)*> & ( for
x being
Point of
(product <*G,F*>) for
x1 being
Point of
G for
x2 being
Point of
F st
x = <*x1,x2*> holds
- x = <*(- x1),(- x2)*> ) & ( for
x being
Point of
(product <*G,F*>) for
x1 being
Point of
G for
x2 being
Point of
F for
a being
real number st
x = <*x1,x2*> holds
a * x = <*(a * x1),(a * x2)*> ) )
begin
Lm5:
for G, F being non empty NORMSTR ex NORMGF being Function of [: the carrier of G, the carrier of F:],REAL st
for g being Point of G
for f being Point of F ex v being Element of REAL 2 st
( v = <*||.g.||,||.f.||*> & NORMGF . (g,f) = |.v.| )
definition
let G,
F be non
empty NORMSTR ;
func prod_NORM (
G,
F)
-> Function of
[: the carrier of G, the carrier of F:],
REAL means :
Def6:
for
g being
Point of
G for
f being
Point of
F ex
v being
Element of
REAL 2 st
(
v = <*||.g.||,||.f.||*> &
it . (
g,
f)
= |.v.| );
existence
ex b1 being Function of [: the carrier of G, the carrier of F:],REAL st
for g being Point of G
for f being Point of F ex v being Element of REAL 2 st
( v = <*||.g.||,||.f.||*> & b1 . (g,f) = |.v.| )
by Lm5;
uniqueness
for b1, b2 being Function of [: the carrier of G, the carrier of F:],REAL st ( for g being Point of G
for f being Point of F ex v being Element of REAL 2 st
( v = <*||.g.||,||.f.||*> & b1 . (g,f) = |.v.| ) ) & ( for g being Point of G
for f being Point of F ex v being Element of REAL 2 st
( v = <*||.g.||,||.f.||*> & b2 . (g,f) = |.v.| ) ) holds
b1 = b2
end;
:: deftheorem Def6 defines prod_NORM PRVECT_3:def 6 :
for G, F being non empty NORMSTR
for b3 being Function of [: the carrier of G, the carrier of F:],REAL holds
( b3 = prod_NORM (G,F) iff for g being Point of G
for f being Point of F ex v being Element of REAL 2 st
( v = <*||.g.||,||.f.||*> & b3 . (g,f) = |.v.| ) );
definition
let G,
F be non
empty NORMSTR ;
func [:G,F:] -> non
empty strict NORMSTR equals
NORMSTR(#
[: the carrier of G, the carrier of F:],
(prod_ZERO (G,F)),
(prod_ADD (G,F)),
(prod_MLT (G,F)),
(prod_NORM (G,F)) #);
correctness
coherence
NORMSTR(# [: the carrier of G, the carrier of F:],(prod_ZERO (G,F)),(prod_ADD (G,F)),(prod_MLT (G,F)),(prod_NORM (G,F)) #) is non empty strict NORMSTR ;
;
end;
:: deftheorem defines [: PRVECT_3:def 7 :
for G, F being non empty NORMSTR holds [:G,F:] = NORMSTR(# [: the carrier of G, the carrier of F:],(prod_ZERO (G,F)),(prod_ADD (G,F)),(prod_MLT (G,F)),(prod_NORM (G,F)) #);
registration
let G,
F be non
empty right_complementable Abelian add-associative right_zeroed vector-distributive scalar-distributive scalar-associative scalar-unital discerning reflexive RealNormSpace-like NORMSTR ;
cluster [:G,F:] -> non
empty right_complementable Abelian add-associative right_zeroed vector-distributive scalar-distributive scalar-associative scalar-unital discerning reflexive strict RealNormSpace-like ;
correctness
coherence
( [:G,F:] is strict & [:G,F:] is reflexive & [:G,F:] is discerning & [:G,F:] is RealNormSpace-like & [:G,F:] is scalar-distributive & [:G,F:] is vector-distributive & [:G,F:] is scalar-associative & [:G,F:] is scalar-unital & [:G,F:] is Abelian & [:G,F:] is add-associative & [:G,F:] is right_zeroed & [:G,F:] is right_complementable );
end;
theorem Th15:
for
X,
Y being
RealNormSpace ex
I being
Function of
[:X,Y:],
(product <*X,Y*>) st
(
I is
one-to-one &
I is
onto & ( for
x being
Point of
X for
y being
Point of
Y holds
I . (
x,
y)
= <*x,y*> ) & ( for
v,
w being
Point of
[:X,Y:] holds
I . (v + w) = (I . v) + (I . w) ) & ( for
v being
Point of
[:X,Y:] for
r being
Element of
REAL holds
I . (r * v) = r * (I . v) ) &
0. (product <*X,Y*>) = I . (0. [:X,Y:]) & ( for
v being
Point of
[:X,Y:] holds
||.(I . v).|| = ||.v.|| ) )
theorem Th16:
Lm6:
for F1, F2 being FinSequence of REAL holds sqr (F1 ^ F2) = (sqr F1) ^ (sqr F2)
by TOPREAL7:11;
theorem Th17:
for
X,
Y being non
empty RealNormSpace-Sequence ex
I being
Function of
[:(product X),(product Y):],
(product (X ^ Y)) st
(
I is
one-to-one &
I is
onto & ( for
x being
Point of
(product X) for
y being
Point of
(product Y) ex
x1,
y1 being
FinSequence st
(
x = x1 &
y = y1 &
I . (
x,
y)
= x1 ^ y1 ) ) & ( for
v,
w being
Point of
[:(product X),(product Y):] holds
I . (v + w) = (I . v) + (I . w) ) & ( for
v being
Point of
[:(product X),(product Y):] for
r being
Element of
REAL holds
I . (r * v) = r * (I . v) ) &
I . (0. [:(product X),(product Y):]) = 0. (product (X ^ Y)) & ( for
v being
Point of
[:(product X),(product Y):] holds
||.(I . v).|| = ||.v.|| ) )
theorem Th18:
for
G,
F being
RealNormSpace holds
( ( for
x being
set holds
(
x is
Point of
[:G,F:] iff ex
x1 being
Point of
G ex
x2 being
Point of
F st
x = [x1,x2] ) ) & ( for
x,
y being
Point of
[:G,F:] for
x1,
y1 being
Point of
G for
x2,
y2 being
Point of
F st
x = [x1,x2] &
y = [y1,y2] holds
x + y = [(x1 + y1),(x2 + y2)] ) &
0. [:G,F:] = [(0. G),(0. F)] & ( for
x being
Point of
[:G,F:] for
x1 being
Point of
G for
x2 being
Point of
F st
x = [x1,x2] holds
- x = [(- x1),(- x2)] ) & ( for
x being
Point of
[:G,F:] for
x1 being
Point of
G for
x2 being
Point of
F for
a being
real number st
x = [x1,x2] holds
a * x = [(a * x1),(a * x2)] ) & ( for
x being
Point of
[:G,F:] for
x1 being
Point of
G for
x2 being
Point of
F st
x = [x1,x2] holds
ex
w being
Element of
REAL 2 st
(
w = <*||.x1.||,||.x2.||*> &
||.x.|| = |.w.| ) ) )
theorem Th19:
for
G,
F being
RealNormSpace holds
( ( for
x being
set holds
(
x is
Point of
(product <*G,F*>) iff ex
x1 being
Point of
G ex
x2 being
Point of
F st
x = <*x1,x2*> ) ) & ( for
x,
y being
Point of
(product <*G,F*>) for
x1,
y1 being
Point of
G for
x2,
y2 being
Point of
F st
x = <*x1,x2*> &
y = <*y1,y2*> holds
x + y = <*(x1 + y1),(x2 + y2)*> ) &
0. (product <*G,F*>) = <*(0. G),(0. F)*> & ( for
x being
Point of
(product <*G,F*>) for
x1 being
Point of
G for
x2 being
Point of
F st
x = <*x1,x2*> holds
- x = <*(- x1),(- x2)*> ) & ( for
x being
Point of
(product <*G,F*>) for
x1 being
Point of
G for
x2 being
Point of
F for
a being
real number st
x = <*x1,x2*> holds
a * x = <*(a * x1),(a * x2)*> ) & ( for
x being
Point of
(product <*G,F*>) for
x1 being
Point of
G for
x2 being
Point of
F st
x = <*x1,x2*> holds
ex
w being
Element of
REAL 2 st
(
w = <*||.x1.||,||.x2.||*> &
||.x.|| = |.w.| ) ) )
theorem
for
X,
Y being non
empty RealNormSpace-Sequence ex
I being
Function of
(product <*(product X),(product Y)*>),
(product (X ^ Y)) st
(
I is
one-to-one &
I is
onto & ( for
x being
Point of
(product X) for
y being
Point of
(product Y) ex
x1,
y1 being
FinSequence st
(
x = x1 &
y = y1 &
I . <*x,y*> = x1 ^ y1 ) ) & ( for
v,
w being
Point of
(product <*(product X),(product Y)*>) holds
I . (v + w) = (I . v) + (I . w) ) & ( for
v being
Point of
(product <*(product X),(product Y)*>) for
r being
Element of
REAL holds
I . (r * v) = r * (I . v) ) &
I . (0. (product <*(product X),(product Y)*>)) = 0. (product (X ^ Y)) & ( for
v being
Point of
(product <*(product X),(product Y)*>) holds
||.(I . v).|| = ||.v.|| ) )
theorem Th21:
for
X,
Y being non
empty RealLinearSpace ex
I being
Function of
[:X,Y:],
[:X,(product <*Y*>):] st
(
I is
one-to-one &
I is
onto & ( for
x being
Point of
X for
y being
Point of
Y holds
I . (
x,
y)
= [x,<*y*>] ) & ( for
v,
w being
Point of
[:X,Y:] holds
I . (v + w) = (I . v) + (I . w) ) & ( for
v being
Point of
[:X,Y:] for
r being
Element of
REAL holds
I . (r * v) = r * (I . v) ) &
I . (0. [:X,Y:]) = 0. [:X,(product <*Y*>):] )
theorem
theorem Th23:
for
X,
Y being non
empty RealNormSpace ex
I being
Function of
[:X,Y:],
[:X,(product <*Y*>):] st
(
I is
one-to-one &
I is
onto & ( for
x being
Point of
X for
y being
Point of
Y holds
I . (
x,
y)
= [x,<*y*>] ) & ( for
v,
w being
Point of
[:X,Y:] holds
I . (v + w) = (I . v) + (I . w) ) & ( for
v being
Point of
[:X,Y:] for
r being
Element of
REAL holds
I . (r * v) = r * (I . v) ) &
I . (0. [:X,Y:]) = 0. [:X,(product <*Y*>):] & ( for
v being
Point of
[:X,Y:] holds
||.(I . v).|| = ||.v.|| ) )
theorem