Skip to content

Commit 3b8deac

Browse files
committed
feat: indicator of a null measurable set is aestronglymeasurable (#31158)
1 parent 22a8ffd commit 3b8deac

File tree

1 file changed

+12
-0
lines changed

1 file changed

+12
-0
lines changed

Mathlib/MeasureTheory/Function/StronglyMeasurable/AEStronglyMeasurable.lean

Lines changed: 12 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -505,11 +505,23 @@ theorem _root_.aestronglyMeasurable_indicator_iff [Zero β] {s : Set α} (hs : M
505505
(indicator_ae_eq_restrict_compl hs).trans (indicator_ae_eq_restrict_compl hs).symm
506506
exact ae_of_ae_restrict_of_ae_restrict_compl _ A B
507507

508+
theorem _root_.aestronglyMeasurable_indicator_iff₀
509+
[Zero β] {s : Set α} (hs : NullMeasurableSet s μ) :
510+
AEStronglyMeasurable (indicator s f) μ ↔ AEStronglyMeasurable f (μ.restrict s) := by
511+
rw [← aestronglyMeasurable_congr (indicator_ae_eq_of_ae_eq_set hs.toMeasurable_ae_eq),
512+
aestronglyMeasurable_indicator_iff (measurableSet_toMeasurable ..),
513+
restrict_congr_set hs.toMeasurable_ae_eq]
514+
508515
@[fun_prop, measurability]
509516
protected theorem indicator [Zero β] (hfm : AEStronglyMeasurable f μ) {s : Set α}
510517
(hs : MeasurableSet s) : AEStronglyMeasurable (s.indicator f) μ :=
511518
(aestronglyMeasurable_indicator_iff hs).mpr hfm.restrict
512519

520+
@[fun_prop, measurability]
521+
protected theorem indicator₀ [Zero β] (hfm : AEStronglyMeasurable f μ) {s : Set α}
522+
(hs : NullMeasurableSet s μ) : AEStronglyMeasurable (s.indicator f) μ :=
523+
(aestronglyMeasurable_indicator_iff₀ hs).2 hfm.restrict
524+
513525
theorem nullMeasurableSet_eq_fun {E} [TopologicalSpace E] [MetrizableSpace E] {f g : α → E}
514526
(hf : AEStronglyMeasurable f μ) (hg : AEStronglyMeasurable g μ) :
515527
NullMeasurableSet { x | f x = g x } μ := by

0 commit comments

Comments
 (0)