Zulip Chat Archive
Stream: general
Topic: initial topology
Anas Himmi (May 20 2020 at 21:36):
is this a good way to define the initial topology?
import topology.order
open topological_space
variables {α : Type*} {β : Type*}
def initial_topology (Y:β → Type*) (T:Π b:β,topological_space (Y b)) (f:Π b:β, (α → (Y b))) : topological_space α :=
generate_from {V | ∃ (b:β) (U) (hU:is_open (T b) U),V=(f b)⁻¹'U}
Mario Carneiro (May 20 2020 at 22:30):
I think you can use the lattice operations to define this
Mario Carneiro (May 20 2020 at 22:36):
def initial_topology (Y : β → Type*) (T : Π b, topological_space (Y b)) (f : Π b, α → Y b) :
topological_space α := ⨆ b, induced (f b) (T b)
Anas Himmi (May 21 2020 at 02:02):
Thank you!
Nicolò Cavalleri (Aug 29 2020 at 15:15):
Was this PRed under some namespace if it was PRed? I cannot find it
Last updated: Dec 20 2023 at 11:08 UTC