Skip to content

Commit 629ca6e

Browse files
committed
feat(MeasureTheory/Measure): comap_apply version for measurable equivs (#31398)
This one is stated in terms of the preimage of the inverse, which is sometimes (but not always!) more useful than the image of the forward map.
1 parent 87f042f commit 629ca6e

File tree

1 file changed

+13
-0
lines changed

1 file changed

+13
-0
lines changed

Mathlib/MeasureTheory/Measure/Restrict.lean

Lines changed: 13 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -891,8 +891,21 @@ theorem _root_.MeasurableEquiv.restrict_map (e : α ≃ᵐ β) (μ : Measure α)
891891
(μ.map e).restrict s = (μ.restrict <| e ⁻¹' s).map e :=
892892
e.measurableEmbedding.restrict_map _ _
893893

894+
lemma _root_.MeasurableEquiv.comap_apply (e : α ≃ᵐ β) (μ : Measure β) (s : Set α) :
895+
comap e μ s = μ (e.symm ⁻¹' s) := by
896+
rw [e.measurableEmbedding.comap_apply, e.image_eq_preimage_symm]
897+
894898
end MeasurableEmbedding
895899

900+
lemma MeasureTheory.Measure.map_eq_comap {_ : MeasurableSpace α} {_ : MeasurableSpace β} {f : α → β}
901+
{g : β → α} {μ : Measure α} (hf : Measurable f) (hg : MeasurableEmbedding g)
902+
(hμg : ∀ᵐ a ∂μ, a ∈ Set.range g) (hfg : ∀ a, f (g a) = a) : μ.map f = μ.comap g := by
903+
ext s hs
904+
rw [map_apply hf hs, hg.comap_apply, ← measure_diff_null hμg]
905+
congr
906+
simp
907+
grind
908+
896909
section Subtype
897910

898911
theorem comap_subtype_coe_apply {_m0 : MeasurableSpace α} {s : Set α} (hs : MeasurableSet s)

0 commit comments

Comments
 (0)