Zulip Chat Archive

Stream: Is there code for X?

Topic: Alexandrov topologies


Adam Topaz (Jan 29 2025 at 17:31):

We have docs#AlexandrovDiscrete but I can't seem to find the following:

  1. given any partial order on a type X, the upper sets form a (alexandrov) topology on X.
  2. the specialization partial order associated to the topology of (1) is the original partial order.
  3. Any alexandrov topological space arises in this way.

Do we have such things in mathlib?

Adam Topaz (Jan 29 2025 at 17:35):

We do have isOpen_iff_forall_specializes which essentially says that the specialization order determines the topology and vice-versa, but I still don't know how to talk about a poset as a topological space.

Junyan Xu (Jan 29 2025 at 17:40):

The "upper" topology in mathlib seems to be coarser than what you describe according to Topology.IsUpper.isUpperSet_of_isOpen

Adam Topaz (Jan 29 2025 at 17:42):

Ok, I guess I'm looking for docs#Topology.IsUpperSet

Adam Topaz (Jan 29 2025 at 17:42):

and yes I agree that "IsUpper" doesn't coincide with this.

Adam Topaz (Jan 29 2025 at 17:45):

and the synonym WithUpperSet is my (1).

Yaël Dillies (Jan 29 2025 at 17:56):

Are you looking for docs#alexDiscEquivPreord ?

Yaël Dillies (Jan 29 2025 at 17:57):

Adam Topaz said:

I still don't know how to talk about a poset as a topological space.

This is docs#WithUpperSet

Yaël Dillies (Jan 29 2025 at 17:57):

Sorry, I'm blind. You already found it

Adam Topaz (Jan 29 2025 at 17:58):

Yes, thanks!

Yaël Dillies (Jan 29 2025 at 17:59):

The thing we're missing is that T1 Alexandrov discrete <=> partial order. I didn't do it, but it should be easy from what we have

Adam Topaz (Jan 29 2025 at 20:41):

@Yaël Dillies do you know off the top of your head where I can find the lemma that says that, given Topology.IsUpperSet X, that the preorder on X agrees with the specialization order coming from the topology?

Yaël Dillies (Jan 29 2025 at 20:46):

We don't have it, pretty sure

Adam Topaz (Jan 29 2025 at 20:47):

ok, thanks.

Yaël Dillies (Jan 29 2025 at 20:47):

Maybe @Christopher Hoskin has it on a branch, but in any case it should be easy to prove

Adam Topaz (Jan 29 2025 at 20:47):

I mean, we do have Topology.WithUpperSet.toUpperSet_specializes_toUpperSet

Adam Topaz (Jan 29 2025 at 20:50):

Indeed it is easy:

example (x y : X) : x  y  y  x := by
  simp only [specializes_iff_closure_subset,
    Topology.IsUpperSet.closure_singleton, Set.Iic_subset_Iic]

Adam Topaz (Jan 30 2025 at 15:56):

It turns out that I didn’t need the lemma for my application, but I added it anyway: #21263


Last updated: May 02 2025 at 03:31 UTC