Skip to content

Commit

Permalink
feat(topology/subset_properties): variant of elim_nhds_subcover for c…
Browse files Browse the repository at this point in the history
…ompact_space (#7304)

I put this in the `compact_space` namespace, although dot notation won't work so if preferred I can move it back to `_root_`.




Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Apr 22, 2021
1 parent b3b74f8 commit 3fb9823
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/topology/subset_properties.lean
Expand Up @@ -495,6 +495,14 @@ lemma cluster_point_of_compact [compact_space α] (f : filter α) [ne_bot f] :
∃ x, cluster_pt x f :=
by simpa using compact_univ (show f ≤ 𝓟 univ, by simp)

lemma compact_space.elim_nhds_subcover {α : Type*} [topological_space α] [compact_space α]
(U : α → set α) (hU : ∀ x, U x ∈ 𝓝 x) :
∃ t : finset α, (⋃ x ∈ t, U x) = ⊤ :=
begin
obtain ⟨t, -, s⟩ := is_compact.elim_nhds_subcover compact_univ U (λ x m, hU x),
exact ⟨t, by { rw eq_top_iff, exact s }⟩,
end

theorem compact_space_of_finite_subfamily_closed {α : Type u} [topological_space α]
(h : Π {ι : Type u} (Z : ι → (set α)), (∀ i, is_closed (Z i)) →
(⋂ i, Z i) = ∅ → ∃ (t : finset ι), (⋂ i ∈ t, Z i) = ∅) :
Expand Down

0 comments on commit 3fb9823

Please sign in to comment.