File tree Expand file tree Collapse file tree 2 files changed +18
-0
lines changed Expand file tree Collapse file tree 2 files changed +18
-0
lines changed Original file line number Diff line number Diff line change @@ -91,6 +91,14 @@ theorem mconv_zero (μ : Measure M) : μ ∗ₘ (0 : Measure M) = (0 : Measure M
91
91
unfold mconv
92
92
simp
93
93
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
+
94
102
@[to_additive]
95
103
theorem mconv_add [MeasurableMul₂ M] (μ : Measure M) (ν : Measure M) (ρ : Measure M) [SFinite μ]
96
104
[SFinite ν] [SFinite ρ] : μ ∗ₘ (ν + ρ) = μ ∗ₘ ν + μ ∗ₘ ρ := by
Original file line number Diff line number Diff line change @@ -715,6 +715,16 @@ lemma IsLocallyFiniteMeasure.withDensity_ofReal {f : α → ℝ} (hf : Continuou
715
715
716
716
section Conv
717
717
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
+
718
728
variable {G : Type *} [Group G] [MeasureSpace G] [MeasurableMul₂ G] [MeasurableInv G]
719
729
{μ : Measure G} [SFinite μ] [IsMulLeftInvariant μ]
720
730
You can’t perform that action at this time.
0 commit comments