Skip to content

Commit

Permalink
chore(measure_theory/measure/lebesgue): delete leftovers (#12951)
Browse files Browse the repository at this point in the history
  • Loading branch information
sgouezel committed Mar 26, 2022
1 parent 1111482 commit b7d9166
Showing 1 changed file with 0 additions and 26 deletions.
26 changes: 0 additions & 26 deletions src/measure_theory/measure/lebesgue.lean
Expand Up @@ -468,7 +468,6 @@ begin
(region_between_subset (ae_measurable.mk f hf) (ae_measurable.mk g hg) s)).symm },
end


theorem volume_region_between_eq_integral' [sigma_finite μ]
(f_int : integrable_on f s μ) (g_int : integrable_on g s μ)
(hs : measurable_set s) (hfg : f ≤ᵐ[μ.restrict s] g ) :
Expand All @@ -493,28 +492,3 @@ volume_region_between_eq_integral' f_int g_int hs
((ae_restrict_iff' hs).mpr (eventually_of_forall hfg))

end region_between

/-
section vitali
def vitali_aux_h (x : ℝ) (h : x ∈ Icc (0:ℝ) 1) :
∃ y ∈ Icc (0:ℝ) 1, ∃ q:ℚ, ↑q = x - y :=
⟨x, h, 0, by simp⟩
def vitali_aux (x : ℝ) (h : x ∈ Icc (0:ℝ) 1) : ℝ :=
classical.some (vitali_aux_h x h)
theorem vitali_aux_mem (x : ℝ) (h : x ∈ Icc (0:ℝ) 1) : vitali_aux x h ∈ Icc (0:ℝ) 1 :=
Exists.fst (classical.some_spec (vitali_aux_h x h):_)
theorem vitali_aux_rel (x : ℝ) (h : x ∈ Icc (0:ℝ) 1) :
∃ q:ℚ, ↑q = x - vitali_aux x h :=
Exists.snd (classical.some_spec (vitali_aux_h x h):_)
def vitali : set ℝ := {x | ∃ h, x = vitali_aux x h}
theorem vitali_nonmeasurable : ¬ null_measurable_set measure_space.μ vitali :=
sorry
end vitali
-/

0 comments on commit b7d9166

Please sign in to comment.