Skip to content

Commit 45960ed

Browse files
committed
feat(MeasureTheory): Add mconv_smul_left and mconv_smul_right (#29825)
1 parent 62b471f commit 45960ed

File tree

2 files changed

+18
-0
lines changed

2 files changed

+18
-0
lines changed

Mathlib/MeasureTheory/Group/Convolution.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -91,6 +91,14 @@ theorem mconv_zero (μ : Measure M) : μ ∗ₘ (0 : Measure M) = (0 : Measure M
9191
unfold mconv
9292
simp
9393

94+
-- `mconv_smul_right` needs an instance to get `SFinite (c • ν)` from `SFinite ν`,
95+
-- hence it is placed in the `WithDensity` file, where the instance is defined.
96+
@[to_additive conv_smul_left]
97+
theorem mconv_smul_left (μ : Measure M) (ν : Measure M) [SFinite ν] (s : ℝ≥0∞) :
98+
(s • μ) ∗ₘ ν = s • (μ ∗ₘ ν) := by
99+
unfold mconv
100+
rw [← Measure.map_smul, Measure.prod_smul_left]
101+
94102
@[to_additive]
95103
theorem mconv_add [MeasurableMul₂ M] (μ : Measure M) (ν : Measure M) (ρ : Measure M) [SFinite μ]
96104
[SFinite ν] [SFinite ρ] : μ ∗ₘ (ν + ρ) = μ ∗ₘ ν + μ ∗ₘ ρ := by

Mathlib/MeasureTheory/Measure/WithDensity.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -715,6 +715,16 @@ lemma IsLocallyFiniteMeasure.withDensity_ofReal {f : α → ℝ} (hf : Continuou
715715

716716
section Conv
717717

718+
variable {M : Type*} [Monoid M] [MeasurableSpace M]
719+
720+
-- `mconv_smul_left` is in the `Convolution` file. This lemma is here because this is the file in
721+
-- which we prove the instance that gives `SFinite (c • ν)`.
722+
@[to_additive conv_smul_right]
723+
theorem Measure.mconv_smul_right (μ : Measure M) (ν : Measure M) [SFinite ν] (s : ℝ≥0∞) :
724+
μ ∗ₘ (s • ν) = s • (μ ∗ₘ ν) := by
725+
unfold mconv
726+
rw [Measure.prod_smul_right, Measure.map_smul]
727+
718728
variable {G : Type*} [Group G] [MeasureSpace G] [MeasurableMul₂ G] [MeasurableInv G]
719729
{μ : Measure G} [SFinite μ] [IsMulLeftInvariant μ]
720730

0 commit comments

Comments
 (0)