Skip to content

Commit

Permalink
feat: port MeasureTheory.MeasurableSpaceDef (#2108)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Feb 6, 2023
1 parent 55c3ac9 commit 3afc583
Show file tree
Hide file tree
Showing 4 changed files with 577 additions and 5 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -766,6 +766,7 @@ import Mathlib.Mathport.Attributes
import Mathlib.Mathport.Notation
import Mathlib.Mathport.Rename
import Mathlib.Mathport.Syntax
import Mathlib.MeasureTheory.MeasurableSpaceDef
import Mathlib.NumberTheory.ClassNumber.AdmissibleAbsoluteValue
import Mathlib.NumberTheory.Divisors
import Mathlib.NumberTheory.FrobeniusNumber
Expand Down
8 changes: 8 additions & 0 deletions Mathlib/Data/Set/Lattice.lean
Expand Up @@ -1105,6 +1105,14 @@ theorem interₛ_eq_univ {S : Set (Set α)} : ⋂₀ S = univ ↔ ∀ s ∈ S, s
infₛ_eq_top
#align set.sInter_eq_univ Set.interₛ_eq_univ

/-- If all sets in a collection are either `∅` or `Set.univ`, then so is their union. -/
theorem unionₛ_mem_empty_univ {S : Set (Set α)} (h : S ⊆ {∅, univ}) :
⋃₀ S ∈ ({∅, univ} :Set (Set α)) := by
simp only [mem_insert_iff, mem_singleton_iff, or_iff_not_imp_left, unionₛ_eq_empty, not_forall]
rintro ⟨s, hs, hne⟩
obtain rfl : s = univ := (h hs).resolve_left hne
exact univ_subset_iff.1 <| subset_unionₛ_of_mem hs

@[simp]
theorem nonempty_unionₛ {S : Set (Set α)} : (⋃₀S).Nonempty ↔ ∃ s ∈ S, Set.Nonempty s := by
simp [nonempty_iff_ne_empty]
Expand Down

0 comments on commit 3afc583

Please sign in to comment.