Commit 5e75b54 1 parent cf0e331 commit 5e75b54 Copy full SHA for 5e75b54
File tree 1 file changed +9
-0
lines changed
Mathlib/MeasureTheory/Function/LpSpace/DomAct
1 file changed +9
-0
lines changed Original file line number Diff line number Diff line change @@ -50,6 +50,14 @@ theorem smul_Lp_const [IsFiniteMeasure μ] (c : Mᵈᵐᵃ) (a : E) :
50
50
c • Lp.const p μ a = Lp.const p μ a :=
51
51
rfl
52
52
53
+ @[to_additive]
54
+ theorem mk_smul_indicatorConstLp (c : M)
55
+ {s : Set α} (hs : MeasurableSet s) (hμs : μ s ≠ ∞) (b : E) :
56
+ mk c • indicatorConstLp p hs hμs b =
57
+ indicatorConstLp p (hs.preimage <| measurable_const_smul c)
58
+ (by rwa [SMulInvariantMeasure.measure_preimage_smul c hs]) b :=
59
+ rfl
60
+
53
61
instance [SMul N α] [SMulCommClass M N α] [SMulInvariantMeasure N α μ] [MeasurableSMul N α] :
54
62
SMulCommClass Mᵈᵐᵃ Nᵈᵐᵃ (Lp E p μ) :=
55
63
Subtype.val_injective.smulCommClass (fun _ _ ↦ rfl) fun _ _ ↦ rfl
@@ -105,6 +113,7 @@ theorem edist_smul_Lp (c : Mᵈᵐᵃ) (f g : Lp E p μ) : edist (c • f) (c
105
113
106
114
variable [Fact (1 ≤ p)]
107
115
116
+ @[to_additive]
108
117
instance : IsometricSMul Mᵈᵐᵃ (Lp E p μ) := ⟨edist_smul_Lp⟩
109
118
110
119
end SMul
You can’t perform that action at this time.
0 commit comments