Zulip Chat Archive

Stream: Is there code for X?

Topic: Range of a map out of Finsupp


Robin Carlier (Oct 10 2023 at 13:08):

import Mathlib.LinearAlgebra.Finsupp

universe u v w

lemma span_map (α : Type u) (R : Type v) (M : Type w) [Semiring R] [AddCommMonoid M] [Module R M]
    (f : (α →₀ R) →ₗ[R] M) : LinearMap.range f =
     (a : α), Submodule.span R {f (Finsupp.lsingle (R := R) (M := R) a 1)} := by
  sorry

Is this already somewhere? This looks doable by combining Finsupp.iSup_lsingle_range and Submodule.span_singlenton_eq_rangeas far as I can see


Last updated: Dec 20 2023 at 11:08 UTC