Ordering on topologies and (co)induced topologies #
Topologies on a fixed type α are ordered, by reverse inclusion.  That is, for topologies t₁ and
t₂ on α, we write t₁ ≤ t₂ if every set open in t₂ is also open in t₁.  (One also calls
t₁ finer than t₂, and t₂ coarser than t₁.)
Any function f : α → β induces
- TopologicalSpace.induced f : TopologicalSpace β → TopologicalSpace α;
- TopologicalSpace.coinduced f : TopologicalSpace α → TopologicalSpace β.
Continuity, the ordering on topologies and (co)induced topologies are related as follows:
- The identity map (α, t₁) → (α, t₂)is continuous ifft₁ ≤ t₂.
- A map f : (α, t) → (β, u)is continuous- iff t ≤ TopologicalSpace.induced f u(continuous_iff_le_induced)
- iff TopologicalSpace.coinduced f t ≤ u(continuous_iff_coinduced_le).
 
- iff 
Topologies on α form a complete lattice, with ⊥ the discrete topology and ⊤ the indiscrete
topology.
For a function f : α → β, (TopologicalSpace.coinduced f, TopologicalSpace.induced f) is a Galois
connection between topologies on α and topologies on β.
Implementation notes #
There is a Galois insertion between topologies on α (with the inclusion ordering) and all
collections of sets in α. The complete lattice structure on topologies on α is defined as the
reverse of the one obtained via this Galois insertion. More precisely, we use the corresponding
Galois coinsertion between topologies on α (with the reversed inclusion ordering) and collections
of sets in α (with the reversed inclusion ordering).
Tags #
finer, coarser, induced topology, coinduced topology
The open sets of the least topology containing a collection of basic sets.
- basic: ∀ {α : Type u} {g : Set (Set α)}, ∀ s ∈ g, TopologicalSpace.GenerateOpen g s
- univ: ∀ {α : Type u} {g : Set (Set α)}, TopologicalSpace.GenerateOpen g Set.univ
- inter: ∀ {α : Type u} {g : Set (Set α)} (s t : Set α), TopologicalSpace.GenerateOpen g s → TopologicalSpace.GenerateOpen g t → TopologicalSpace.GenerateOpen g (s ∩ t)
- sUnion: ∀ {α : Type u} {g : Set (Set α)} (S : Set (Set α)), (∀ s ∈ S, TopologicalSpace.GenerateOpen g s) → TopologicalSpace.GenerateOpen g (⋃₀ S)
Instances For
The smallest topological space containing the collection g of basic sets
Equations
- TopologicalSpace.generateFrom g = { IsOpen := TopologicalSpace.GenerateOpen g, isOpen_univ := ⋯, isOpen_inter := ⋯, isOpen_sUnion := ⋯ }
Instances For
Alias of the reverse direction of TopologicalSpace.tendsto_nhds_generateFrom_iff.
Construct a topology on α given the filter of neighborhoods of each point of α.
Equations
- TopologicalSpace.mkOfNhds n = { IsOpen := fun (s : Set α) => ∀ a ∈ s, s ∈ n a, isOpen_univ := ⋯, isOpen_inter := ⋯, isOpen_sUnion := ⋯ }
Instances For
The ordering on topologies on the type α. t ≤ s if every set open in s is also open in t
(t is finer than s).
Equations
- TopologicalSpace.instPartialOrder = let __src := PartialOrder.lift (fun (t : TopologicalSpace α) => OrderDual.toDual IsOpen) ⋯; PartialOrder.mk ⋯
If s equals the collection of open sets in the topology it generates, then s defines a
topology.
Equations
- TopologicalSpace.mkOfClosure s hs = { IsOpen := fun (u : Set α) => u ∈ s, isOpen_univ := ⋯, isOpen_inter := ⋯, isOpen_sUnion := ⋯ }
Instances For
The Galois coinsertion between TopologicalSpace α and (Set (Set α))ᵒᵈ whose lower part sends
a topology to its collection of open subsets, and whose upper part sends a collection of subsets
of α to the topology they generate.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Topologies on α form a complete lattice, with ⊥ the discrete topology
and ⊤ the indiscrete topology. The infimum of a collection of topologies
is the topology generated by all their open sets, while the supremum is the
topology whose open sets are those sets open in every member of the collection.
Equations
- TopologicalSpace.instCompleteLattice = (TopologicalSpace.gciGenerateFrom α).liftCompleteLattice
A topological space is discrete if every set is open, that is,
its topology equals the discrete topology ⊥.
- The - TopologicalSpacestructure on a type with discrete topology is equal to- ⊥.
Instances
The TopologicalSpace structure on a type with discrete topology is equal to ⊥.
A function to a discrete topological space is continuous if and only if the preimage of every singleton is open.
Alias of the reverse direction of TopologicalSpace.ext_iff_nhds.
Alias of the reverse direction of TopologicalSpace.ext_iff_nhds.
This lemma characterizes discrete topological spaces as those whose singletons are neighbourhoods.
If the codomain of a continuous injective function has discrete topology, then so does the domain.
See also Embedding.discreteTopology for an important special case.
Equations
- ⋯ = ⋯
Equations
Equations
Equations
Equations
Equations
Equations
Equations
This construction is left adjoint to the operation sending a topology on α
to its neighborhood filter at a fixed point a : α.
Equations
- nhdsAdjoint a f = { IsOpen := fun (s : Set α) => a ∈ s → s ∈ f, isOpen_univ := ⋯, isOpen_inter := ⋯, isOpen_sUnion := ⋯ }
Instances For
Alias of nhds_nhdsAdjoint_same.
Alias of the reverse direction of continuous_generateFrom_iff.