Skip to content

Commit e518fb0

Browse files
committed
feat: ae strongly measurable with respect to compProd (#22381)
Co-authored-by: EtienneC30 <66847262+EtienneC30@users.noreply.github.com>
1 parent 3415a36 commit e518fb0

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

Mathlib/Probability/Kernel/Composition/MeasureCompProd.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -180,6 +180,12 @@ lemma setLIntegral_compProd [SFinite μ] [IsSFiniteKernel κ]
180180
rw [compProd, Kernel.setLIntegral_compProd _ _ _ hf hs ht]
181181
simp
182182

183+
lemma _root_.MeasureTheory.AEStronglyMeasurable.ae_of_compProd [SFinite μ] [IsSFiniteKernel κ]
184+
{E : Type*} [NormedAddCommGroup E] {f : α → β → E}
185+
(hf : AEStronglyMeasurable f.uncurry (μ ⊗ₘ κ)) :
186+
∀ᵐ x ∂μ, AEStronglyMeasurable (f x) (κ x) := by
187+
simpa using hf.compProd_mk_left
188+
183189
lemma integrable_compProd_iff [SFinite μ] [IsSFiniteKernel κ] {E : Type*} [NormedAddCommGroup E]
184190
{f : α × β → E} (hf : AEStronglyMeasurable f (μ ⊗ₘ κ)) :
185191
Integrable f (μ ⊗ₘ κ) ↔

0 commit comments

Comments
 (0)