theorem Th1:
for
X being
set holds
(
X = {} or ex
a being
set st
(
{a} = X or ex
a,
b being
set st
(
a <> b &
a in X &
b in X ) ) )
set Z = {1};
Lm1:
1 in {1}
by TARSKI:def 1;
Lm2:
{[1,1,1]} c= [:{1},{1},{1}:]
reconsider Z = {1} as non empty set ;
reconsider RR = {[1,1,1]} as Relation3 of Z by Def1, Lm2;
reconsider CLS = CollStr(# Z,RR #) as non empty CollStr ;
Lm3:
now for a, b, c, p, q, r being Point of CLS holds
( ( ( a = b or a = c or b = c ) implies [a,b,c] in the Collinearity of CLS ) & ( a <> b & [a,b,p] in the Collinearity of CLS & [a,b,q] in the Collinearity of CLS & [a,b,r] in the Collinearity of CLS implies [p,q,r] in the Collinearity of CLS ) )
let a,
b,
c,
p,
q,
r be
Point of
CLS;
( ( ( a = b or a = c or b = c ) implies [a,b,c] in the Collinearity of CLS ) & ( a <> b & [a,b,p] in the Collinearity of CLS & [a,b,q] in the Collinearity of CLS & [a,b,r] in the Collinearity of CLS implies [p,q,r] in the Collinearity of CLS ) )A1:
for
z1,
z2,
z3 being
Point of
CLS holds
[z1,z2,z3] in the
Collinearity of
CLS
hence
( (
a = b or
a = c or
b = c ) implies
[a,b,c] in the
Collinearity of
CLS )
;
( a <> b & [a,b,p] in the Collinearity of CLS & [a,b,q] in the Collinearity of CLS & [a,b,r] in the Collinearity of CLS implies [p,q,r] in the Collinearity of CLS )thus
(
a <> b &
[a,b,p] in the
Collinearity of
CLS &
[a,b,q] in the
Collinearity of
CLS &
[a,b,r] in the
Collinearity of
CLS implies
[p,q,r] in the
Collinearity of
CLS )
by A1;
verum
end;
definition
let IT be non
empty CollStr ;
attr IT is
transitive means :
Def4:
for
a,
b,
p,
q,
r being
Point of
IT st
a <> b &
[a,b,p] in the
Collinearity of
IT &
[a,b,q] in the
Collinearity of
IT &
[a,b,r] in the
Collinearity of
IT holds
[p,q,r] in the
Collinearity of
IT;
end;
::
deftheorem Def4 defines
transitive COLLSP:def 4 :
for IT being non empty CollStr holds
( IT is transitive iff for a, b, p, q, r being Point of IT st a <> b & [a,b,p] in the Collinearity of IT & [a,b,q] in the Collinearity of IT & [a,b,r] in the Collinearity of IT holds
[p,q,r] in the Collinearity of IT );
theorem Th3:
for
CLSP being
CollSp for
a,
b,
p,
q,
r being
Point of
CLSP st
a <> b &
a,
b,
p are_collinear &
a,
b,
q are_collinear &
a,
b,
r are_collinear holds
p,
q,
r are_collinear by Def4;
theorem Th9:
for
CLSP being
CollSp for
a,
b,
p,
q,
r being
Point of
CLSP st
p <> q &
a,
b,
p are_collinear &
a,
b,
q are_collinear &
p,
q,
r are_collinear holds
a,
b,
r are_collinear
set Z = {1,2,3};
set RR = { [i,j,k] where i, j, k is Element of NAT : ( ( i = j or j = k or k = i ) & i in {1,2,3} & j in {1,2,3} & k in {1,2,3} ) } ;
Lm4:
{ [i,j,k] where i, j, k is Element of NAT : ( ( i = j or j = k or k = i ) & i in {1,2,3} & j in {1,2,3} & k in {1,2,3} ) } c= [:{1,2,3},{1,2,3},{1,2,3}:]
reconsider Z = {1,2,3} as non empty set by ENUMSET1:def 1;
reconsider RR = { [i,j,k] where i, j, k is Element of NAT : ( ( i = j or j = k or k = i ) & i in {1,2,3} & j in {1,2,3} & k in {1,2,3} ) } as Relation3 of Z by Def1, Lm4;
reconsider CLS = CollStr(# Z,RR #) as non empty CollStr ;
Lm5:
for a, b, c being Point of CLS holds
( [a,b,c] in RR iff ( ( a = b or b = c or c = a ) & a in Z & b in Z & c in Z ) )
Lm6:
for a, b, c, p, q, r being Point of CLS st a <> b & [a,b,p] in the Collinearity of CLS & [a,b,q] in the Collinearity of CLS & [a,b,r] in the Collinearity of CLS holds
[p,q,r] in the Collinearity of CLS
Lm7:
not for a, b, c being Point of CLS holds a,b,c are_collinear
Lm8:
CLS is CollSp
Lm9:
for CLSP being proper CollSp
for P being LINE of CLSP
for x being set st x in P holds
x is Point of CLSP
:: * COLLINEARITY *
:: *********************