Zulip Chat Archive

Stream: Is there code for X?

Topic: covBy_iff_lt_iff_le


Violeta Hernández (Oct 28 2024 at 14:25):

Do we by chance have something like this?

import Mathlib.Order.Cover

theorem covBy_iff_lt_iff_le [LinearOrder α] {x y : α} : x  y   {z}, z < y  z  x where
  mp := fun hx _z  hx.le_of_lt, fun hz  hz.trans_lt hx.lt
  mpr := fun H  H.2 le_rfl, fun _z hx hz  (H.1 hz).not_lt hx

Ruben Van de Velde (Oct 28 2024 at 14:31):

@Yaël Dillies

Yaël Dillies (Oct 28 2024 at 14:31):

Not that I know of

Violeta Hernández (Oct 28 2024 at 14:32):

Alright, will PR later

Eric Wieser (Oct 29 2024 at 09:02):

The version with the relations swapped would be good to have too


Last updated: May 02 2025 at 03:31 UTC