Skip to content

Commit

Permalink
feat: port LinearAlgebra.Dfinsupp (#2550)
Browse files Browse the repository at this point in the history
  • Loading branch information
LukasMias committed Mar 2, 2023
1 parent 49552cd commit 8890255
Show file tree
Hide file tree
Showing 3 changed files with 584 additions and 1 deletion.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -910,6 +910,7 @@ import Mathlib.LinearAlgebra.Basic
import Mathlib.LinearAlgebra.Basis
import Mathlib.LinearAlgebra.Basis.Bilinear
import Mathlib.LinearAlgebra.BilinearMap
import Mathlib.LinearAlgebra.Dfinsupp
import Mathlib.LinearAlgebra.Finsupp
import Mathlib.LinearAlgebra.GeneralLinearGroup
import Mathlib.LinearAlgebra.LinearIndependent
Expand Down
5 changes: 4 additions & 1 deletion Mathlib/Data/Dfinsupp/Basic.lean
Expand Up @@ -382,10 +382,13 @@ instance distribMulAction [Monoid γ] [∀ i, AddMonoid (β i)] [∀ i, DistribM

/-- Dependent functions with finite support inherit a module structure from such a structure on
each coordinate. -/
instance [Semiring γ] [∀ i, AddCommMonoid (β i)] [∀ i, Module γ (β i)] : Module γ (Π₀ i, β i) :=
instance module [Semiring γ] [∀ i, AddCommMonoid (β i)] [∀ i, Module γ (β i)] :
Module γ (Π₀ i, β i) :=
{ inferInstanceAs (DistribMulAction γ (Π₀ i, β i)) with
zero_smul := fun c => ext fun i => by simp only [smul_apply, zero_smul, zero_apply]
add_smul := fun c x y => ext fun i => by simp only [add_apply, smul_apply, add_smul] }
#align dfinsupp.module Dfinsupp.module


end Algebra

Expand Down

0 comments on commit 8890255

Please sign in to comment.