theorem Th4:
for
a,
b,
c,
a9,
b9,
c9 being
Complex st ( for
x being
Real holds
Polynom (
a,
b,
c,
x)
= Polynom (
a9,
b9,
c9,
x) ) holds
(
a = a9 &
b = b9 &
c = c9 )
theorem Th5:
for
a,
b,
c being
Real st
a <> 0 &
delta (
a,
b,
c)
>= 0 holds
for
x being
Real holds
( not
Polynom (
a,
b,
c,
x)
= 0 or
x = ((- b) + (sqrt (delta (a,b,c)))) / (2 * a) or
x = ((- b) - (sqrt (delta (a,b,c)))) / (2 * a) )
3 = (2 * 1) + 1
;
then Lm1:
3 is odd
by ABIAN:1;
theorem Th12:
for
a,
a9,
b,
b9,
c,
c9,
d,
d9 being
Real st ( for
x being
Real holds
Polynom (
a,
b,
c,
d,
x)
= Polynom (
a9,
b9,
c9,
d9,
x) ) holds
(
a = a9 &
b = b9 &
c = c9 &
d = d9 )
theorem
for
a,
b,
c,
d,
x1,
x2,
x3 being
Real st
a <> 0 & ( for
x being
Real holds
Polynom (
a,
b,
c,
d,
x)
= Tri (
a,
x1,
x2,
x3,
x) ) holds
(
b / a = - ((x1 + x2) + x3) &
c / a = ((x1 * x2) + (x2 * x3)) + (x1 * x3) &
d / a = - ((x1 * x2) * x3) )
theorem Th15:
for
a,
b,
c,
d,
x being
Real st
a <> 0 &
Polynom (
a,
b,
c,
d,
x)
= 0 holds
for
a1,
a2,
a3,
h,
y being
Real st
y = x + (b / (3 * a)) &
h = - (b / (3 * a)) &
a1 = b / a &
a2 = c / a &
a3 = d / a holds
((y |^ 3) + ((((3 * h) + a1) * (y ^2)) + ((((3 * (h ^2)) + (2 * (a1 * h))) + a2) * y))) + (((h |^ 3) + (a1 * (h ^2))) + ((a2 * h) + a3)) = 0
theorem
for
a,
b,
c,
d,
x being
Real st
a <> 0 &
Polynom (
a,
b,
c,
d,
x)
= 0 holds
for
a1,
a2,
a3,
h,
y being
Real st
y = x + (b / (3 * a)) &
h = - (b / (3 * a)) &
a1 = b / a &
a2 = c / a &
a3 = d / a holds
(((y |^ 3) + (0 * (y ^2))) + (((((3 * a) * c) - (b ^2)) / (3 * (a ^2))) * y)) + ((2 * ((b / (3 * a)) |^ 3)) + ((((3 * a) * d) - (b * c)) / (3 * (a ^2)))) = 0
theorem
for
b,
c,
d,
x being
Real st
b <> 0 &
delta (
b,
c,
d)
> 0 &
Polynom (
0,
b,
c,
d,
x)
= 0 & not
x = ((- c) + (sqrt (delta (b,c,d)))) / (2 * b) holds
x = ((- c) - (sqrt (delta (b,c,d)))) / (2 * b)
theorem
for
a,
c,
d,
p,
q,
x being
Real st
a <> 0 &
p = c / a &
q = d / a &
Polynom (
a,
0,
c,
d,
x)
= 0 holds
for
u,
v being
Real st
x = u + v &
((3 * v) * u) + p = 0 & not
x = (3 -root ((- (d / (2 * a))) + (sqrt (((d ^2) / (4 * (a ^2))) + ((c / (3 * a)) |^ 3))))) + (3 -root ((- (d / (2 * a))) - (sqrt (((d ^2) / (4 * (a ^2))) + ((c / (3 * a)) |^ 3))))) & not
x = (3 -root ((- (d / (2 * a))) + (sqrt (((d ^2) / (4 * (a ^2))) + ((c / (3 * a)) |^ 3))))) + (3 -root ((- (d / (2 * a))) + (sqrt (((d ^2) / (4 * (a ^2))) + ((c / (3 * a)) |^ 3))))) holds
x = (3 -root ((- (d / (2 * a))) - (sqrt (((d ^2) / (4 * (a ^2))) + ((c / (3 * a)) |^ 3))))) + (3 -root ((- (d / (2 * a))) - (sqrt (((d ^2) / (4 * (a ^2))) + ((c / (3 * a)) |^ 3)))))
theorem
for
a,
b,
c,
x being
Real st
a <> 0 &
delta (
a,
b,
c)
>= 0 &
Polynom (
a,
b,
c,
0,
x)
= 0 & not
x = 0 & not
x = ((- b) + (sqrt (delta (a,b,c)))) / (2 * a) holds
x = ((- b) - (sqrt (delta (a,b,c)))) / (2 * a)