Skip to content

Commit

Permalink
feat: MvPolynomial.X_ne_zero (#11071)
Browse files Browse the repository at this point in the history
Proves that a variable is not the zero polynomial, analogous to `Polynomial.X_ne_zero`.
  • Loading branch information
BoltonBailey authored and Louddy committed Apr 15, 2024
1 parent 0b3d803 commit ea91810
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions Mathlib/Data/MvPolynomial/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -818,6 +818,13 @@ theorem ne_zero_iff {p : MvPolynomial σ R} : p ≠ 0 ↔ ∃ d, coeff d p ≠ 0
rfl
#align mv_polynomial.ne_zero_iff MvPolynomial.ne_zero_iff

@[simp]
theorem X_ne_zero [Nontrivial R] (s : σ) :
X (R := R) s ≠ 0 := by
rw [ne_zero_iff]
use Finsupp.single s 1
simp only [coeff_X, ne_eq, one_ne_zero, not_false_eq_true]

@[simp]
theorem support_eq_empty {p : MvPolynomial σ R} : p.support = ∅ ↔ p = 0 :=
Finsupp.support_eq_empty
Expand Down

0 comments on commit ea91810

Please sign in to comment.