scheme
EXPermutation{
F1()
-> non
empty set ,
P1[
object ,
object ] } :
provided
A1:
for
x being
Element of
F1() ex
y being
Element of
F1() st
P1[
x,
y]
and A2:
for
y being
Element of
F1() ex
x being
Element of
F1() st
P1[
x,
y]
and A3:
for
x,
y,
x9 being
Element of
F1() st
P1[
x,
y] &
P1[
x9,
y] holds
x = x9
and A4:
for
x,
y,
y9 being
Element of
F1() st
P1[
x,
y] &
P1[
x,
y9] holds
y = y9
Lm1:
for A being non empty set
for f, g, h being Permutation of A st f * g = f * h holds
g = h
Lm2:
for A being non empty set
for f, g, h being Permutation of A st g * f = h * f holds
g = h
theorem Th15:
for
A being non
empty set for
f,
g being
Permutation of
A for
R being
Relation of
[:A,A:] st ( for
a,
b,
x,
y,
z,
t being
Element of
A st
[[x,y],[a,b]] in R &
[[a,b],[z,t]] in R &
a <> b holds
[[x,y],[z,t]] in R ) & ( for
x,
y,
z being
Element of
A holds
[[x,x],[y,z]] in R ) &
f is_FormalIz_of R &
g is_FormalIz_of R holds
f * g is_FormalIz_of R
::
deftheorem defines
is_automorphism_of TRANSGEO:def 3 :
for A being non empty set
for f being Permutation of A
for R being Relation of [:A,A:] holds
( f is_automorphism_of R iff for x, y, z, t being Element of A holds
( [[x,y],[z,t]] in R iff [[(f . x),(f . y)],[(f . z),(f . t)]] in R ) );
theorem
for
A being non
empty set for
f being
Permutation of
A for
R being
Relation of
[:A,A:] st ( for
a,
b,
x,
y,
z,
t being
Element of
A st
[[x,y],[a,b]] in R &
[[a,b],[z,t]] in R &
a <> b holds
[[x,y],[z,t]] in R ) & ( for
x,
y,
z being
Element of
A holds
[[x,x],[y,z]] in R ) &
R is_symmetric_in [:A,A:] &
f is_FormalIz_of R holds
f is_automorphism_of R
definition
let IT be non
empty AffinStruct ;
attr IT is
CongrSpace-like means :
Def5:
( ( for
x,
y,
z,
t,
a,
b being
Element of
IT st
x,
y // a,
b &
a,
b // z,
t &
a <> b holds
x,
y // z,
t ) & ( for
x,
y,
z being
Element of
IT holds
x,
x // y,
z ) & ( for
x,
y,
z,
t being
Element of
IT st
x,
y // z,
t holds
z,
t // x,
y ) & ( for
x,
y being
Element of
IT holds
x,
y // x,
y ) );
end;
::
deftheorem Def5 defines
CongrSpace-like TRANSGEO:def 5 :
for IT being non empty AffinStruct holds
( IT is CongrSpace-like iff ( ( for x, y, z, t, a, b being Element of IT st x,y // a,b & a,b // z,t & a <> b holds
x,y // z,t ) & ( for x, y, z being Element of IT holds x,x // y,z ) & ( for x, y, z, t being Element of IT st x,y // z,t holds
z,t // x,y ) & ( for x, y being Element of IT holds x,y // x,y ) ) );
Lm3:
for CS being CongrSpace holds the CONGR of CS is_reflexive_in [: the carrier of CS, the carrier of CS:]
Lm4:
for CS being CongrSpace holds the CONGR of CS is_symmetric_in [: the carrier of CS, the carrier of CS:]
theorem Th48:
for
OAS being
OAffinSpace for
a,
b,
c,
d being
Element of
OAS holds
( not
a,
b '||' c,
d or
a,
c '||' b,
d or ex
x being
Element of
OAS st
(
a,
c,
x are_collinear &
b,
d,
x are_collinear ) )
Lm5:
for OAS being OAffinSpace
for a, b being Element of OAS
for f being Permutation of the carrier of OAS st f is translation & not a,f . a,b are_collinear holds
( a,b // f . a,f . b & a,f . a // b,f . b )
Lm6:
for OAS being OAffinSpace
for a, b being Element of OAS
for f being Permutation of the carrier of OAS st f is translation & a <> f . a & a,f . a,b are_collinear holds
a,f . a // b,f . b
Lm7:
for OAS being OAffinSpace
for a, b being Element of OAS
for f being Permutation of the carrier of OAS st f is translation & Mid a,f . a,b & a <> f . a holds
a,b // f . a,f . b
Lm8:
for OAS being OAffinSpace
for a, b being Element of OAS
for f being Permutation of the carrier of OAS st f is translation & a <> f . a & b <> f . a & Mid a,b,f . a holds
a,b // f . a,f . b
Lm9:
for OAS being OAffinSpace
for a, b being Element of OAS
for f being Permutation of the carrier of OAS st f is translation & a <> f . a & a,f . a,b are_collinear holds
a,b // f . a,f . b
theorem Th75:
for
AFS being
AffinSpace for
a,
b,
c,
d being
Element of
AFS holds
( not
a,
b // c,
d or
a,
c // b,
d or ex
x being
Element of
AFS st
(
LIN a,
c,
x &
LIN b,
d,
x ) )
theorem Th80:
for
AFS being
AffinSpace for
a,
b,
c,
d1,
d2 being
Element of
AFS st not
LIN a,
b,
c &
a,
b // c,
d1 &
a,
b // c,
d2 &
a,
c // b,
d1 &
a,
c // b,
d2 holds
d1 = d2