Zulip Chat Archive

Stream: Is there code for X?

Topic: the linear equivalence (ι →₀ M) ≃ₗ[A] ⨁ (i : ι), M


Joël Riou (Oct 28 2024 at 22:24):

import Mathlib.Algebra.DirectSum.Module
import Mathlib.Data.Finsupp.ToDFinsupp

open DirectSum

def finsuppLinearEquivDFinsupp (A M ι : Type*) [Ring A] [AddCommGroup M] [Module A M]
    [DecidableEq ι] [ (m : M), Decidable (m  0)]:
    (ι →₀ M) ≃ₗ[A]  (i : ι), M := by
  sorry

We have the additive equivalence finsuppAddEquivDFinsupp, but I do not find the linear equivalence version!?

Eric Wieser (Oct 28 2024 at 22:58):

docs#finsuppLequivDFinsupp

Eric Wieser (Oct 28 2024 at 22:58):

Probably it should be renamed

Joël Riou (Oct 28 2024 at 23:47):

Thanks very much!


Last updated: May 02 2025 at 03:31 UTC