Skip to content

Commit

Permalink
chore(Topology/Bases): minor golf (#6584)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Aug 16, 2023
1 parent 979bb0f commit 6c1ea0d
Showing 1 changed file with 4 additions and 5 deletions.
9 changes: 4 additions & 5 deletions Mathlib/Topology/Bases.lean
Expand Up @@ -230,11 +230,10 @@ theorem IsTopologicalBasis.isOpenMap_iff {β} [TopologicalSpace β] {B : Set (Se
#align topological_space.is_topological_basis.is_open_map_iff TopologicalSpace.IsTopologicalBasis.isOpenMap_iff

theorem IsTopologicalBasis.exists_nonempty_subset {B : Set (Set α)} (hb : IsTopologicalBasis B)
{u : Set α} (hu : u.Nonempty) (ou : IsOpen u) : ∃ v ∈ B, Set.Nonempty v ∧ v ⊆ u := by
cases' hu with x hx
rw [hb.open_eq_sUnion' ou, mem_sUnion] at hx
rcases hx with ⟨v, hv, hxv⟩
exact ⟨v, hv.1, ⟨x, hxv⟩, hv.2
{u : Set α} (hu : u.Nonempty) (ou : IsOpen u) : ∃ v ∈ B, Set.Nonempty v ∧ v ⊆ u :=
let ⟨x, hx⟩ := hu
let ⟨v, vB, xv, vu⟩ := hb.exists_subset_of_mem_open hx ou
⟨v, vB, ⟨x, xv⟩, vu⟩
#align topological_space.is_topological_basis.exists_nonempty_subset TopologicalSpace.IsTopologicalBasis.exists_nonempty_subset

theorem isTopologicalBasis_opens : IsTopologicalBasis { U : Set α | IsOpen U } :=
Expand Down

0 comments on commit 6c1ea0d

Please sign in to comment.