Zulip Chat Archive

Stream: Is there code for X?

Topic: polynomials spanned by monomials


Damiano Testa (Jan 10 2022 at 08:43):

Dear All,

is something along these lines already in mathlib? Thanks!

import data.polynomial.basic

variables {R : Type*} [semiring R] {r : R}

open polynomial finset

lemma polynomial.add_submonoid_closure_monomial_eq_top :
  add_submonoid.closure { m : polynomial R |  n a, m = monomial n a} =  :=
sorry

Eric Wieser (Jan 10 2022 at 08:48):

I think I've seen something similar, but I think it was about add_monoid_algebra and single, and possibly also submodule

Riccardo Brasca (Jan 10 2022 at 08:55):

I am with my phone so I it's difficult to search the library, but there is something like this in finsupp

Damiano Testa (Jan 10 2022 at 09:05):

Ok, thank you for your answers: I will keep looking!


Last updated: Dec 20 2023 at 11:08 UTC