begin
definition
let IT be non
empty AffinStruct ;
attr IT is
WeakAffVect-like means :
Def1:
( ( for
a,
b,
c being
Element of
IT st
a,
b // c,
c holds
a = b ) & ( for
a,
b,
c,
d,
p,
q being
Element of
IT st
a,
b // p,
q &
c,
d // p,
q holds
a,
b // c,
d ) & ( for
a,
b,
c being
Element of
IT ex
d being
Element of
IT st
a,
b // c,
d ) & ( for
a,
b,
c,
a9,
b9,
c9 being
Element of
IT st
a,
b // a9,
b9 &
a,
c // a9,
c9 holds
b,
c // b9,
c9 ) & ( for
a,
c being
Element of
IT ex
b being
Element of
IT st
a,
b // b,
c ) & ( for
a,
b,
c,
d being
Element of
IT st
a,
b // c,
d holds
a,
c // b,
d ) );
end;
:: deftheorem Def1 defines WeakAffVect-like AFVECT0:def 1 :
for IT being non empty AffinStruct holds
( IT is WeakAffVect-like iff ( ( for a, b, c being Element of IT st a,b // c,c holds
a = b ) & ( for a, b, c, d, p, q being Element of IT st a,b // p,q & c,d // p,q holds
a,b // c,d ) & ( for a, b, c being Element of IT ex d being Element of IT st a,b // c,d ) & ( for a, b, c, a9, b9, c9 being Element of IT st a,b // a9,b9 & a,c // a9,c9 holds
b,c // b9,c9 ) & ( for a, c being Element of IT ex b being Element of IT st a,b // b,c ) & ( for a, b, c, d being Element of IT st a,b // c,d holds
a,c // b,d ) ) );
theorem
canceled;
theorem Th2:
theorem
theorem Th4:
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
theorem
theorem
for
AFV being
WeakAffVect for
b,
c,
b9,
c9,
a,
d,
d9 being
Element of
AFV st
b,
c // b9,
c9 &
a,
d // b,
c &
a,
d9 // b9,
c9 holds
d = d9
theorem
for
AFV being
WeakAffVect for
a,
b,
a9,
b9,
c,
d,
d9 being
Element of
AFV st
a,
b // a9,
b9 &
c,
d // b,
a &
c,
d9 // b9,
a9 holds
d = d9
theorem
for
AFV being
WeakAffVect for
a,
b,
a9,
b9,
c,
d,
c9,
d9,
f,
f9 being
Element of
AFV st
a,
b // a9,
b9 &
c,
d // c9,
d9 &
b,
f // c,
d &
b9,
f9 // c9,
d9 holds
a,
f // a9,
f9
theorem Th13:
for
AFV being
WeakAffVect for
a,
b,
a9,
b9,
c,
c9 being
Element of
AFV st
a,
b // a9,
b9 &
a,
c // c9,
b9 holds
b,
c // c9,
a9
definition
let AFV be
WeakAffVect;
let a,
b be
Element of
AFV;
pred MDist a,
b means :
Def2:
(
a,
b // b,
a &
a <> b );
irreflexivity
for a being Element of AFV holds
( not a,a // a,a or not a <> a )
;
symmetry
for a, b being Element of AFV st a,b // b,a & a <> b holds
( b,a // a,b & b <> a )
by Th4;
end;
:: deftheorem Def2 defines MDist AFVECT0:def 2 :
for AFV being WeakAffVect
for a, b being Element of AFV holds
( MDist a,b iff ( a,b // b,a & a <> b ) );
theorem
canceled;
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
:: deftheorem Def3 defines Mid AFVECT0:def 3 :
for AFV being WeakAffVect
for a, b, c being Element of AFV holds
( Mid a,b,c iff a,b // b,c );
theorem
canceled;
theorem Th21:
theorem
theorem Th23:
theorem Th24:
theorem Th25:
theorem Th26:
theorem Th27:
theorem Th28:
theorem Th29:
theorem Th30:
for
AFV being
WeakAffVect for
a,
p,
a9,
b,
b9 being
Element of
AFV st
Mid a,
p,
a9 &
Mid b,
p,
b9 holds
a,
b // b9,
a9
theorem
for
AFV being
WeakAffVect for
a,
p,
a9,
b,
q,
b9 being
Element of
AFV st
Mid a,
p,
a9 &
Mid b,
q,
b9 &
MDist p,
q holds
a,
b // b9,
a9
definition
let AFV be
WeakAffVect;
let a,
b be
Element of
AFV;
func PSym (
a,
b)
-> Element of
AFV means :
Def4:
Mid b,
a,
it;
correctness
existence
ex b1 being Element of AFV st Mid b,a,b1;
uniqueness
for b1, b2 being Element of AFV st Mid b,a,b1 & Mid b,a,b2 holds
b1 = b2;
by Th26, Th27;
end;
:: deftheorem Def4 defines PSym AFVECT0:def 4 :
for AFV being WeakAffVect
for a, b, b4 being Element of AFV holds
( b4 = PSym (a,b) iff Mid b,a,b4 );
theorem
canceled;
theorem
theorem
canceled;
theorem Th35:
theorem Th36:
theorem Th37:
theorem
theorem Th39:
theorem Th40:
for
AFV being
WeakAffVect for
a,
b,
c,
d,
p being
Element of
AFV holds
(
a,
b // c,
d iff
PSym (
p,
a),
PSym (
p,
b)
// PSym (
p,
c),
PSym (
p,
d) )
theorem
theorem Th42:
for
AFV being
WeakAffVect for
a,
b,
c,
p being
Element of
AFV holds
(
Mid a,
b,
c iff
Mid PSym (
p,
a),
PSym (
p,
b),
PSym (
p,
c) )
theorem Th43:
theorem Th44:
theorem
theorem Th46:
theorem
theorem
definition
let AFV be
WeakAffVect;
let o,
a,
b be
Element of
AFV;
func Padd (
o,
a,
b)
-> Element of
AFV means :
Def5:
o,
a // b,
it;
correctness
existence
ex b1 being Element of AFV st o,a // b,b1;
uniqueness
for b1, b2 being Element of AFV st o,a // b,b1 & o,a // b,b2 holds
b1 = b2;
by Def1, Th6;
end;
:: deftheorem Def5 defines Padd AFVECT0:def 5 :
for AFV being WeakAffVect
for o, a, b, b5 being Element of AFV holds
( b5 = Padd (o,a,b) iff o,a // b,b5 );
Lm1:
for AFV being WeakAffVect
for o, a, b being Element of AFV holds
( Pcom (o,a) = b iff a,o // o,b )
definition
let AFV be
WeakAffVect;
let o be
Element of
AFV;
canceled;func Padd o -> BinOp of the
carrier of
AFV means :
Def7:
for
a,
b being
Element of
AFV holds
it . (
a,
b)
= Padd (
o,
a,
b);
existence
ex b1 being BinOp of the carrier of AFV st
for a, b being Element of AFV holds b1 . (a,b) = Padd (o,a,b)
uniqueness
for b1, b2 being BinOp of the carrier of AFV st ( for a, b being Element of AFV holds b1 . (a,b) = Padd (o,a,b) ) & ( for a, b being Element of AFV holds b2 . (a,b) = Padd (o,a,b) ) holds
b1 = b2
end;
:: deftheorem AFVECT0:def 6 :
canceled;
:: deftheorem Def7 defines Padd AFVECT0:def 7 :
for AFV being WeakAffVect
for o being Element of AFV
for b3 being BinOp of the carrier of AFV holds
( b3 = Padd o iff for a, b being Element of AFV holds b3 . (a,b) = Padd (o,a,b) );
:: deftheorem Def8 defines Pcom AFVECT0:def 8 :
for AFV being WeakAffVect
for o being Element of AFV
for b3 being UnOp of the carrier of AFV holds
( b3 = Pcom o iff for a being Element of AFV holds b3 . a = Pcom (o,a) );
:: deftheorem defines GroupVect AFVECT0:def 9 :
for AFV being WeakAffVect
for o being Element of AFV holds GroupVect (AFV,o) = addLoopStr(# the carrier of AFV,(Padd o),o #);
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
canceled;
theorem
Lm2:
for AFV being WeakAffVect
for o being Element of AFV
for a, b being Element of (GroupVect (AFV,o)) holds a + b = b + a
Lm3:
for AFV being WeakAffVect
for o being Element of AFV
for a, b, c being Element of (GroupVect (AFV,o)) holds (a + b) + c = a + (b + c)
Lm4:
for AFV being WeakAffVect
for o being Element of AFV
for a being Element of (GroupVect (AFV,o)) holds a + (0. (GroupVect (AFV,o))) = a
Lm5:
for AFV being WeakAffVect
for o being Element of AFV holds
( GroupVect (AFV,o) is Abelian & GroupVect (AFV,o) is add-associative & GroupVect (AFV,o) is right_zeroed )
Lm6:
for AFV being WeakAffVect
for o being Element of AFV holds GroupVect (AFV,o) is right_complementable
theorem Th58:
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th66:
theorem Th67:
theorem
canceled;
theorem
theorem Th70:
theorem Th71:
theorem
:: deftheorem Def10 defines is_Iso_of AFVECT0:def 10 :
for X, Y being non empty addLoopStr
for f being Function of the carrier of X, the carrier of Y holds
( f is_Iso_of X,Y iff ( f is one-to-one & rng f = the carrier of Y & ( for a, b being Element of X holds
( f . (a + b) = (f . a) + (f . b) & f . (0. X) = 0. Y & f . (- a) = - (f . a) ) ) ) );
:: deftheorem Def11 defines are_Iso AFVECT0:def 11 :
for X, Y being non empty addLoopStr holds
( X,Y are_Iso iff ex f being Function of the carrier of X, the carrier of Y st f is_Iso_of X,Y );
theorem
canceled;
theorem
canceled;
theorem Th75:
theorem Th76:
theorem Th77:
theorem