Zulip Chat Archive
Stream: Is there code for X?
Topic: connected_space.is_connected_univ
Nicolò Cavalleri (Jun 27 2021 at 18:43):
Is this really not in mathlib?
lemma connected_space.is_connected_univ {α : Type*} [topological_space α] [connected_space α] :
is_connected (univ : set α) := ⟨univ_nonempty, is_preconnected_univ⟩
Adam Topaz (Jun 27 2021 at 18:47):
It should be called docs#is_connected_univ I would guess...
Nicolò Cavalleri (Jun 27 2021 at 18:50):
Shouldn't it be called as in the title with that namespace?
Adam Topaz (Jun 27 2021 at 18:51):
We have things like docs#compact_univ
Adam Topaz (Jun 27 2021 at 18:51):
I think the naming here should follow the same convention
Last updated: Dec 20 2023 at 11:08 UTC