Zulip Chat Archive

Stream: Is there code for X?

Topic: finsupp.map_range


Heather Macbeth (Jan 14 2022 at 02:27):

The dfinsupp version of map_range is more flexible than the finsupp version, in that it allows for homomorphisms varying by index:
docs#finsupp.map_range
docs#dfinsupp.map_range
Is there a fast way to get this flexibility in the finsupp case?

import linear_algebra.finsupp

noncomputable theory
variables {ι : Type*} {R : Type*} [ring R]
variables {M : Type*} [add_comm_group M] [module R M]
variables {N : Type*} [add_comm_group N] [module R N]

example (f : ι  (M →ₗ[R] N)) : (ι →₀ M) →ₗ[R] (ι →₀ N) := sorry

Eric Wieser (Jan 14 2022 at 06:42):

Presumably the thing to do is just to modify finsupp.map_range


Last updated: Dec 20 2023 at 11:08 UTC