Lem01:
for a, b, c, d being Real st a <> 0 & b <> 0 & a * d = b * c holds
ex e being Real st
( e = d / b & e = c / a & c = e * a & d = e * b )
Lem02:
for a, b, c, d being Real st a <> 0 & b = 0 & a * d = b * c holds
ex e being Real st
( c = e * a & d = e * b )
theorem
for
a,
b,
c,
d being
Real st (
a <> 0 or
b <> 0 ) &
a * d = b * c holds
ex
e being
Real st
(
c = e * a &
d = e * b )
theorem
for
a,
b,
c being
Real st
(a ^2) + (b ^2) = 1 &
((c * a) ^2) + ((c * b) ^2) = 1 & not
c = 1 holds
c = - 1
theorem
for
a,
b being
Real st
(a ^2) + (b ^2) = 1 &
a = 0 & not
b = 1 holds
b = - 1
Lem03:
for a being Real holds 1 + (a ^2) <> 0
Lem04:
for a, b being Real holds
( not a ^2 = 1 / b or a = 1 / (sqrt b) or a = (- 1) / (sqrt b) )
Lem05:
for z being non zero Complex holds ((1 / z) ^2) * (z ^2) = 1
Lem06:
for a, b, c being Real holds ((a * b) ^2) + ((a * c) ^2) = (a ^2) * ((b ^2) + (c ^2))
;
Lem07:
for a being Real st - 1 < a & a < 1 holds
ex b being Real st (((((1 + (a * a)) * b) * b) - (2 * b)) + 1) - (b * b) = 0
theorem
for
a,
b,
c being
Real st
(a ^2) + (b ^2) = 1 &
- 1
< c &
c < 1 holds
ex
d,
e,
f being
Real st
(
e = ((d * c) * a) + ((1 - d) * (- b)) &
f = ((d * c) * b) + ((1 - d) * a) &
(e ^2) + (f ^2) = d ^2 )
Lem08:
for a, b, c being Real st 0 <= a & c <= 0 holds
0 <= delta (a,b,c)
theorem
for
a,
b,
c,
d being
Real for
u,
v,
w being
Element of
(TOP-REAL 3) st
u = |[a,b,1]| &
v = |[c,d,1]| &
w = |[((a + c) / 2),((b + d) / 2),1]| holds
|{u,v,w}| = 0
Lem09:
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,1) = ((a11 * b11) + (a12 * b21)) + (a13 * b31) & (A * B) * (1,2) = ((a11 * b12) + (a12 * b22)) + (a13 * b32) & (A * B) * (1,3) = ((a11 * b13) + (a12 * b23)) + (a13 * b33) & (A * B) * (2,1) = ((a21 * b11) + (a22 * b21)) + (a23 * b31) & (A * B) * (2,2) = ((a21 * b12) + (a22 * b22)) + (a23 * b32) & (A * B) * (2,3) = ((a21 * b13) + (a22 * b23)) + (a23 * b33) & (A * B) * (3,1) = ((a31 * b11) + (a32 * b21)) + (a33 * b31) & (A * B) * (3,2) = ((a31 * b12) + (a32 * b22)) + (a33 * b32) & (A * B) * (3,3) = ((a31 * b13) + (a32 * b23)) + (a33 * b33) )
theorem
for
a,
b,
c being
Element of
F_Real for
M,
N being
Matrix of 3,
F_Real st
N = <*<*a,0,0*>,<*0,b,0*>,<*0,0,c*>*> holds
(
((M @) * (N * M)) * (1,1)
= (((a * (M * (1,1))) * (M * (1,1))) + ((b * (M * (2,1))) * (M * (2,1)))) + ((c * (M * (3,1))) * (M * (3,1))) &
((M @) * (N * M)) * (1,2)
= (((a * (M * (1,1))) * (M * (1,2))) + ((b * (M * (2,1))) * (M * (2,2)))) + ((c * (M * (3,1))) * (M * (3,2))) &
((M @) * (N * M)) * (1,3)
= (((a * (M * (1,1))) * (M * (1,3))) + ((b * (M * (2,1))) * (M * (2,3)))) + ((c * (M * (3,1))) * (M * (3,3))) &
((M @) * (N * M)) * (2,1)
= (((a * (M * (1,2))) * (M * (1,1))) + ((b * (M * (2,2))) * (M * (2,1)))) + ((c * (M * (3,2))) * (M * (3,1))) &
((M @) * (N * M)) * (2,2)
= (((a * (M * (1,2))) * (M * (1,2))) + ((b * (M * (2,2))) * (M * (2,2)))) + ((c * (M * (3,2))) * (M * (3,2))) &
((M @) * (N * M)) * (2,3)
= (((a * (M * (1,2))) * (M * (1,3))) + ((b * (M * (2,2))) * (M * (2,3)))) + ((c * (M * (3,2))) * (M * (3,3))) &
((M @) * (N * M)) * (3,1)
= (((a * (M * (1,3))) * (M * (1,1))) + ((b * (M * (2,3))) * (M * (2,1)))) + ((c * (M * (3,3))) * (M * (3,1))) &
((M @) * (N * M)) * (3,2)
= (((a * (M * (1,3))) * (M * (1,2))) + ((b * (M * (2,3))) * (M * (2,2)))) + ((c * (M * (3,3))) * (M * (3,2))) &
((M @) * (N * M)) * (3,3)
= (((a * (M * (1,3))) * (M * (1,3))) + ((b * (M * (2,3))) * (M * (2,3)))) + ((c * (M * (3,3))) * (M * (3,3))) )
theorem Th39:
for
r,
a,
b,
c,
d,
e,
f,
g,
h,
i being
Element of
F_Real for
M being
Matrix of 3,
F_Real st
M = <*<*a,b,c*>,<*d,e,f*>,<*g,h,i*>*> holds
r * M = <*<*(r * a),(r * b),(r * c)*>,<*(r * d),(r * e),(r * f)*>,<*(r * g),(r * h),(r * i)*>*>
theorem Th40:
for
a being
Real for
ra2 being
Element of
F_Real st
ra2 = a * a holds
(symmetric_3 (a,a,(- a),0,0,0)) * (symmetric_3 (a,a,(- a),0,0,0)) = ra2 * (1. (F_Real,3))
theorem Th41:
for
a being non
zero Real holds
(symmetric_3 (a,a,(- a),0,0,0)) * (symmetric_3 ((1 / a),(1 / a),(- (1 / a)),0,0,0)) = 1. (
F_Real,3)
theorem Th42:
for
a being non
zero Real holds
(symmetric_3 ((1 / a),(1 / a),(- (1 / a)),0,0,0)) * (symmetric_3 (a,a,(- a),0,0,0)) = 1. (
F_Real,3)
theorem Th43:
(symmetric_3 (1,1,(- 1),0,0,0)) * (symmetric_3 (1,1,(- 1),0,0,0)) = 1. (
F_Real,3)
theorem Th44:
(
symmetric_3 (1,1,
(- 1),
0,
0,
0) is
invertible Matrix of 3,
F_Real &
(symmetric_3 (1,1,(- 1),0,0,0)) ~ = symmetric_3 (1,1,
(- 1),
0,
0,
0) )
theorem Th48:
for
a being
Element of
F_Real holds
symmetric_3 (
a,
a,
(- a),
0,
0,
0)
= a * (symmetric_3 (1,1,(- 1),0,0,0))
theorem Th49:
for
a being
Element of
F_Real for
M being
Matrix of 3,
F_Real st
M = symmetric_3 (
a,
a,
(- a),
0,
0,
0) holds
(M * M) * M = ((a * a) * a) * (symmetric_3 (1,1,(- 1),0,0,0))
theorem
for
NR,
MR being
Matrix of 3,
REAL for
p1,
p2,
p3 being
FinSequence of
REAL st
p1 = <*1,0,0*> &
p2 = <*0,1,0*> &
p3 = <*0,0,1*> &
NR * p1 = MR * p1 &
NR * p2 = MR * p2 &
NR * p3 = MR * p3 holds
NR = MR
definition
let a,
b,
c,
d,
e,
f be
Real;
func negative_conic (
a,
b,
c,
d,
e,
f)
-> Subset of
(ProjectiveSpace (TOP-REAL 3)) equals
{ P where P is Point of (ProjectiveSpace (TOP-REAL 3)) : for u being Element of (TOP-REAL 3) st not u is zero & P = Dir u holds
qfconic (a,b,c,d,e,f,u) is negative } ;
coherence
{ P where P is Point of (ProjectiveSpace (TOP-REAL 3)) : for u being Element of (TOP-REAL 3) st not u is zero & P = Dir u holds
qfconic (a,b,c,d,e,f,u) is negative } is Subset of (ProjectiveSpace (TOP-REAL 3))
end;
::
deftheorem defines
negative_conic BKMODEL1:def 6 :
for a, b, c, d, e, f being Real holds negative_conic (a,b,c,d,e,f) = { P where P is Point of (ProjectiveSpace (TOP-REAL 3)) : for u being Element of (TOP-REAL 3) st not u is zero & P = Dir u holds
qfconic (a,b,c,d,e,f,u) is negative } ;
theorem
for
a,
b,
c,
d,
e,
f being
Real for
u1,
u2 being non
zero Element of
(TOP-REAL 3) st
Dir u1 = Dir u2 &
qfconic (
a,
b,
c,
d,
e,
f,
u1) is
negative holds
qfconic (
a,
b,
c,
d,
e,
f,
u2) is
negative
theorem
for
ra being non
zero Real for
O,
N,
M being
invertible Matrix of 3,
F_Real st
O = symmetric_3 (1,1,
(- 1),
0,
0,
0) &
M = symmetric_3 (
ra,
ra,
(- ra),
0,
0,
0) &
M = ((N @) * O) * N &
(homography M) .: absolute = absolute holds
(homography N) .: absolute = absolute