Skip to content

Commit cb8ebaf

Browse files
committed
refactor(Probability/Kernel/CondCdf): mv prod_iInter (#10037)
Co-authored-by: Moritz Firsching <firsching@google.com>
1 parent 62acece commit cb8ebaf

File tree

2 files changed

+8
-8
lines changed

2 files changed

+8
-8
lines changed

Mathlib/Data/Set/Lattice.lean

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1989,6 +1989,13 @@ theorem prod_sInter {T : Set (Set β)} (hT : T.Nonempty) (s : Set α) :
19891989
simp_rw [singleton_prod, mem_image, iInter_exists, biInter_and', iInter_iInter_eq_right]
19901990
#align set.prod_sInter Set.prod_sInter
19911991

1992+
theorem prod_iInter {s : Set α} {t : ι → Set β} [hι : Nonempty ι] :
1993+
(s ×ˢ ⋂ i, t i) = ⋂ i, s ×ˢ t i := by
1994+
ext x
1995+
simp only [mem_prod, mem_iInter]
1996+
exact ⟨fun h i => ⟨h.1, h.2 i⟩, fun h => ⟨(h hι.some).1, fun i => (h i).2⟩⟩
1997+
#align prod_Inter Set.prod_iInter
1998+
19921999
end Prod
19932000

19942001
section Image2

Mathlib/Probability/Kernel/CondCdf.lean

Lines changed: 1 addition & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2023 Rémy Degenne. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Rémy Degenne
55
-/
6+
import Mathlib.Data.Set.Lattice
67
import Mathlib.MeasureTheory.Measure.Stieltjes
78
import Mathlib.MeasureTheory.Decomposition.RadonNikodym
89
import Mathlib.MeasureTheory.Constructions.Prod.Basic
@@ -66,14 +67,6 @@ theorem sequence_le (a : α) : f (hf.sequence f (Encodable.encode a + 1)) ≤ f
6667

6768
end Directed
6869

69-
-- todo: move to data/set/lattice next to prod_sUnion or prod_sInter
70-
theorem prod_iInter {s : Set α} {t : ι → Set β} [hι : Nonempty ι] :
71-
(s ×ˢ ⋂ i, t i) = ⋂ i, s ×ˢ t i := by
72-
ext x
73-
simp only [mem_prod, mem_iInter]
74-
exact ⟨fun h i => ⟨h.1, h.2 i⟩, fun h => ⟨(h hι.some).1, fun i => (h i).2⟩⟩
75-
#align prod_Inter prod_iInter
76-
7770
theorem Real.iUnion_Iic_rat : ⋃ r : ℚ, Iic (r : ℝ) = univ := by
7871
ext1 x
7972
simp only [mem_iUnion, mem_Iic, mem_univ, iff_true_iff]

0 commit comments

Comments
 (0)