Zulip Chat Archive
Stream: Is there code for X?
Topic: Preconnection in sigma
Yaël Dillies (Oct 22 2021 at 08:59):
For X : α → Type*
, how does one get to the fact that the connected components of sigma X
are each in one of the X a
?
Johan Commelin (Oct 22 2021 at 09:41):
I'm assuming that \alpha
is discrete, and X a
carries a topology for each a
?
Yaël Dillies (Oct 22 2021 at 09:43):
Yup, I'm trying to prove
import topology.connected
lemma sigma.is_connected_iff {α : Type*} {X : α → Type*} [∀ a, topological_space (X a)]
{s : set (Σ a, X a)} :
is_connected s ↔ ∃ (a : α) (t : set (X a)), is_connected t ∧ s = sigma.mk _ '' t :=
begin
refine ⟨λ hs, _, _⟩,
{ obtain ⟨⟨a, x⟩, hx⟩ := hs.nonempty,
refine ⟨a, sigma.mk a ⁻¹' s, ⟨⟨x, hx⟩, _⟩, _⟩,
sorry,
sorry
},
{ rintro ⟨a, t, ht, rfl⟩,
exact ht.image _ continuous_sigma_mk.continuous_on }
end
Am I missing discrete α
?
Johan Commelin (Oct 22 2021 at 09:43):
No, I guess you don't need it.
Johan Commelin (Oct 22 2021 at 09:43):
I just wanted to be sure that you weren't doing something weird with a topology on \alpha
Yaël Dillies (Oct 22 2021 at 09:44):
Ah yeah, no
Johan Commelin (Oct 22 2021 at 09:45):
You need to know that sigma.mk _ '' set.univ
is open.
Johan Commelin (Oct 22 2021 at 09:47):
If s
is connected and t
is clopen, then s
is contained in t
or disjoint from t
.
Johan Commelin (Oct 22 2021 at 09:47):
Some variant of that observation should go into mathlib.
Yaël Dillies (Oct 22 2021 at 09:47):
Hmm... >We don't seem to have that yet.
Yaël Dillies (Oct 22 2021 at 09:48):
Also, am I right in thinking the preimage of a preconnected set under a continuous embedding is preconnected?
Johan Commelin (Oct 22 2021 at 10:02):
@Yaël Dillies No, that doesn't work. You can embed a "half-moon" shape into the plane, and pull-back another "half-moon" shape that intersects the other one only at the two tips.
Johan Commelin (Oct 22 2021 at 10:02):
I can make it more precise if that counterexample is too vague.
Johan Commelin (Oct 22 2021 at 10:03):
Alternative: pull-back the area below the graph of sin
under the embedding of the upper half-plane.
Yaël Dillies (Oct 22 2021 at 10:14):
Sad... So I need to add as a condition that the set lies entirely in the range of the embedding.
Johan Commelin (Oct 22 2021 at 10:15):
Where?
Yaël Dillies (Oct 22 2021 at 10:21):
For the preimage to be preconnected
Johan Commelin (Oct 22 2021 at 10:26):
But that lemma is not related to your OP right?
Johan Commelin (Oct 22 2021 at 10:27):
Oh, maybe it is for the version that you posted in code, for your construction of t
Johan Commelin (Oct 22 2021 at 10:28):
If you only want to know that s
is contained in some X a
, that's "easier"
Yaël Dillies (Oct 22 2021 at 10:36):
Oh?
Johan Commelin (Oct 22 2021 at 10:42):
If you have the lemma that I mentioned before, you only need to prove that sigma.mk a '' set.univ
is clopen. But you'll need to do that anyway.
Reid Barton (Oct 22 2021 at 12:41):
Johan Commelin said:
You need to know that
sigma.mk _ '' set.univ
is open.
Yaël Dillies (Oct 22 2021 at 13:52):
Johan Commelin said:
If
s
is connected andt
is clopen, thens
is contained int
or disjoint fromt
.
We don't have that lemma, right?
Yaël Dillies (Oct 22 2021 at 13:54):
Also, how does that help me with is_preconnected (sigma.mk a ⁻¹' s)
? I need to pullback preconnection at point or another, right?
Yaël Dillies (Oct 22 2021 at 14:25):
I pushed, feel free to explain me in further details/finish off yourself.
Last updated: Dec 20 2023 at 11:08 UTC