Intervals #
In any preorder, we define intervals (which on each side can be either infinite, open or closed) using the following naming conventions:
i
: infiniteo
: openc
: closed
Each interval has the name I
+ letter for left side + letter for right side.
For instance, Ioc a b
denotes the interval (a, b]
.
The definitions can be found in Mathlib.Order.Interval.Set.Defs
.
This file contains basic facts on inclusion of and set operations on intervals
(where the precise statements depend on the order's properties;
statements requiring LinearOrder
are in Mathlib.Order.Interval.Set.LinearOrder
).
TODO: This is just the beginning; a lot of rules are missing
Alias of Set.Ici_toDual
.
Alias of Set.Iic_toDual
.
Alias of Set.Ioi_toDual
.
Alias of Set.Iio_toDual
.
Alias of Set.Icc_toDual
.
Alias of Set.Ioc_toDual
.
Alias of Set.Ico_toDual
.
Alias of Set.Ioo_toDual
.
In an order without maximal elements, the intervals Ioi
are nonempty.
In an order without minimal elements, the intervals Iio
are nonempty.
Alias of the reverse direction of Set.Ici_subset_Ici
.
Alias of the reverse direction of Set.Ici_ssubset_Ici
.
Alias of the reverse direction of Set.Iic_subset_Iic
.
Alias of the reverse direction of Set.Iic_ssubset_Iic
.
Alias of the reverse direction of Set.Ioi_eq_empty_iff
.
Alias of the reverse direction of Set.Iio_eq_empty_iff
.
Equations
- Set.instIccUnique = { default := ⟨a, ⋯⟩, uniq := ⋯ }