Skip to content

Commit bafc1ac

Browse files
committed
feat: add MeasurableEmbedding.comap_add (#10795)
Also add a simp attribute to `AbsolutelyContinuous.zero`. Co-authored-by: Rémy Degenne <remydegenne@gmail.com>
1 parent 807b7b4 commit bafc1ac

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

Mathlib/MeasureTheory/Measure/MeasureSpace.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1617,6 +1617,7 @@ instance instIsRefl [MeasurableSpace α] : IsRefl (Measure α) (· ≪ ·) :=
16171617
fun _ => AbsolutelyContinuous.rfl⟩
16181618
#align measure_theory.measure.absolutely_continuous.is_refl MeasureTheory.Measure.AbsolutelyContinuous.instIsRefl
16191619

1620+
@[simp]
16201621
protected lemma zero (μ : Measure α) : 0 ≪ μ := fun s _ ↦ by simp
16211622

16221623
@[trans]
@@ -2123,6 +2124,11 @@ nonrec theorem map_apply (μ : Measure α) (s : Set β) : μ.map f s = μ (f ⁻
21232124
_ = μ (f ⁻¹' s) := by rw [map_apply hf.measurable htm, hft, measure_toMeasurable]
21242125
#align measurable_embedding.map_apply MeasurableEmbedding.map_apply
21252126

2127+
lemma comap_add (μ ν : Measure β) : (μ + ν).comap f = μ.comap f + ν.comap f := by
2128+
ext s hs
2129+
simp only [← comapₗ_eq_comap _ hf.injective (fun _ ↦ hf.measurableSet_image.mpr) _ hs,
2130+
_root_.map_add, add_apply]
2131+
21262132
end MeasurableEmbedding
21272133

21282134
namespace MeasurableEquiv

0 commit comments

Comments
 (0)