theorem bag1a:
for
Z being non
empty set for
B1,
B2 being
bag of
Z holds
(
B1 divides B2 iff ex
B3 being
bag of
Z st
B2 = B1 + B3 )
ro1:
for R being non degenerated comRing
for p, q being Polynomial of R
for a being Element of R st a is_a_root_of p holds
a is_a_root_of p *' q
ZZ1e:
for F being Field
for p, q being non zero Polynomial of F
for a being Element of F st a is_a_root_of p *' q & not a is_a_root_of p holds
a is_a_root_of q
ZZ3b:
for R being domRing
for p, q being Polynomial of R st q divides p holds
Roots q c= Roots p
lemsq:
for R being non degenerated comRing
for p being Polynomial of R holds
( p is square-free iff for q being non constant Polynomial of R holds not q `^ 2 divides p )
lemgcd0:
for R being gcdDomain
for a being Element of R
for g being a_gcd of a, 0. R holds g is_associated_to a
lemgcdh:
for F being Field
for p, q being Element of (Polynom-Ring F) ex a, b being Element of (Polynom-Ring F) st p gcd q = (a * p) + (b * q)
divfin2:
for F being Field
for p being Ppoly of F ex n being Nat st
( card (MonicDivisors p) = n & n <= 2 |^ (deg p) )