Lm1:
for K being non empty well-unital doubleLoopStr
for h, e being Element of (opp K) st e = 1. K holds
( h * e = h & e * h = h )
Lm3:
for K being non empty right_complementable add-associative right_zeroed doubleLoopStr
for x, y being Scalar of K
for a, b being Scalar of (opp K) st x = a & y = b holds
( x + y = a + b & x * y = b * a & - x = - a )
Lm4:
for K being non empty doubleLoopStr
for x, y, z, u being Scalar of K
for a, b, c, d being Scalar of (opp K) st x = a & y = b & z = c & u = d holds
( (x + y) + z = (a + b) + c & x + (y + z) = a + (b + c) & (x * y) * z = c * (b * a) & x * (y * z) = (c * b) * a & x * (y + z) = (b + c) * a & (y + z) * x = a * (b + c) & (x * y) + (z * u) = (b * a) + (d * c) )
Lm5:
for F being non empty commutative doubleLoopStr
for x, y being Element of F holds x * y = y * x
;
definition
let K be non
empty doubleLoopStr ;
let V be non
empty ModuleStr over
K;
existence
ex b1 being strict RightModStr over opp K st
for o being Function of [: the carrier of V, the carrier of (opp K):], the carrier of V st o = ~ the lmult of V holds
b1 = RightModStr(# the carrier of V, the addF of V,(0. V),o #)
uniqueness
for b1, b2 being strict RightModStr over opp K st ( for o being Function of [: the carrier of V, the carrier of (opp K):], the carrier of V st o = ~ the lmult of V holds
b1 = RightModStr(# the carrier of V, the addF of V,(0. V),o #) ) & ( for o being Function of [: the carrier of V, the carrier of (opp K):], the carrier of V st o = ~ the lmult of V holds
b2 = RightModStr(# the carrier of V, the addF of V,(0. V),o #) ) holds
b1 = b2
end;
definition
let K be non
empty doubleLoopStr ;
let W be non
empty RightModStr over
K;
existence
ex b1 being strict ModuleStr over opp K st
for o being Function of [: the carrier of (opp K), the carrier of W:], the carrier of W st o = ~ the rmult of W holds
b1 = ModuleStr(# the carrier of W, the addF of W,(0. W),o #)
uniqueness
for b1, b2 being strict ModuleStr over opp K st ( for o being Function of [: the carrier of (opp K), the carrier of W:], the carrier of W st o = ~ the rmult of W holds
b1 = ModuleStr(# the carrier of W, the addF of W,(0. W),o #) ) & ( for o being Function of [: the carrier of (opp K), the carrier of W:], the carrier of W st o = ~ the rmult of W holds
b2 = ModuleStr(# the carrier of W, the addF of W,(0. W),o #) ) holds
b1 = b2
end;
registration
let K,
L be non
empty doubleLoopStr ;
coherence
for b1 being Function of K,L st b1 is antilinear holds
( b1 is additive & b1 is antimultiplicative & b1 is unity-preserving )
;
coherence
for b1 being Function of K,L st b1 is additive & b1 is antimultiplicative & b1 is unity-preserving holds
b1 is antilinear
;
coherence
for b1 being Function of K,L st b1 is monomorphism holds
( b1 is linear & b1 is one-to-one )
;
coherence
for b1 being Function of K,L st b1 is linear & b1 is one-to-one holds
b1 is monomorphism
;
coherence
for b1 being Function of K,L st b1 is antimonomorphism holds
( b1 is antilinear & b1 is one-to-one )
;
coherence
for b1 being Function of K,L st b1 is antilinear & b1 is one-to-one holds
b1 is antimonomorphism
;
coherence
for b1 being Function of K,L st b1 is epimorphism holds
( b1 is linear & b1 is onto )
;
coherence
for b1 being Function of K,L st b1 is linear & b1 is onto holds
b1 is epimorphism
;
coherence
for b1 being Function of K,L st b1 is antiepimorphism holds
( b1 is antilinear & b1 is onto )
;
coherence
for b1 being Function of K,L st b1 is antilinear & b1 is onto holds
b1 is antiepimorphism
;
coherence
for b1 being Function of K,L st b1 is isomorphism holds
( b1 is monomorphism & b1 is onto )
;
coherence
for b1 being Function of K,L st b1 is monomorphism & b1 is onto holds
b1 is isomorphism
;
coherence
for b1 being Function of K,L st b1 is antiisomorphism holds
( b1 is antimonomorphism & b1 is onto )
;
coherence
for b1 being Function of K,L st b1 is antimonomorphism & b1 is onto holds
b1 is antiisomorphism
;
end;
Lm6:
for K, L being Ring
for J being Function of K,L st J is additive holds
J . (0. K) = 0. L
Lm7:
for K, L being Ring
for J being Function of K,L
for x being Scalar of K st J is linear holds
J . (- x) = - (J . x)
Lm8:
for K, L being Ring
for J being Function of K,L
for x, y being Scalar of K st J is linear holds
J . (x - y) = (J . x) - (J . y)
Lm9:
for K, L being Ring
for J being Function of K,L st J is antilinear holds
J . (0. K) = 0. L
Lm10:
for K, L being Ring
for J being Function of K,L
for x being Scalar of K st J is antilinear holds
J . (- x) = - (J . x)
Lm11:
for K, L being Ring
for J being Function of K,L
for x, y being Scalar of K st J is antilinear holds
J . (x - y) = (J . x) - (J . y)
Lm12:
for K being non empty right_complementable add-associative right_zeroed doubleLoopStr
for L being non empty right_complementable well-unital add-associative right_zeroed doubleLoopStr
for J being Function of K,L st J is linear holds
opp J is additive
Lm13:
for G, H being AddGroup
for f being Homomorphism of G,H holds f . (0. G) = 0. H
Lm14:
for G, H being AddGroup
for f being Homomorphism of G,H
for x being Element of G holds f . (- x) = - (f . x)
Lm15:
for G, H being AddGroup
for f being Homomorphism of G,H
for x, y being Element of G holds f . (x - y) = (f . x) - (f . y)
Lm16:
for K, L being Ring
for V being LeftMod of K
for W being LeftMod of L
for x, y being Vector of V holds (ZeroMap (V,W)) . (x + y) = ((ZeroMap (V,W)) . x) + ((ZeroMap (V,W)) . y)
Lm17:
for K, L being Ring
for J being Function of K,L
for V being LeftMod of K
for W being LeftMod of L
for a being Scalar of K
for x being Vector of V holds (ZeroMap (V,W)) . (a * x) = (J . a) * ((ZeroMap (V,W)) . x)