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

Commit b7db508

Browse files
committed
feat(analysis/topology/topological_space): basis elements are open
1 parent 6dd2bc0 commit b7db508

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

analysis/topology/topological_space.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -970,6 +970,16 @@ begin
970970
{ rw [hb.2.1], trivial } }
971971
end
972972

973+
lemma is_open_of_is_topological_basis {s : set α} {b : set (set α)}
974+
(hb : is_topological_basis b) (hs : s ∈ b) : _root_.is_open s :=
975+
is_open_iff_mem_nhds.2 $ λ a as,
976+
(mem_nhds_of_is_topological_basis hb).2 ⟨s, hs, as, subset.refl _⟩
977+
978+
lemma mem_basis_subset_of_mem_open {b : set (set α)}
979+
(hb : is_topological_basis b) {a:α} (u : set α) (au : a ∈ u)
980+
(ou : _root_.is_open u) : ∃v ∈ b, a ∈ v ∧ v ⊆ u :=
981+
(mem_nhds_of_is_topological_basis hb).1 $ mem_nhds_sets ou au
982+
973983
variables (α)
974984

975985
/-- A separable space is one with a countable dense subset. -/

0 commit comments

Comments
 (0)