theorem Th05:
for
a11,
a12,
a13,
a21,
a22,
a23,
a31,
a32,
a33 being
Element of
F_Real for
A being
Matrix of 3,
F_Real st
A = <*<*a11,a12,a13*>,<*a21,a22,a23*>,<*a31,a32,a33*>*> holds
(
Line (
A,1)
= <*a11,a12,a13*> &
Line (
A,2)
= <*a21,a22,a23*> &
Line (
A,3)
= <*a31,a32,a33*> )
theorem Th06:
for
a11,
a12,
a13,
a21,
a22,
a23,
a31,
a32,
a33 being
Element of
F_Real for
A being
Matrix of 3,
F_Real st
A = <*<*a11,a12,a13*>,<*a21,a22,a23*>,<*a31,a32,a33*>*> holds
(
Col (
A,1)
= <*a11,a21,a31*> &
Col (
A,2)
= <*a12,a22,a32*> &
Col (
A,3)
= <*a13,a23,a33*> )
theorem Th07:
for
a11,
a12,
a13,
a21,
a22,
a23,
a31,
a32,
a33,
b11,
b12,
b13,
b21,
b22,
b23,
b31,
b32,
b33 being
Element of
F_Real for
A,
B being
Matrix of 3,
F_Real st
A = <*<*a11,a12,a13*>,<*a21,a22,a23*>,<*a31,a32,a33*>*> &
B = <*<*b11,b12,b13*>,<*b21,b22,b23*>,<*b31,b32,b33*>*> holds
A * B = <*<*(((a11 * b11) + (a12 * b21)) + (a13 * b31)),(((a11 * b12) + (a12 * b22)) + (a13 * b32)),(((a11 * b13) + (a12 * b23)) + (a13 * b33))*>,<*(((a21 * b11) + (a22 * b21)) + (a23 * b31)),(((a21 * b12) + (a22 * b22)) + (a23 * b32)),(((a21 * b13) + (a22 * b23)) + (a23 * b33))*>,<*(((a31 * b11) + (a32 * b21)) + (a33 * b31)),(((a31 * b12) + (a32 * b22)) + (a33 * b32)),(((a31 * b13) + (a32 * b23)) + (a33 * b33))*>*>
theorem Th08:
for
a11,
a12,
a13,
a21,
a22,
a23,
a31,
a32,
a33,
b1,
b2,
b3 being
Element of
F_Real for
A being
Matrix of 3,3,
F_Real for
B being
Matrix of 3,1,
F_Real st
A = <*<*a11,a12,a13*>,<*a21,a22,a23*>,<*a31,a32,a33*>*> &
B = <*<*b1*>,<*b2*>,<*b3*>*> holds
A * B = <*<*(((a11 * b1) + (a12 * b2)) + (a13 * b3))*>,<*(((a21 * b1) + (a22 * b2)) + (a23 * b3))*>,<*(((a31 * b1) + (a32 * b2)) + (a33 * b3))*>*>
Lem01:
for a11, a12, a13, a21, a22, a23, a31, a32, a33, b11, b12, b13, b21, b22, b23, b31, b32, b33 being Element of F_Real
for A, B being Matrix of 3,F_Real st A = <*<*a11,a12,a13*>,<*a21,a22,a23*>,<*a31,a32,a33*>*> & B = <*<*b11,b12,b13*>,<*b21,b22,b23*>,<*b31,b32,b33*>*> holds
( (A * B) . 1 = <*(((a11 * b11) + (a12 * b21)) + (a13 * b31)),(((a11 * b12) + (a12 * b22)) + (a13 * b32)),(((a11 * b13) + (a12 * b23)) + (a13 * b33))*> & (A * B) . 2 = <*(((a21 * b11) + (a22 * b21)) + (a23 * b31)),(((a21 * b12) + (a22 * b22)) + (a23 * b32)),(((a21 * b13) + (a22 * b23)) + (a23 * b33))*> & (A * B) . 3 = <*(((a31 * b11) + (a32 * b21)) + (a33 * b31)),(((a31 * b12) + (a32 * b22)) + (a33 * b32)),(((a31 * b13) + (a32 * b23)) + (a33 * b33))*> )
theorem Th09:
for
a,
b,
c being non
zero Element of
F_Real for
M1,
M2 being
Matrix of 3,
F_Real st
M1 = <*<*a,0,0*>,<*0,b,0*>,<*0,0,c*>*> &
M2 = <*<*(1 / a),0,0*>,<*0,(1 / b),0*>,<*0,0,(1 / c)*>*> holds
(
M1 * M2 = 1. (
F_Real,3) &
M2 * M1 = 1. (
F_Real,3) )
theorem Th10:
for
a,
b,
c being non
zero Element of
F_Real holds
<*<*a,0,0*>,<*0,b,0*>,<*0,0,c*>*> is
invertible Matrix of 3,
F_Real
Lem02:
for i being Nat
for u being Element of (TOP-REAL 3)
for p1 being FinSequence of 1 -tuples_on REAL
for uf being FinSequence of F_Real
for N being Matrix of 3,F_Real st i in Seg 3 & u = uf & p1 = N * uf holds
p1 . i = <*((N * (<*uf*> @)) * (i,1))*>
Lem03:
for i being Nat
for r being Real
for u, v being Element of (TOP-REAL 3)
for pf, uf being FinSequence of F_Real
for N being Matrix of 3,F_Real st i in Seg 3 & u = uf & pf = v & r <> 0 & v = r * u holds
(N * (<*uf*> @)) * (i,1) = (1 / r) * ((Line (N,i)) "*" pf)
Lem04:
for i being Nat
for r being Real
for u, v being Element of (TOP-REAL 3)
for p1 being FinSequence of 1 -tuples_on REAL
for pf, uf being FinSequence of F_Real
for N being Matrix of 3,F_Real st i in Seg 3 & u = uf & pf = v & p1 = N * uf & r <> 0 & v = r * u holds
(p1 . i) . 1 = (1 / r) * ((Line (N,i)) "*" pf)
Lem05:
for i being Nat
for v being Element of (TOP-REAL 3)
for pf being FinSequence of F_Real
for N being Matrix of 3,F_Real st i in Seg 3 & pf = v holds
(Line (N,i)) "*" pf = ((N * pf) . i) . 1
Lem06:
for a being non zero Element of F_Real
for uf being FinSequence of F_Real st len uf = 3 holds
(a * (1. (F_Real,3))) * (<*uf*> @) = a * (<*uf*> @)
set GH3 = GroupHomography3 ;
Lm1:
now for e being Element of GroupHomography3 st e = homography (1. (F_Real,3)) holds
for h being Element of GroupHomography3 holds
( h * e = h & e * h = h )
let e be
Element of
GroupHomography3;
( e = homography (1. (F_Real,3)) implies for h being Element of GroupHomography3 holds
( h * e = h & e * h = h ) )assume A1:
e = homography (1. (F_Real,3))
;
for h being Element of GroupHomography3 holds
( h * e = h & e * h = h )let h be
Element of
GroupHomography3;
( h * e = h & e * h = h )reconsider h1 =
h,
h2 =
e as
Element of
EnsHomography3 ;
consider N1,
N2 being
invertible Matrix of 3,
F_Real such that A10:
h1 = homography N1
and A11:
h2 = homography N2
and A12:
h1 (*) h2 = homography (N1 * N2)
by Def01;
homography (N1 * N2) = homography N1
hence
h * e = h
by Def02, A10, A12;
e * h = hconsider N2,
N1 being
invertible Matrix of 3,
F_Real such that A15:
h2 = homography N2
and A16:
h1 = homography N1
and A17:
h2 (*) h1 = homography (N2 * N1)
by Def01;
homography (N2 * N1) = homography N1
hence
e * h = h
by Def02, A16, A17;
verum
end;
Lm2:
now for e, h, g being Element of GroupHomography3
for N, Ng being invertible Matrix of 3,F_Real st h = homography N & g = homography Ng & Ng = N ~ & e = homography (1. (F_Real,3)) holds
( h * g = e & g * h = e )
let e,
h,
g be
Element of
GroupHomography3;
for N, Ng being invertible Matrix of 3,F_Real st h = homography N & g = homography Ng & Ng = N ~ & e = homography (1. (F_Real,3)) holds
( h * g = e & g * h = e )let N,
Ng be
invertible Matrix of 3,
F_Real;
( h = homography N & g = homography Ng & Ng = N ~ & e = homography (1. (F_Real,3)) implies ( h * g = e & g * h = e ) )assume that A9:
h = homography N
and B1:
g = homography Ng
and B2:
Ng = N ~
and B3:
e = homography (1. (F_Real,3))
;
( h * g = e & g * h = e )reconsider h1 =
h as
Element of
EnsHomography3 ;
A23:
Ng is_reverse_of N
by B2, MATRIX_6:def 4;
reconsider g1 =
g as
Element of
EnsHomography3 ;
consider N1,
N2 being
invertible Matrix of 3,
F_Real such that A19:
h1 = homography N1
and A20:
g1 = homography N2
and A21:
h1 (*) g1 = homography (N1 * N2)
by Def01;
homography (N1 * N2) = homography (N * Ng)
then
h1 (*) g1 = e
by B3, A21, A23, MATRIX_6:def 2;
hence
h * g = e
by Def02;
g * h = econsider N1,
N2 being
invertible Matrix of 3,
F_Real such that A27:
g1 = homography N1
and A28:
h1 = homography N2
and A29:
g1 (*) h1 = homography (N1 * N2)
by Def01;
homography (N1 * N2) = homography (Ng * N)
then
g1 (*) h1 = e
by A29, A23, B3, MATRIX_6:def 2;
hence
g * h = e
by Def02;
verum
end;
set e = homography (1. (F_Real,3));
homography (1. (F_Real,3)) in EnsHomography3
;
then reconsider e = homography (1. (F_Real,3)) as Element of GroupHomography3 ;
definition
coherence
Dir |[1,0,0]| is Point of (ProjectiveSpace (TOP-REAL 3))
by Th11, ANPROJ_1:26;
coherence
Dir |[0,1,0]| is Point of (ProjectiveSpace (TOP-REAL 3))
by Th11, ANPROJ_1:26;
coherence
Dir |[0,0,1]| is Point of (ProjectiveSpace (TOP-REAL 3))
by Th11, ANPROJ_1:26;
coherence
Dir |[1,1,1]| is Point of (ProjectiveSpace (TOP-REAL 3))
by Th11, ANPROJ_1:26;
end;
theorem Th21:
for
N being
invertible Matrix of 3,
F_Real for
a,
b,
c being non
zero Element of
F_Real st
N = <*<*a,0,0*>,<*0,b,0*>,<*0,0,c*>*> holds
(
(homography N) . Dir100 = Dir100 &
(homography N) . Dir010 = Dir010 &
(homography N) . Dir001 = Dir001 )
Lem07:
for a, b, c being Element of F_Real
for P being Point of (ProjectiveSpace (TOP-REAL 3)) st P = Dir |[a,b,c]| & ( a <> 0 or b <> 0 or c <> 0 ) holds
( ( not Dir100 , Dir010 ,P are_collinear implies c <> 0 ) & ( not Dir100 , Dir001 ,P are_collinear implies b <> 0 ) & ( not Dir010 , Dir001 ,P are_collinear implies a <> 0 ) )
theorem Th23:
for
P being
Point of
(ProjectiveSpace (TOP-REAL 3)) st not
Dir100 ,
Dir010 ,
P are_collinear & not
Dir100 ,
Dir001 ,
P are_collinear & not
Dir010 ,
Dir001 ,
P are_collinear holds
ex
a,
b,
c being non
zero Element of
F_Real st
P = Dir |[a,b,c]|
theorem Th24:
for
a,
b,
c,
ia,
ib,
ic being non
zero Element of
F_Real for
P being
Point of
(ProjectiveSpace (TOP-REAL 3)) for
N being
invertible Matrix of 3,
F_Real st
P = Dir |[a,b,c]| &
ia = 1
/ a &
ib = 1
/ b &
ic = 1
/ c &
N = <*<*ia,0,0*>,<*0,ib,0*>,<*0,0,ic*>*> holds
(homography N) . P = Dir |[1,1,1]|
theorem Th25:
for
P being
Point of
(ProjectiveSpace (TOP-REAL 3)) st not
Dir100 ,
Dir010 ,
P are_collinear & not
Dir100 ,
Dir001 ,
P are_collinear & not
Dir010 ,
Dir001 ,
P are_collinear holds
ex
a,
b,
c being non
zero Element of
F_Real st
for
N being
invertible Matrix of 3,
F_Real st
N = <*<*a,0,0*>,<*0,b,0*>,<*0,0,c*>*> holds
(homography N) . P = Dir111
theorem Th26:
for
P1,
P2,
P3,
P4 being
Point of
(ProjectiveSpace (TOP-REAL 3)) st not
P1,
P2,
P3 are_collinear & not
P1,
P2,
P4 are_collinear & not
P1,
P3,
P4 are_collinear & not
P2,
P3,
P4 are_collinear holds
ex
N being
invertible Matrix of 3,
F_Real st
(
(homography N) . P1 = Dir100 &
(homography N) . P2 = Dir010 &
(homography N) . P3 = Dir001 &
(homography N) . P4 = Dir111 )
theorem
for
P1,
P2,
P3,
P4,
Q1,
Q2,
Q3,
Q4 being
Point of
(ProjectiveSpace (TOP-REAL 3)) st not
P1,
P2,
P3 are_collinear & not
P1,
P2,
P4 are_collinear & not
P1,
P3,
P4 are_collinear & not
P2,
P3,
P4 are_collinear & not
Q1,
Q2,
Q3 are_collinear & not
Q1,
Q2,
Q4 are_collinear & not
Q1,
Q3,
Q4 are_collinear & not
Q2,
Q3,
Q4 are_collinear holds
ex
N being
invertible Matrix of 3,
F_Real st
(
(homography N) . P1 = Q1 &
(homography N) . P2 = Q2 &
(homography N) . P3 = Q3 &
(homography N) . P4 = Q4 )