Zulip Chat Archive
Stream: Is there code for X?
Topic: Finite chain has a maximal element
Eduardo Freire (Jun 27 2022 at 12:30):
Hello, is there code showing that finite chains have maximal elements? I'm thinking about making a PR to mathlib adding Tukey's lemma and it needs this result, but my current proof of it is quite ugly.
Here is the lemma:
import order.chain
import data.set
lemma max_of_fin_chain {α : Type*} [partial_order α] :
∀ {c : set α}, c.finite → is_chain (≤) c → c.nonempty → ∃m ∈ c, ∀ {b}, b ∈ c → b ≤ m := sorry
Yaël Dillies (Jun 27 2022 at 12:34):
Do you know about docs#finset.exists_min_image, docs#finset.exists_minimal?
Yaël Dillies (Jun 27 2022 at 12:35):
Isn't Tukey's lemma a direct special case of Hausdorff's maximality principle?
Eduardo Freire (Jun 27 2022 at 12:40):
Yaël Dillies said:
Do you know about docs#finset.exists_min_image, docs#finset.exists_minimal?
I didn't, was looking for this thanks
Yaël Dillies (Jun 27 2022 at 12:41):
We're missing a few variants that I was adding the other day. Opening the PR soon.
Eduardo Freire (Jun 27 2022 at 12:58):
Yaël Dillies said:
Isn't Tukey's lemma a direct special case of Hausdorff's maximality principle?
I used zorn_subset_nonempty
instead, not sure if it is more or less direct though :thinking:
Last updated: Dec 20 2023 at 11:08 UTC