File tree Expand file tree Collapse file tree 1 file changed +6
-0
lines changed
Mathlib/MeasureTheory/Measure Expand file tree Collapse file tree 1 file changed +6
-0
lines changed Original file line number Diff line number Diff line change @@ -1617,6 +1617,7 @@ instance instIsRefl [MeasurableSpace α] : IsRefl (Measure α) (· ≪ ·) :=
1617
1617
⟨fun _ => AbsolutelyContinuous.rfl⟩
1618
1618
#align measure_theory.measure.absolutely_continuous.is_refl MeasureTheory.Measure.AbsolutelyContinuous.instIsRefl
1619
1619
1620
+ @[simp]
1620
1621
protected lemma zero (μ : Measure α) : 0 ≪ μ := fun s _ ↦ by simp
1621
1622
1622
1623
@[trans]
@@ -2123,6 +2124,11 @@ nonrec theorem map_apply (μ : Measure α) (s : Set β) : μ.map f s = μ (f ⁻
2123
2124
_ = μ (f ⁻¹' s) := by rw [map_apply hf.measurable htm, hft, measure_toMeasurable]
2124
2125
#align measurable_embedding.map_apply MeasurableEmbedding.map_apply
2125
2126
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
+
2126
2132
end MeasurableEmbedding
2127
2133
2128
2134
namespace MeasurableEquiv
You can’t perform that action at this time.
0 commit comments