We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 3415a36 commit e518fb0Copy full SHA for e518fb0
Mathlib/Probability/Kernel/Composition/MeasureCompProd.lean
@@ -180,6 +180,12 @@ lemma setLIntegral_compProd [SFinite μ] [IsSFiniteKernel κ]
180
rw [compProd, Kernel.setLIntegral_compProd _ _ _ hf hs ht]
181
simp
182
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
+
189
lemma integrable_compProd_iff [SFinite μ] [IsSFiniteKernel κ] {E : Type*} [NormedAddCommGroup E]
190
{f : α × β → E} (hf : AEStronglyMeasurable f (μ ⊗ₘ κ)) :
191
Integrable f (μ ⊗ₘ κ) ↔
0 commit comments