Partial derivatives of polynomials
This file defines the notion of the formal partial derivative of a polynomial, the derivative with respect to a single variable. This derivative is not connected to the notion of derivative from analysis. It is based purely on the polynomial exponents and coefficients.
Main declarations
mv_polynomial.pderivative i p
: the partial derivative ofp
with respect toi
.
Notation
As in other polynomial files, we typically use the notation:
σ : Type*
(indexing the variables)R : Type*
[comm_ring R]
(the coefficients)s : σ →₀ ℕ
, a function fromσ
toℕ
which is zero away from a finite set. This will give rise to a monomial inmv_polynomial σ R
which mathematicians might callX^s
a : R
i : σ
, with corresponding monomialX i
, often denotedX_i
by mathematiciansp : mv_polynomial σ R
pderivative i p
is the partial derivative of p
with respect to i
Equations
- mv_polynomial.pderivative i = {to_fun := λ (p : mv_polynomial σ R), finsupp.sum p (λ (A : σ →₀ ℕ) (B : R), mv_polynomial.monomial (A - finsupp.single i 1) (B * ↑(⇑A i))), map_add' := _, map_smul' := _}