begin
scheme
ElementEq{
F1()
-> set ,
P1[
set ] } :
for
X1,
X2 being
Element of
F1() st ( for
x being
set holds
(
x in X1 iff
P1[
x] ) ) & ( for
x being
set holds
(
x in X2 iff
P1[
x] ) ) holds
X1 = X2
scheme
TriOpEq{
F1()
-> non
empty set ,
F2(
Element of
F1(),
Element of
F1(),
Element of
F1())
-> set } :
for
f1,
f2 being
TriOp of
F1() st ( for
a,
b,
c being
Element of
F1() holds
f1 . (
a,
b,
c)
= F2(
a,
b,
c) ) & ( for
a,
b,
c being
Element of
F1() holds
f2 . (
a,
b,
c)
= F2(
a,
b,
c) ) holds
f1 = f2
scheme
QuaOpEq{
F1()
-> non
empty set ,
F2(
Element of
F1(),
Element of
F1(),
Element of
F1(),
Element of
F1())
-> set } :
for
f1,
f2 being
QuaOp of
F1() st ( for
a,
b,
c,
d being
Element of
F1() holds
f1 . (
a,
b,
c,
d)
= F2(
a,
b,
c,
d) ) & ( for
a,
b,
c,
d being
Element of
F1() holds
f2 . (
a,
b,
c,
d)
= F2(
a,
b,
c,
d) ) holds
f1 = f2
scheme
Fr3{
F1()
-> set ,
F2()
-> set ,
F3()
-> non
empty set ,
P1[
set ] } :
(
F1()
in F2() iff ex
a being
Element of
F3() st
(
F1()
= a &
P1[
a] ) )
provided
A1:
F2()
= { a where a is Element of F3() : P1[a] }
scheme
Fr4{
F1()
-> non
empty set ,
F2()
-> non
empty set ,
F3()
-> set ,
F4()
-> Element of
F1(),
F5(
set )
-> set ,
P1[
set ,
set ],
P2[
set ,
set ] } :
(
F4()
in F5(
F3()) iff for
b being
Element of
F2() st
b in F3() holds
P1[
F4(),
b] )
provided
A1:
F5(
F3())
= { a where a is Element of F1() : P2[a,F3()] }
and A2:
(
P2[
F4(),
F3()] iff for
b being
Element of
F2() st
b in F3() holds
P1[
F4(),
b] )
begin
Lm1:
for G being AbGroup
for a, b, c being Element of G holds
( - (a - b) = (- a) - (- b) & (a - b) + c = (a + c) - b )
theorem Th1:
theorem Th2:
theorem
theorem Th4:
theorem Th5:
theorem Th6:
begin
:: deftheorem Def1 defines SUBMODULE_DOMAIN LMOD_7:def 1 :
for K being Ring
for V being LeftMod of K
for b3 being non empty set holds
( b3 is SUBMODULE_DOMAIN of V iff for x being set st x in b3 holds
x is strict Subspace of V );
:: deftheorem defines LINE LMOD_7:def 2 :
for K being Ring
for V being LeftMod of K st not V is trivial holds
for b3 being strict Subspace of V holds
( b3 is LINE of V iff ex a being Vector of V st
( a <> 0. V & b3 = <:a:> ) );
:: deftheorem Def3 defines LINE_DOMAIN LMOD_7:def 3 :
for K being Ring
for V being LeftMod of K
for b3 being non empty set holds
( b3 is LINE_DOMAIN of V iff for x being set st x in b3 holds
x is LINE of V );
:: deftheorem defines lines LMOD_7:def 4 :
for K being Ring
for V being LeftMod of K
for b3 being LINE_DOMAIN of V holds
( b3 = lines V iff for x being set holds
( x in b3 iff x is LINE of V ) );
:: deftheorem defines HIPERPLANE LMOD_7:def 5 :
for K being Ring
for V being LeftMod of K st not V is trivial & V is free holds
for b3 being strict Subspace of V holds
( b3 is HIPERPLANE of V iff ex a being Vector of V st
( a <> 0. V & V is_the_direct_sum_of <:a:>,b3 ) );
:: deftheorem Def6 defines HIPERPLANE_DOMAIN LMOD_7:def 6 :
for K being Ring
for V being LeftMod of K
for b3 being non empty set holds
( b3 is HIPERPLANE_DOMAIN of V iff for x being set st x in b3 holds
x is HIPERPLANE of V );
:: deftheorem defines hiperplanes LMOD_7:def 7 :
for K being Ring
for V being LeftMod of K
for b3 being HIPERPLANE_DOMAIN of V holds
( b3 = hiperplanes V iff for x being set holds
( x in b3 iff x is HIPERPLANE of V ) );
begin
:: deftheorem defines Sum LMOD_7:def 8 :
for K being Ring
for V being LeftMod of K
for Li being FinSequence of Submodules V holds Sum Li = (SubJoin V) $$ Li;
:: deftheorem defines /\ LMOD_7:def 9 :
for K being Ring
for V being LeftMod of K
for Li being FinSequence of Submodules V holds /\ Li = (SubMeet V) $$ Li;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
begin
:: deftheorem defines + LMOD_7:def 10 :
for K being Ring
for V being LeftMod of K
for A1, A2, b5 being Subset of V holds
( b5 = A1 + A2 iff for x being set holds
( x in b5 iff ex a1, a2 being Vector of V st
( a1 in A1 & a2 in A2 & x = a1 + a2 ) ) );
begin
:: deftheorem Def11 defines Vector LMOD_7:def 11 :
for K being Ring
for V being LeftMod of K
for A being Subset of V st A <> {} holds
for b4 being Vector of V holds
( b4 is Vector of A iff b4 is Element of A );
theorem
theorem Th17:
theorem Th18:
:: deftheorem Def12 defines .. LMOD_7:def 12 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for b4 being set holds
( b4 = V .. W iff for x being set holds
( x in b4 iff ex a being Vector of V st x = a + W ) );
:: deftheorem defines .. LMOD_7:def 13 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for a being Vector of V holds a .. W = a + W;
theorem Th19:
theorem
:: deftheorem defines - LMOD_7:def 14 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for S1, b5 being Element of V .. W holds
( b5 = - S1 iff for a being Vector of V st S1 = a .. W holds
b5 = (- a) .. W );
:: deftheorem Def15 defines + LMOD_7:def 15 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for S1, S2, b6 being Element of V .. W holds
( b6 = S1 + S2 iff for a1, a2 being Vector of V st S1 = a1 .. W & S2 = a2 .. W holds
b6 = (a1 + a2) .. W );
definition
let K be
Ring;
let V be
LeftMod of
K;
let W be
Subspace of
V;
deffunc H1(
Element of
V .. W)
-> Element of
V .. W =
- $1;
func COMPL W -> UnOp of
(V .. W) means
for
S1 being
Element of
V .. W holds
it . S1 = - S1;
existence
ex b1 being UnOp of (V .. W) st
for S1 being Element of V .. W holds b1 . S1 = - S1
uniqueness
for b1, b2 being UnOp of (V .. W) st ( for S1 being Element of V .. W holds b1 . S1 = - S1 ) & ( for S1 being Element of V .. W holds b2 . S1 = - S1 ) holds
b1 = b2
deffunc H2(
Element of
V .. W,
Element of
V .. W)
-> Element of
V .. W = $1
+ $2;
func ADD W -> BinOp of
(V .. W) means :
Def17:
for
S1,
S2 being
Element of
V .. W holds
it . (
S1,
S2)
= S1 + S2;
existence
ex b1 being BinOp of (V .. W) st
for S1, S2 being Element of V .. W holds b1 . (S1,S2) = S1 + S2
uniqueness
for b1, b2 being BinOp of (V .. W) st ( for S1, S2 being Element of V .. W holds b1 . (S1,S2) = S1 + S2 ) & ( for S1, S2 being Element of V .. W holds b2 . (S1,S2) = S1 + S2 ) holds
b1 = b2
end;
:: deftheorem defines COMPL LMOD_7:def 16 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for b4 being UnOp of (V .. W) holds
( b4 = COMPL W iff for S1 being Element of V .. W holds b4 . S1 = - S1 );
:: deftheorem Def17 defines ADD LMOD_7:def 17 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for b4 being BinOp of (V .. W) holds
( b4 = ADD W iff for S1, S2 being Element of V .. W holds b4 . (S1,S2) = S1 + S2 );
:: deftheorem defines . LMOD_7:def 18 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V holds V . W = addLoopStr(# (V .. W),(ADD W),((0. V) .. W) #);
theorem
:: deftheorem defines . LMOD_7:def 19 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for a being Vector of V holds a . W = a .. W;
theorem Th22:
theorem
theorem Th24:
:: deftheorem Def20 defines * LMOD_7:def 20 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for r being Scalar of K
for S, b6 being Element of (V . W) holds
( b6 = r * S iff for a being Vector of V st S = a . W holds
b6 = (r * a) . W );
definition
let K be
Ring;
let V be
LeftMod of
K;
let W be
Subspace of
V;
func LMULT W -> Function of
[: the carrier of K, the carrier of (V . W):], the
carrier of
(V . W) means :
Def21:
for
r being
Scalar of
K for
S being
Element of
(V . W) holds
it . (
r,
S)
= r * S;
existence
ex b1 being Function of [: the carrier of K, the carrier of (V . W):], the carrier of (V . W) st
for r being Scalar of K
for S being Element of (V . W) holds b1 . (r,S) = r * S
uniqueness
for b1, b2 being Function of [: the carrier of K, the carrier of (V . W):], the carrier of (V . W) st ( for r being Scalar of K
for S being Element of (V . W) holds b1 . (r,S) = r * S ) & ( for r being Scalar of K
for S being Element of (V . W) holds b2 . (r,S) = r * S ) holds
b1 = b2
end;
:: deftheorem Def21 defines LMULT LMOD_7:def 21 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for b4 being Function of [: the carrier of K, the carrier of (V . W):], the carrier of (V . W) holds
( b4 = LMULT W iff for r being Scalar of K
for S being Element of (V . W) holds b4 . (r,S) = r * S );
begin
:: deftheorem defines / LMOD_7:def 22 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V holds V / W = VectSpStr(# the carrier of (V . W), the addF of (V . W),((0. V) . W),(LMULT W) #);
theorem
canceled;
theorem
theorem
:: deftheorem defines / LMOD_7:def 23 :
for K being Ring
for V being LeftMod of K
for W being Subspace of V
for a being Vector of V holds a / W = a . W;
theorem Th28:
theorem
theorem Th30:
Lm2:
for K being Ring
for V being LeftMod of K
for W being Subspace of V holds
( V / W is Abelian & V / W is add-associative & V / W is right_zeroed & V / W is right_complementable )
theorem Th31: