Zulip Chat Archive
Stream: Is there code for X?
Topic: Covering relation
Yaël Dillies (Nov 22 2021 at 14:44):
Do we agree that we don't have the covering relation?
variables {α : Type*}
def covers [has_le α] (a b : α) : Prop := a ≤ b ∧ ∀ ⦃c⦄, a ≤ c → ¬ c ≤ b
Yury G. Kudryashov (Nov 23 2021 at 04:14):
variables {α : Type*}
def covers [has_le α] (a b : α) : Prop := a ≤ b ∧ ∀ ⦃c⦄, a ≤ c → ¬ c ≤ b
lemma not_covers [preorder α] (a b : α) (h : covers a b) : false :=
begin
cases h with hle h,
apply h hle,
refl
end
Yury G. Kudryashov (Nov 23 2021 at 04:15):
So, with this definition we have it, and it is called λ _ _, false
.
Yaël Dillies (Nov 23 2021 at 09:24):
Whoops sorry! I obviously meant <
:sweat_smile:
Last updated: Dec 20 2023 at 11:08 UTC