Skip to content

Commit

Permalink
feat(ring_theory/polynomial/content): monic polynomials are primitive (
Browse files Browse the repository at this point in the history
…#4862)

Adds the lemma `monic.is_primitive`.
  • Loading branch information
awainverse committed Nov 2, 2020
1 parent ecdc319 commit 556079b
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/ring_theory/polynomial/content.lean
Expand Up @@ -174,6 +174,10 @@ def is_primitive (p : polynomial R) : Prop := p.content = 1
lemma is_primitive_one : is_primitive (1 : polynomial R) :=
by rw [is_primitive, ← C_1, content_C, normalize_one]

lemma monic.is_primitive {p : polynomial R} (hp : p.monic) : p.is_primitive :=
by rw [is_primitive, content_eq_gcd_leading_coeff_content_erase_lead,
hp.leading_coeff, gcd_one_left]

lemma is_primitive.ne_zero {p : polynomial R} (hp : p.is_primitive) : p ≠ 0 :=
begin
rintro rfl,
Expand Down

0 comments on commit 556079b

Please sign in to comment.