Skip to content

Commit

Permalink
feat(topology/basic): intersection of a finset-indexed open sets is o…
Browse files Browse the repository at this point in the history
…pen (#16075)
  • Loading branch information
mcdoll committed Aug 17, 2022
1 parent 4a0c497 commit ae132cd
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/topology/basic.lean
Expand Up @@ -147,6 +147,10 @@ lemma is_open_Inter_prop {p : Prop} {s : p → set α}
(h : ∀ h : p, is_open (s h)) : is_open (Inter s) :=
by by_cases p; simp *

lemma is_open_bInter_finset {s : finset β} {f : β → set α} (h : ∀ i ∈ s, is_open (f i)) :
is_open (⋂ i ∈ s, f i) :=
is_open_bInter (to_finite _) h

lemma is_open_const {p : Prop} : is_open {a : α | p} :=
by_cases
(assume : p, begin simp only [this]; exact is_open_univ end)
Expand Down

0 comments on commit ae132cd

Please sign in to comment.