Zulip Chat Archive
Stream: Is there code for X?
Topic: is_atomic_of_well_founded
Scott Morrison (May 05 2022 at 04:36):
Can anyone help me with the following?
import order.atoms
example {α : Type*} [partial_order α] [order_bot α] (h : well_founded ((>) : α → α → Prop)) :
is_atomic α := sorry
Junyan Xu (May 05 2022 at 05:58):
import order.atoms
example {α : Type*} [partial_order α] [order_bot α] (h : well_founded ((<) : α → α → Prop)) :
is_atomic α :=
⟨ λ a, or_iff_not_imp_left.2 $
λ ha, let ⟨b,hb,hm⟩ := h.has_min { b | b ≠ ⊥ ∧ b ≤ a } ⟨a,ha,le_rfl⟩ in
⟨b, ⟨hb.1, λ c, not_imp_not.1 $ λ hc hl, hm c ⟨hc,hl.le.trans hb.2⟩ hl⟩, hb.2⟩ ⟩
Scott Morrison (May 05 2022 at 06:32):
Last updated: Dec 20 2023 at 11:08 UTC