Zulip Chat Archive
Stream: Is there code for X?
Topic: exists countable cofinal chain for directed posets
Andrew Yang (Dec 30 2024 at 12:04):
Do we have something like this in mathlib?
import Mathlib.SetTheory.Cardinal.Cofinality
example {α : Type*} [Preorder α] [IsDirected α (· ≤ ·)]
(h : Order.cof (α := α) (· ≤ ·) ≤ .aleph0) :
∃ l : ℕ →o α, IsCofinal (Set.range l) := sorry
Nir Paz (Dec 30 2024 at 15:13):
I don't think we do.
Junyan Xu (Dec 30 2024 at 16:19):
Apparently there is no connection between the two concepts in mathlib
@loogle IsCofinal, Order.cof
loogle (Dec 30 2024 at 16:19):
:shrug: nothing found
Violeta Hernández (Jan 27 2025 at 09:21):
Junyan Xu said:
Apparently there is no connection between the two concepts in mathlib
loogle IsCofinal, Order.cof
IsCofinal
was introduced by me not long ago. My goal is to redefine Order.cof
as the least cardinality of an IsCofinal
subset of a preorder, but I've been busy with other things and haven't quite been able to do that refactor yet.
Violeta Hernández (Jan 27 2025 at 09:34):
As of the original post, we don't currently have anything like that for either IsCofinal
or Order.cof
.
Violeta Hernández (Jan 27 2025 at 09:34):
Closest thing would be the API around docs#Ordinal.IsFundamentalSequence which unfortunately sucks
Last updated: May 02 2025 at 03:31 UTC