Skip to content

Commit

Permalink
chore(Probability/Kernel/CondCdf): cleanup (#10635)
Browse files Browse the repository at this point in the history
- [x] depends on: #10298 


Co-authored-by: Moritz Firsching <firsching@google.com>
  • Loading branch information
2 people authored and callesonne committed Apr 22, 2024
1 parent a04c5d9 commit 3f80110
Show file tree
Hide file tree
Showing 2 changed files with 23 additions and 22 deletions.
26 changes: 23 additions & 3 deletions Mathlib/Data/Real/Archimedean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,10 +3,10 @@ Copyright (c) 2018 Mario Carneiro. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Floris van Doorn
-/
import Mathlib.Data.Real.Basic
import Mathlib.Data.Set.Image
import Mathlib.Algebra.Order.Archimedean
import Mathlib.Algebra.Bounds
import Mathlib.Algebra.Order.Archimedean
import Mathlib.Data.Real.Basic
import Mathlib.Data.Set.Intervals.Disjoint

#align_import data.real.basic from "leanprover-community/mathlib"@"cb42593171ba005beaaf4549fcfe0dece9ada4c9"

Expand Down Expand Up @@ -346,4 +346,24 @@ theorem iInf_Ioi_eq_iInf_rat_gt {f : ℝ → ℝ} (x : ℝ) (hf : BddBelow (f ''
norm_cast
#align infi_Ioi_eq_infi_rat_gt Real.iInf_Ioi_eq_iInf_rat_gt

theorem not_bddAbove_coe : ¬ (BddAbove <| range (fun (x : ℚ) ↦ (x : ℝ))) := by
dsimp only [BddAbove, upperBounds]
rw [Set.not_nonempty_iff_eq_empty]
ext
simpa using exists_rat_gt _

theorem not_bddBelow_coe : ¬ (BddBelow <| range (fun (x : ℚ) ↦ (x : ℝ))) := by
dsimp only [BddBelow, lowerBounds]
rw [Set.not_nonempty_iff_eq_empty]
ext
simpa using exists_rat_lt _

theorem iUnion_Iic_rat : ⋃ r : ℚ, Iic (r : ℝ) = univ := by
exact iUnion_Iic_of_not_bddAbove_range not_bddAbove_coe
#align real.Union_Iic_rat Real.iUnion_Iic_rat

theorem iInter_Iic_rat : ⋂ r : ℚ, Iic (r : ℝ) = ∅ := by
exact iInter_Iic_eq_empty_iff.mpr not_bddBelow_coe
#align real.Inter_Iic_rat Real.iInter_Iic_rat

end Real
19 changes: 0 additions & 19 deletions Mathlib/Probability/Kernel/CondCdf.lean
Original file line number Diff line number Diff line change
Expand Up @@ -49,25 +49,6 @@ open MeasureTheory Set Filter TopologicalSpace

open scoped NNReal ENNReal MeasureTheory Topology

section AuxLemmasToBeMoved

variable {α β ι : Type*}

theorem Real.iUnion_Iic_rat : ⋃ r : ℚ, Iic (r : ℝ) = univ := by
ext1 x
simp only [mem_iUnion, mem_Iic, mem_univ, iff_true_iff]
obtain ⟨r, hr⟩ := exists_rat_gt x
exact ⟨r, hr.le⟩
#align real.Union_Iic_rat Real.iUnion_Iic_rat

theorem Real.iInter_Iic_rat : ⋂ r : ℚ, Iic (r : ℝ) = ∅ := by
ext1 x
simp only [mem_iInter, mem_Iic, mem_empty_iff_false, iff_false_iff, not_forall, not_le]
exact exists_rat_lt x
#align real.Inter_Iic_rat Real.iInter_Iic_rat

end AuxLemmasToBeMoved

namespace MeasureTheory.Measure

variable {α β : Type*} {mα : MeasurableSpace α} (ρ : Measure (α × ℝ))
Expand Down

0 comments on commit 3f80110

Please sign in to comment.