Skip to content

Commit

Permalink
feat(measure_theory/measure_space): add finite_measure_sub instance (
Browse files Browse the repository at this point in the history
  • Loading branch information
JasonKYi committed Jul 12, 2021
1 parent 5ea9a07 commit cde5748
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/measure_theory/measure_space.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1914,6 +1914,9 @@ begin
rw [add_apply, sub_apply h_s_meas h₁, ennreal.sub_add_cancel_of_le (h₁ s h_s_meas)],
end

lemma sub_le : μ - ν ≤ μ :=
Inf_le (measure.le_add_right (le_refl _))

end measure_sub

lemma restrict_sub_eq_restrict_sub_restrict (h_meas_s : measurable_set s) :
Expand Down Expand Up @@ -1978,6 +1981,10 @@ begin
repeat {simp [*]},
end

instance finite_measure_sub [finite_measure μ] : finite_measure (μ - ν) :=
{ measure_univ_lt_top := lt_of_le_of_lt
(measure.sub_le set.univ measurable_set.univ) (measure_lt_top _ _) }

end measure

end measure_theory
Expand Down

0 comments on commit cde5748

Please sign in to comment.