begin
:: deftheorem Def1 defines |' PROJPL_1:def 1 :
for G being IncProjStr
for a, b being POINT of G
for P being LINE of G holds
( a,b |' P iff ( a |' P & b |' P ) );
:: deftheorem Def2 defines on PROJPL_1:def 2 :
for G being IncProjStr
for a being POINT of G
for P, Q being LINE of G holds
( a on P,Q iff ( a on P & a on Q ) );
:: deftheorem Def3 defines on PROJPL_1:def 3 :
for G being IncProjStr
for a being POINT of G
for P, Q, R being LINE of G holds
( a on P,Q,R iff ( a on P & a on Q & a on R ) );
theorem Th1:
for
G being
IncProjStr for
a,
b,
c being
POINT of
G for
P,
Q,
R being
LINE of
G holds
( (
{a,b} on P implies
{b,a} on P ) & (
{a,b,c} on P implies (
{a,c,b} on P &
{b,a,c} on P &
{b,c,a} on P &
{c,a,b} on P &
{c,b,a} on P ) ) & (
a on P,
Q implies
a on Q,
P ) & (
a on P,
Q,
R implies (
a on P,
R,
Q &
a on Q,
P,
R &
a on Q,
R,
P &
a on R,
P,
Q &
a on R,
Q,
P ) ) )
:: deftheorem Def4 defines configuration PROJPL_1:def 4 :
for IT being IncProjStr holds
( IT is configuration iff for p, q being POINT of IT
for P, Q being LINE of IT st p on P & q on P & p on Q & q on Q & not p = q holds
P = Q );
theorem Th2:
theorem Th3:
theorem Th4:
for
G being
IncProjStr holds
(
G is
IncProjSp iff (
G is
configuration & ( for
p,
q being
POINT of
G ex
P being
LINE of
G st
{p,q} on P ) & ex
p being
POINT of
G ex
P being
LINE of
G st
p |' P & ( for
P being
LINE of
G ex
a,
b,
c being
POINT of
G st
(
a,
b,
c are_mutually_different &
{a,b,c} on P ) ) & ( for
a,
b,
c,
d,
p being
POINT of
G for
M,
N,
P,
Q being
LINE of
G st
{a,b,p} on M &
{c,d,p} on N &
{a,c} on P &
{b,d} on Q &
p |' P &
p |' Q &
M <> N holds
ex
q being
POINT of
G st
q on P,
Q ) ) )
:: deftheorem Def5 defines is_collinear PROJPL_1:def 5 :
for G being IncProjStr
for a, b, c being POINT of G holds
( a,b,c is_collinear iff ex P being LINE of G st {a,b,c} on P );
theorem Th5:
theorem
definition
let G be
IncProjStr ;
let a,
b,
c,
d be
POINT of
G;
pred a,
b,
c,
d is_a_quadrangle means :
Def6:
(
a,
b,
c is_a_triangle &
b,
c,
d is_a_triangle &
c,
d,
a is_a_triangle &
d,
a,
b is_a_triangle );
end;
:: deftheorem Def6 defines is_a_quadrangle PROJPL_1:def 6 :
for G being IncProjStr
for a, b, c, d being POINT of G holds
( a,b,c,d is_a_quadrangle iff ( a,b,c is_a_triangle & b,c,d is_a_triangle & c,d,a is_a_triangle & d,a,b is_a_triangle ) );
theorem Th7:
theorem Th8:
theorem Th9:
theorem Th10:
theorem Th11:
for
G being
IncProjStr for
a,
b,
c being
POINT of
G st
a,
b,
c is_collinear holds
(
a,
c,
b is_collinear &
b,
a,
c is_collinear &
b,
c,
a is_collinear &
c,
a,
b is_collinear &
c,
b,
a is_collinear )
theorem
for
G being
IncProjStr for
a,
b,
c being
POINT of
G st
a,
b,
c is_a_triangle holds
(
a,
c,
b is_a_triangle &
b,
a,
c is_a_triangle &
b,
c,
a is_a_triangle &
c,
a,
b is_a_triangle &
c,
b,
a is_a_triangle )
by Th11;
theorem Th13:
for
G being
IncProjStr for
a,
b,
c,
d being
POINT of
G st
a,
b,
c,
d is_a_quadrangle holds
(
a,
c,
b,
d is_a_quadrangle &
b,
a,
c,
d is_a_quadrangle &
b,
c,
a,
d is_a_quadrangle &
c,
a,
b,
d is_a_quadrangle &
c,
b,
a,
d is_a_quadrangle &
a,
b,
d,
c is_a_quadrangle &
a,
c,
d,
b is_a_quadrangle &
b,
a,
d,
c is_a_quadrangle &
b,
c,
d,
a is_a_quadrangle &
c,
a,
d,
b is_a_quadrangle &
c,
b,
d,
a is_a_quadrangle &
a,
d,
b,
c is_a_quadrangle &
a,
d,
c,
b is_a_quadrangle &
b,
d,
a,
c is_a_quadrangle &
b,
d,
c,
a is_a_quadrangle &
c,
d,
a,
b is_a_quadrangle &
c,
d,
b,
a is_a_quadrangle &
d,
a,
b,
c is_a_quadrangle &
d,
a,
c,
b is_a_quadrangle &
d,
b,
a,
c is_a_quadrangle &
d,
b,
c,
a is_a_quadrangle &
d,
c,
a,
b is_a_quadrangle &
d,
c,
b,
a is_a_quadrangle )
theorem Th14:
for
G being
IncProjStr for
a1,
a2,
b1,
b2 being
POINT of
G for
A,
B being
LINE of
G st
G is
configuration &
{a1,a2} on A &
{b1,b2} on B &
a1,
a2 |' B &
b1,
b2 |' A &
a1 <> a2 &
b1 <> b2 holds
a1,
a2,
b1,
b2 is_a_quadrangle
theorem Th15:
definition
let G be
IncProjSp;
mode Quadrangle of
G -> Element of
[: the Points of G, the Points of G, the Points of G, the Points of G:] means
it `1 ,
it `2 ,
it `3 ,
it `4 is_a_quadrangle ;
existence
ex b1 being Element of [: the Points of G, the Points of G, the Points of G, the Points of G:] st b1 `1 ,b1 `2 ,b1 `3 ,b1 `4 is_a_quadrangle
end;
:: deftheorem defines Quadrangle PROJPL_1:def 7 :
for G being IncProjSp
for b2 being Element of [: the Points of G, the Points of G, the Points of G, the Points of G:] holds
( b2 is Quadrangle of G iff b2 `1 ,b2 `2 ,b2 `3 ,b2 `4 is_a_quadrangle );
:: deftheorem Def8 defines * PROJPL_1:def 8 :
for G being IncProjSp
for a, b being POINT of G st a <> b holds
for b4 being LINE of G holds
( b4 = a * b iff {a,b} on b4 );
theorem Th16:
begin
theorem Th17:
theorem Th18:
for
G being
IncProjStr st ex
a,
b,
c,
d being
POINT of
G st
a,
b,
c,
d is_a_quadrangle holds
ex
a,
b,
c being
POINT of
G st
a,
b,
c is_a_triangle
theorem Th19:
theorem Th20:
for
G being
IncProjStr for
a,
b,
c,
d being
POINT of
G for
P,
Q,
R being
LINE of
G st
a,
b,
c,
d is_a_quadrangle &
{a,b} on P &
{a,c} on Q &
{a,d} on R holds
P,
Q,
R are_mutually_different
theorem Th21:
for
G being
IncProjStr for
a,
p,
q,
r being
POINT of
G for
P,
Q,
R,
A being
LINE of
G st
G is
configuration &
a on P,
Q,
R &
P,
Q,
R are_mutually_different &
a |' A &
p on A,
P &
q on A,
Q &
r on A,
R holds
p,
q,
r are_mutually_different
theorem Th22:
for
G being
IncProjStr st
G is
configuration & ( for
p,
q being
POINT of
G ex
M being
LINE of
G st
{p,q} on M ) & ( for
P,
Q being
LINE of
G ex
a being
POINT of
G st
a on P,
Q ) & ex
a,
b,
c,
d being
POINT of
G st
a,
b,
c,
d is_a_quadrangle holds
for
P being
LINE of
G ex
a,
b,
c being
POINT of
G st
(
a,
b,
c are_mutually_different &
{a,b,c} on P )
theorem Th23:
for
G being
IncProjStr holds
(
G is
IncProjectivePlane iff (
G is
configuration & ( for
p,
q being
POINT of
G ex
M being
LINE of
G st
{p,q} on M ) & ( for
P,
Q being
LINE of
G ex
a being
POINT of
G st
a on P,
Q ) & ex
a,
b,
c,
d being
POINT of
G st
a,
b,
c,
d is_a_quadrangle ) )
:: deftheorem Def9 defines * PROJPL_1:def 9 :
for G being IncProjectivePlane
for A, B being LINE of G st A <> B holds
for b4 being POINT of G holds
( b4 = A * B iff b4 on A,B );
theorem Th24:
theorem
begin
theorem Th26:
theorem
theorem Th28:
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th35:
theorem
theorem