Zulip Chat Archive

Stream: Is there code for X?

Topic: Polynomial vs MvPolynomial


Antoine Chambert-Loir (Mar 14 2025 at 18:29):

Is there somewhere in Mathlib the algebraic equivalence of Polynomial R with MvPolynomial Unit R — the unique e : AlgEquiv (Polynomial R) (MvPolynomial Unit R) that sends Polynomial.X to MvPolynomial.X default — as well as the comparison between this isomorphism and evaluations?

Yaël Dillies (Mar 14 2025 at 18:30):

docs#MvPolynomial.pUnitAlgEquiv

Yaël Dillies (Mar 14 2025 at 18:31):

I do not know about the evaluation part

Antoine Chambert-Loir (Mar 14 2025 at 19:04):

At this point, it's not hard

Jireh Loreaux (Mar 14 2025 at 19:37):

Why is that stated with pUnit instead of an arbitrary type with a Unique instance?

Jz Pan (Mar 15 2025 at 07:57):

Yaël Dillies said:

I do not know about the evaluation part

That should be provable just by simp since MvPolynomial.pUnitAlgEquiv has @[simps] lemma

Yaël Dillies (Mar 15 2025 at 08:00):

Not sure what you mean. eval is not a projection of polynomials (nor of mv polynomials). simps only generates lemmas for projections (although it would be cool if that could be extended)

Antoine Chambert-Loir (Mar 15 2025 at 21:21):

Anyway, the lemma is in the PR for evaluation of power series. #15019, I believe.


Last updated: May 02 2025 at 03:31 UTC