Skip to content

Commit

Permalink
feat(measure_theory/measure_space): if f restricted to s is measu…
Browse files Browse the repository at this point in the history
…rable, then `f` is `ae_measurable` wrt `μ.restrict s` (#8098)
  • Loading branch information
ADedecker committed Jul 7, 2021
1 parent 06f0d51 commit 47c7c01
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions src/measure_theory/measure_space.lean
Expand Up @@ -2436,6 +2436,20 @@ begin
exact ⟨f', measurable.mono hf'_meas hm le_rfl, hff'.symm⟩,
end

lemma ae_measurable_restrict_of_measurable_subtype {s : set α}
(hs : measurable_set s) (hf : measurable (λ x : s, f x)) : ae_measurable f (μ.restrict s) :=
begin
by_cases h : nonempty β,
{ refine ⟨s.piecewise f (λ x, classical.choice h), _, (ae_restrict_iff' hs).mpr $ ae_of_all _
(λ x hx, (piecewise_eq_of_mem s _ _ hx).symm)⟩,
intros t ht,
rw piecewise_preimage,
refine measurable_set.union _ ((measurable_const ht).diff hs),
rw [← subtype.image_preimage_coe, ← preimage_comp],
exact hs.subtype_image (hf ht) },
{ exact (measurable_of_not_nonempty (mt (nonempty.map f) h) f).ae_measurable }
end

end

namespace is_compact
Expand Down

0 comments on commit 47c7c01

Please sign in to comment.