HM11:
for F being Field
for X, Y being VectSp of F
for T being linear-transformation of X,Y
for A being Subset of X st T is bijective & A is Basis of X holds
T .: A is Basis of Y
HM13:
for F being Field
for X, Y being VectSp of F
for T being linear-transformation of X,Y st T is bijective & X is finite-dimensional holds
Y is finite-dimensional
definition
let K be
Ring;
let V,
U be
VectSp of
K;
let W be
Subspace of
V;
let f be
linear-transformation of
V,
U;
assume A1:
the
carrier of
W c= the
carrier of
(ker f)
;
existence
ex b1 being linear-transformation of (VectQuot (V,W)),U st
for A being Vector of (VectQuot (V,W))
for a being Vector of V st A = a + W holds
b1 . A = f . a
uniqueness
for b1, b2 being linear-transformation of (VectQuot (V,W)),U st ( for A being Vector of (VectQuot (V,W))
for a being Vector of V st A = a + W holds
b1 . A = f . a ) & ( for A being Vector of (VectQuot (V,W))
for a being Vector of V st A = a + W holds
b2 . A = f . a ) holds
b1 = b2
end;
Lm3:
for K being Ring
for G being VectorSpace-Sequence of K
for v1, w1 being Element of product (carr G)
for i being Element of dom (carr G) holds
( ([:(addop G):] . (v1,w1)) . i = the addF of (G . i) . ((v1 . i),(w1 . i)) & ( for vi, wi being Vector of (G . i) st vi = v1 . i & wi = w1 . i holds
([:(addop G):] . (v1,w1)) . i = vi + wi ) )
Lm4:
for K being Ring
for G being VectorSpace-Sequence of K
for r being Element of K
for v being Element of product (carr G)
for i being Element of dom (carr G) holds
( ([:(multop G):] . (r,v)) . i = the lmult of (G . i) . (r,(v . i)) & ( for vi being Vector of (G . i) st vi = v . i holds
([:(multop G):] . (r,v)) . i = r * vi ) )
Lm5:
for K being Ring
for G being VectorSpace-Sequence of K holds
( product G is vector-distributive & product G is scalar-distributive & product G is scalar-associative & product G is scalar-unital )
definition
let K be
Ring;
let G,
F be non
empty ModuleStr over
K;
existence
ex b1 being Function of [: the carrier of K,[: the carrier of G, the carrier of F:]:],[: the carrier of G, the carrier of F:] st
for r being Element of K
for g being Vector of G
for f being Vector of F holds b1 . (r,[g,f]) = [(r * g),(r * f)]
uniqueness
for b1, b2 being Function of [: the carrier of K,[: the carrier of G, the carrier of F:]:],[: the carrier of G, the carrier of F:] st ( for r being Element of K
for g being Vector of G
for f being Vector of F holds b1 . (r,[g,f]) = [(r * g),(r * f)] ) & ( for r being Element of K
for g being Vector of G
for f being Vector of F holds b2 . (r,[g,f]) = [(r * g),(r * f)] ) holds
b1 = b2
end;
theorem
for
K being
Ring for
G,
F being non
empty ModuleStr over
K holds
( ( for
x being
set holds
(
x is
Vector of
[:G,F:] iff ex
x1 being
Vector of
G ex
x2 being
Vector of
F st
x = [x1,x2] ) ) & ( for
x,
y being
Vector of
[:G,F:] for
x1,
y1 being
Vector of
G for
x2,
y2 being
Vector 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
Vector of
[:G,F:] for
x1 being
Vector of
G for
x2 being
Vector of
F for
a being
Element of
K st
x = [x1,x2] holds
a * x = [(a * x1),(a * x2)] ) )
by YDef2, PRVECT_3:def 1, SUBSET_1:43;
theorem Th12:
for
K being
Ring for
X,
Y being
VectSp of
K ex
I being
Function of
[:X,Y:],
(product <*X,Y*>) st
(
I is
one-to-one &
I is
onto & ( for
x being
Vector of
X for
y being
Vector of
Y holds
I . (
x,
y)
= <*x,y*> ) & ( for
v,
w being
Vector of
[:X,Y:] holds
I . (v + w) = (I . v) + (I . w) ) & ( for
v being
Vector of
[:X,Y:] for
r being
Element of
K holds
I . (r * v) = r * (I . v) ) &
I . (0. [:X,Y:]) = 0. (product <*X,Y*>) )
theorem
for
K being
Ring for
G,
F being
VectSp of
K holds
( ( for
x being
set holds
(
x is
Vector of
(product <*G,F*>) iff ex
x1 being
Vector of
G ex
x2 being
Vector of
F st
x = <*x1,x2*> ) ) & ( for
x,
y being
Vector of
(product <*G,F*>) for
x1,
y1 being
Vector of
G for
x2,
y2 being
Vector 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
Vector of
(product <*G,F*>) for
x1 being
Vector of
G for
x2 being
Vector of
F st
x = <*x1,x2*> holds
- x = <*(- x1),(- x2)*> ) & ( for
x being
Vector of
(product <*G,F*>) for
x1 being
Vector of
G for
x2 being
Vector of
F for
a being
Element of
K st
x = <*x1,x2*> holds
a * x = <*(a * x1),(a * x2)*> ) )