Skip to content

Commit 39ad44a

Browse files
committed
chore(Algebra/MonoidAlgebra): split Defs.lean further (#28030)
This is a resurrection of #19091. This PR further splits the almost-big file `MonoidAlgebra/Defs.lean` to focus on the ring structure on (`Add`)`MonoidAlgebra`. The following files have been split off: * `MonoidAlgebra/Lift.lean`: definition of `liftNC` * `MonoidAlgebra/Module.lean`: module structure (and some submodule results) * `MonoidAlgebra/Opposite.lean`: results on the `MulOpposite` ring structure I also changed one proof about scalar multiplication by natural numbers, so that it wouldn't need a full on module structure on `Finsupp`. This required adding a pair of lemmas on the definition of multiplying `Finsupp`s by natural numbers. Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
1 parent 67e2d50 commit 39ad44a

File tree

13 files changed

+657
-409
lines changed

13 files changed

+657
-409
lines changed

Mathlib.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -729,8 +729,11 @@ import Mathlib.Algebra.MonoidAlgebra.Degree
729729
import Mathlib.Algebra.MonoidAlgebra.Division
730730
import Mathlib.Algebra.MonoidAlgebra.Grading
731731
import Mathlib.Algebra.MonoidAlgebra.Ideal
732+
import Mathlib.Algebra.MonoidAlgebra.Lift
732733
import Mathlib.Algebra.MonoidAlgebra.MapDomain
734+
import Mathlib.Algebra.MonoidAlgebra.Module
733735
import Mathlib.Algebra.MonoidAlgebra.NoZeroDivisors
736+
import Mathlib.Algebra.MonoidAlgebra.Opposite
734737
import Mathlib.Algebra.MonoidAlgebra.Support
735738
import Mathlib.Algebra.MonoidAlgebra.ToDirectSum
736739
import Mathlib.Algebra.MvPolynomial.Basic

Mathlib/Algebra/Group/Finsupp.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -289,6 +289,10 @@ variable [AddMonoid M]
289289
unless `F i`'s addition is commutative. -/
290290
instance instNatSMul : SMul ℕ (ι →₀ M) where smul n v := v.mapRange (n • ·) (nsmul_zero _)
291291

292+
@[simp, norm_cast] lemma coe_nsmul (n : ℕ) (f : ι →₀ M) : ⇑(n • f) = n • ⇑f := rfl
293+
294+
lemma nsmul_apply (n : ℕ) (f : ι →₀ M) (x : ι) : (n • f) x = n • f x := rfl
295+
292296
instance instAddMonoid : AddMonoid (ι →₀ M) :=
293297
fast_instance% DFunLike.coe_injective.addMonoid _ coe_zero coe_add fun _ _ => rfl
294298

Mathlib/Algebra/MonoidAlgebra/Basic.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -7,6 +7,7 @@ import Mathlib.Algebra.Algebra.Equiv
77
import Mathlib.Algebra.Algebra.NonUnitalHom
88
import Mathlib.Algebra.Module.BigOperators
99
import Mathlib.Algebra.MonoidAlgebra.MapDomain
10+
import Mathlib.Algebra.MonoidAlgebra.Module
1011
import Mathlib.Data.Finsupp.SMul
1112
import Mathlib.LinearAlgebra.Finsupp.SumProd
1213

0 commit comments

Comments
 (0)