Zulip Chat Archive
Stream: Is there code for X?
Topic: max with IsCoatom equal top iff
Xavier Roblot (May 04 2025 at 14:19):
Do we have something like this:
import Mathlib
example {α : Type*} {a b : α} [SemilatticeSup α] [OrderTop α] (ha : IsCoatom a) :
a ⊔ b = ⊤ ↔ ¬ b ≤ a := by
by_cases hb : b = ⊤
· simpa [hb] using ha.1
· exact ⟨fun h ↦ left_lt_sup.mp (h ▸ IsCoatom.lt_top ha), fun h ↦ ha.2 _ (left_lt_sup.mpr h)⟩
Last updated: Dec 20 2025 at 21:32 UTC