Skip to content

Commit ce0b441

Browse files
committed
feat(Polynomial): Monic.C_ne_zero (#26508)
shortcut lemma Co-authored-by: Yakov Pechersky <pechersky@users.noreply.github.com>
1 parent df074b2 commit ce0b441

File tree

1 file changed

+5
-1
lines changed

1 file changed

+5
-1
lines changed

Mathlib/Algebra/Polynomial/Degree/Definitions.lean

Lines changed: 5 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -456,7 +456,7 @@ theorem leadingCoeff_one : leadingCoeff (1 : R[X]) = 1 :=
456456
theorem monic_one : Monic (1 : R[X]) :=
457457
leadingCoeff_C _
458458

459-
theorem Monic.ne_zero {R : Type*} [Semiring R] [Nontrivial R] {p : R[X]} (hp : p.Monic) :
459+
theorem Monic.ne_zero [Nontrivial R] {p : R[X]} (hp : p.Monic) :
460460
p ≠ 0 := by
461461
rintro rfl
462462
simp [Monic] at hp
@@ -465,6 +465,10 @@ theorem Monic.ne_zero_of_ne (h : (0 : R) ≠ 1) {p : R[X]} (hp : p.Monic) : p
465465
nontriviality R
466466
exact hp.ne_zero
467467

468+
lemma Monic.ne_zero_of_C [Nontrivial R] {c : R} (hc : Monic (C c)) : c ≠ 0 := by
469+
rintro rfl
470+
simp [Monic] at hc
471+
468472
theorem Monic.ne_zero_of_polynomial_ne {r} (hp : Monic p) (hne : q ≠ r) : p ≠ 0 :=
469473
haveI := Nontrivial.of_polynomial_ne hne
470474
hp.ne_zero

0 commit comments

Comments
 (0)