Skip to content

Commit

Permalink
feat: add LocallyFinite.smul_{left,right} (#10020)
Browse files Browse the repository at this point in the history
From sphere-eversion. Will be used to show a point-wise version of `SmoothPartitionOfUnity.contMDiff_finsum_smul`.




Co-authored-by: Oliver Nash <github@olivernash.org>
  • Loading branch information
grunweg and ocfnash committed Jan 26, 2024
1 parent e165098 commit 5821f8c
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions Mathlib/Topology/Support.lean
Expand Up @@ -420,4 +420,14 @@ theorem locallyFinite_mulSupport_iff [CommMonoid M] {f : ι → X → M} :
(LocallyFinite fun i ↦ mulSupport <| f i) ↔ LocallyFinite fun i ↦ mulTSupport <| f i :=
⟨LocallyFinite.closure, fun H ↦ H.subset fun _ ↦ subset_closure⟩

theorem LocallyFinite.smul_left [Zero R] [Zero M] [SMulWithZero R M]
{s : ι → X → R} (h : LocallyFinite fun i ↦ support <| s i) (f : ι → X → M) :
LocallyFinite fun i ↦ support <| s i • f i :=
h.subset fun i x ↦ mt <| fun h ↦ by rw [Pi.smul_apply', h, zero_smul]

theorem LocallyFinite.smul_right [Zero M] [SMulZeroClass R M]
{f : ι → X → M} (h : LocallyFinite fun i ↦ support <| f i) (s : ι → X → R) :
LocallyFinite fun i ↦ support <| s i • f i :=
h.subset fun i x ↦ mt <| fun h ↦ by rw [Pi.smul_apply', h, smul_zero]

end LocallyFinite

0 comments on commit 5821f8c

Please sign in to comment.