Skip to content

Commit 5e75b54

Browse files
committed
feat(LpSpace/DomAct): add a lemma + @[to_additive] (#14488)
1 parent cf0e331 commit 5e75b54

File tree

1 file changed

+9
-0
lines changed
  • Mathlib/MeasureTheory/Function/LpSpace/DomAct

1 file changed

+9
-0
lines changed

Mathlib/MeasureTheory/Function/LpSpace/DomAct/Basic.lean

+9
Original file line numberDiff line numberDiff line change
@@ -50,6 +50,14 @@ theorem smul_Lp_const [IsFiniteMeasure μ] (c : Mᵈᵐᵃ) (a : E) :
5050
c • Lp.const p μ a = Lp.const p μ a :=
5151
rfl
5252

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+
5361
instance [SMul N α] [SMulCommClass M N α] [SMulInvariantMeasure N α μ] [MeasurableSMul N α] :
5462
SMulCommClass Mᵈᵐᵃ Nᵈᵐᵃ (Lp E p μ) :=
5563
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
105113

106114
variable [Fact (1 ≤ p)]
107115

116+
@[to_additive]
108117
instance : IsometricSMul Mᵈᵐᵃ (Lp E p μ) := ⟨edist_smul_Lp⟩
109118

110119
end SMul

0 commit comments

Comments
 (0)