dtr:
for F being Field
for V being VectSp of F holds
( V is trivial iff the carrier of V = {(0. V)} )
canlininj1:
for F being Field
for U, V being VectSp of F
for B being non empty finite Subset of U
for f being Function of B,V
for l2 being Linear_Combination of rng f ex l1 being Linear_Combination of B st
for u being Element of U st u in B holds
l1 . u = l2 . (f . u)
XXX1:
for F being Field
for U, V being VectSp of F
for B being non empty Subset of U
for f being Function of B,V st f is one-to-one holds
for v being Element of V st v in rng f holds
f " {v} = {((f ") . v)}
lemadd2b:
for F being Field
for U, V being VectSp of F
for B being non empty finite Subset of U
for f being Function of B,V
for l being Linear_Combination of B
for v being Element of V st not v in rng f holds
(f (#) l) . v = 0. F
lemadd:
for F being Field
for U, V being VectSp of F
for B being non empty finite Subset of U
for f being Function of B,V
for l1, l2, l3 being Linear_Combination of B st l3 = l1 + l2 holds
Sum (f (#) l3) = (Sum (f (#) l1)) + (Sum (f (#) l2))
lemmult:
for F being Field
for U, V being VectSp of F
for B being non empty finite Subset of U
for f being Function of B,V
for l1, l2 being Linear_Combination of B
for a being Element of F st a * l1 = l2 holds
Sum (f (#) l2) = a * (Sum (f (#) l1))
lemminus:
for F being Field
for U, V being VectSp of F
for B being non empty finite Subset of U
for f being Function of B,V
for l1, l2, l3 being Linear_Combination of B st l3 = l1 - l2 holds
Sum (f (#) l3) = (Sum (f (#) l1)) - (Sum (f (#) l2))
XXX4a:
for F being Field
for U being non trivial finite-dimensional VectSp of F
for V being finite-dimensional VectSp of F
for B being Basis of U
for f being Function of B,V st f is one-to-one holds
for l being Linear_Combination of rng f holds (canLinTrans f) . (Sum (l (#) f)) = Sum l
canLininjrngA:
for F being Field
for U being non trivial finite-dimensional VectSp of F
for V being finite-dimensional VectSp of F
for B being Basis of U
for f being Function of B,V st canLinTrans f is one-to-one holds
rng f is linearly-independent
canLininjrngB:
for F being Field
for U being non trivial finite-dimensional VectSp of F
for V being finite-dimensional VectSp of F
for B being Basis of U
for f being Function of B,V st f is one-to-one & rng f is linearly-independent holds
canLinTrans f is one-to-one
definition
let R be
Ring;
let n be
Nat;
existence
ex b1 being BinOp of (n -tuples_on the carrier of R) st
for u, v being Tuple of n, the carrier of R holds b1 . (u,v) = u + v
uniqueness
for b1, b2 being BinOp of (n -tuples_on the carrier of R) st ( for u, v being Tuple of n, the carrier of R holds b1 . (u,v) = u + v ) & ( for u, v being Tuple of n, the carrier of R holds b2 . (u,v) = u + v ) holds
b1 = b2
existence
ex b1 being Function of [: the carrier of R,(n -tuples_on the carrier of R):],(n -tuples_on the carrier of R) st
for a being Element of R
for u being Tuple of n, the carrier of R holds b1 . (a,u) = a * u
uniqueness
for b1, b2 being Function of [: the carrier of R,(n -tuples_on the carrier of R):],(n -tuples_on the carrier of R) st ( for a being Element of R
for u being Tuple of n, the carrier of R holds b1 . (a,u) = a * u ) & ( for a being Element of R
for u being Tuple of n, the carrier of R holds b2 . (a,u) = a * u ) holds
b1 = b2
end;
lemBB:
for R being Ring
for n being Nat
for u being Element of (R ^* n)
for v being Element of n -tuples_on the carrier of R
for a being Element of R st u = v holds
a * u = a * v
lemBA:
for R being Ring
for n being Nat
for v being Element of n -tuples_on the carrier of R
for a being Element of R
for i being Nat st 1 <= i & i <= n holds
( (a * (i _th_unit_vector (n,R))) . i = a & ( for j being Nat st j <> i & 1 <= j & j <= n holds
(a * (j _th_unit_vector (n,R))) . i = 0. R ) )
lemBC:
for R being Ring
for n being Nat
for u, v being Element of (R ^* n)
for a, b being Element of n -tuples_on the carrier of R st u = a & v = b holds
a + b = u + v
lemspan1:
for R being non degenerated commutative Ring
for n being Nat
for o being Element of (R ^* n) ex l being Linear_Combination of Base (R,n) st Sum l = o
definition
let X be non
empty set ;
let L be non
empty addLoopStr ;
existence
ex b1 being BinOp of (Funcs (X, the carrier of L)) st
for f, g being Function of X,L holds b1 . (f,g) = f '+' g
uniqueness
for b1, b2 being BinOp of (Funcs (X, the carrier of L)) st ( for f, g being Function of X,L holds b1 . (f,g) = f '+' g ) & ( for f, g being Function of X,L holds b2 . (f,g) = f '+' g ) holds
b1 = b2
end;
definition
let X be non
empty set ;
let L be non
empty multLoopStr ;
existence
ex b1 being Function of [: the carrier of L,(Funcs (X, the carrier of L)):],(Funcs (X, the carrier of L)) st
for f being Function of X,L
for a being Element of L holds b1 . (a,f) = a '*' f
uniqueness
for b1, b2 being Function of [: the carrier of L,(Funcs (X, the carrier of L)):],(Funcs (X, the carrier of L)) st ( for f being Function of X,L
for a being Element of L holds b1 . (a,f) = a '*' f ) & ( for f being Function of X,L
for a being Element of L holds b2 . (a,f) = a '*' f ) holds
b1 = b2
end;
definition
let X be non
empty set ;
let L be non
empty doubleLoopStr ;
existence
ex b1 being strict ModuleStr over L st
( the carrier of b1 = Funcs (X, the carrier of L) & the addF of b1 = mapAdd (X,L) & the ZeroF of b1 = X --> (0. L) & the lmult of b1 = mapMult (X,L) )
uniqueness
for b1, b2 being strict ModuleStr over L st the carrier of b1 = Funcs (X, the carrier of L) & the addF of b1 = mapAdd (X,L) & the ZeroF of b1 = X --> (0. L) & the lmult of b1 = mapMult (X,L) & the carrier of b2 = Funcs (X, the carrier of L) & the addF of b2 = mapAdd (X,L) & the ZeroF of b2 = X --> (0. L) & the lmult of b2 = mapMult (X,L) holds
b1 = b2
;
end;
definition
let X be non
empty set ;
let R be non
empty addLoopStr ;
let L be non
empty ModuleStr over
R;
existence
ex b1 being BinOp of (Funcs (X, the carrier of L)) st
for f, g being Function of X,L holds b1 . (f,g) = f '+' g
uniqueness
for b1, b2 being BinOp of (Funcs (X, the carrier of L)) st ( for f, g being Function of X,L holds b1 . (f,g) = f '+' g ) & ( for f, g being Function of X,L holds b2 . (f,g) = f '+' g ) holds
b1 = b2
end;
definition
let X be non
empty set ;
let R be non
empty multLoopStr ;
let L be non
empty ModuleStr over
R;
existence
ex b1 being Function of [: the carrier of R,(Funcs (X, the carrier of L)):],(Funcs (X, the carrier of L)) st
for f being Function of X,L
for a being Element of R holds b1 . (a,f) = a '*' f
uniqueness
for b1, b2 being Function of [: the carrier of R,(Funcs (X, the carrier of L)):],(Funcs (X, the carrier of L)) st ( for f being Function of X,L
for a being Element of R holds b1 . (a,f) = a '*' f ) & ( for f being Function of X,L
for a being Element of R holds b2 . (a,f) = a '*' f ) holds
b1 = b2
end;
definition
let X be non
empty set ;
let R be non
empty doubleLoopStr ;
let L be non
empty ModuleStr over
R;
existence
ex b1 being strict ModuleStr over R st
( the carrier of b1 = Funcs (X, the carrier of L) & the addF of b1 = mapAdd (X,L) & the ZeroF of b1 = X --> (0. L) & the lmult of b1 = mapMult (X,L) )
uniqueness
for b1, b2 being strict ModuleStr over R st the carrier of b1 = Funcs (X, the carrier of L) & the addF of b1 = mapAdd (X,L) & the ZeroF of b1 = X --> (0. L) & the lmult of b1 = mapMult (X,L) & the carrier of b2 = Funcs (X, the carrier of L) & the addF of b2 = mapAdd (X,L) & the ZeroF of b2 = X --> (0. L) & the lmult of b2 = mapMult (X,L) holds
b1 = b2
;
end;