Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 3fb9823

Browse files
committed
feat(topology/subset_properties): variant of elim_nhds_subcover for compact_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>
1 parent b3b74f8 commit 3fb9823

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

src/topology/subset_properties.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -495,6 +495,14 @@ lemma cluster_point_of_compact [compact_space α] (f : filter α) [ne_bot f] :
495495
∃ x, cluster_pt x f :=
496496
by simpa using compact_univ (show f ≤ 𝓟 univ, by simp)
497497

498+
lemma compact_space.elim_nhds_subcover {α : Type*} [topological_space α] [compact_space α]
499+
(U : α → set α) (hU : ∀ x, U x ∈ 𝓝 x) :
500+
∃ t : finset α, (⋃ x ∈ t, U x) = ⊤ :=
501+
begin
502+
obtain ⟨t, -, s⟩ := is_compact.elim_nhds_subcover compact_univ U (λ x m, hU x),
503+
exact ⟨t, by { rw eq_top_iff, exact s }⟩,
504+
end
505+
498506
theorem compact_space_of_finite_subfamily_closed {α : Type u} [topological_space α]
499507
(h : Π {ι : Type u} (Z : ι → (set α)), (∀ i, is_closed (Z i)) →
500508
(⋂ i, Z i) = ∅ → ∃ (t : finset ι), (⋂ i ∈ t, Z i) = ∅) :

0 commit comments

Comments
 (0)