File tree Expand file tree Collapse file tree 1 file changed +5
-1
lines changed
Mathlib/Algebra/Polynomial/Degree Expand file tree Collapse file tree 1 file changed +5
-1
lines changed Original file line number Diff line number Diff line change @@ -456,7 +456,7 @@ theorem leadingCoeff_one : leadingCoeff (1 : R[X]) = 1 :=
456
456
theorem monic_one : Monic (1 : R[X]) :=
457
457
leadingCoeff_C _
458
458
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) :
460
460
p ≠ 0 := by
461
461
rintro rfl
462
462
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
465
465
nontriviality R
466
466
exact hp.ne_zero
467
467
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
+
468
472
theorem Monic.ne_zero_of_polynomial_ne {r} (hp : Monic p) (hne : q ≠ r) : p ≠ 0 :=
469
473
haveI := Nontrivial.of_polynomial_ne hne
470
474
hp.ne_zero
You can’t perform that action at this time.
0 commit comments