lemmul:
for L being non empty right_complementable add-associative right_zeroed distributive doubleLoopStr
for p, q being Polynomial of L st p <> 0_. L & q <> 0_. L holds
(p *' q) . ((((len p) + (len q)) - 1) -' 1) = (p . ((len p) -' 1)) * (q . ((len q) -' 1))
lemlp1:
for R being non degenerated Ring
for p being non zero Polynomial of R holds { i where i is Nat : p . i <> 0. R } is non empty Subset of NAT
AS0:
for R being Ring
for a being Element of R st a is square holds
a is sum_of_squares
S1:
for R being Ring
for a, b being Element of R st a is sum_of_squares & b is sum_of_squares holds
a + b is sum_of_squares
S2:
for R being commutative Ring
for a, b being Element of R st a is square & b is sum_of_squares holds
a * b is sum_of_squares
SM1:
for R being commutative Ring
for a, b being Element of R st a is square & b is square holds
a * b is square
S3:
for R being commutative Ring
for a, b being Element of R st a is sum_of_squares & b is sum_of_squares holds
a * b is sum_of_squares
SQ0:
for R being Ring holds 0. R in SQ R
;
QS0:
for R being Ring holds 0. R in QS R
;
lemminus:
for R being Ring
for S being Subring of R
for a being Element of R
for b being Element of S st a = b holds
- a = - b
lemminus1:
for R being Ring
for S being Subring of R
for S1 being Subset of R
for S2 being Subset of S st S1 = S2 holds
- S1 = - S2
lemsum:
for R being Ring
for S being Subring of R
for f being FinSequence of R
for g being FinSequence of S st f = g holds
Sum f = Sum g
lemEX:
for S being Subset of F_Real st S = { x where x is Element of REAL : 0 <= x } holds
S is positive_cone
EX:
F_Real is ordered
lemsubpreord:
for R being preordered Ring
for P being Preordering of R
for S being Subring of R
for Q being Subset of S st Q = P /\ the carrier of S holds
Q is prepositive_cone
lemsubord:
for R being ordered Ring
for O being Ordering of R
for S being Subring of R
for Q being Subset of S st Q = O /\ the carrier of S holds
Q is positive_cone
lemminuspoly:
for R being Ring
for a being Element of (Polynom-Ring R)
for b being Polynomial of R st a = b holds
- a = - b
lemlowp1:
for R being non degenerated preordered Ring
for P being Preordering of R
for p, q being non zero Polynomial of R st p . (min* { i where i is Nat : p . i <> 0. R } ) in P & q . (min* { i where i is Nat : q . i <> 0. R } ) in P holds
(p + q) . (min* { i where i is Nat : (p + q) . i <> 0. R } ) in P
lemlowp3:
for R being domRing
for p, q being non zero Polynomial of R holds (p *' q) . (min* { i where i is Nat : (p *' q) . i <> 0. R } ) = (p . (min* { i where i is Nat : p . i <> 0. R } )) * (q . (min* { i where i is Nat : q . i <> 0. R } ))