The covering relation #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines the covering relation in an order. b
is said to cover a
if a < b
and there
is no element in between. We say that b
weakly covers a
if a ≤ b
and there is no element
between a
and b
. In a partial order this is equivalent to a ⋖ b ∨ a = b
, in a preorder this
is equivalent to a ⋖ b ∨ (a ≤ b ∧ b ≤ a)
Notation #
a ⋖ b
means thatb
coversa
.a ⩿ b
means thatb
weakly coversa
.
Alias of wcovby_of_le_of_le
.
Alias of the reverse direction of to_dual_wcovby_to_dual_iff
.
Alias of the reverse direction of of_dual_wcovby_of_dual_iff
.
An iff
version of wcovby.eq_or_eq
and wcovby_of_eq_or_eq
.
Alias of the reverse direction of to_dual_covby_to_dual_iff
.
Alias of the reverse direction of of_dual_covby_of_dual_iff
.
Alias of the forward direction of wcovby_iff_covby_or_eq
.
Alias of the forward direction of wcovby_iff_eq_or_covby
.
An iff
version of covby.eq_or_eq
and covby_of_eq_or_eq
.
If a
, b
, c
are consecutive and a < x < c
then x = b
.