Upper / lower bounds
In this file we define:
upper_bounds
,lower_bounds
: the set of upper bounds (resp., lower bounds) of a set;bdd_above s
,bdd_below s
: the sets
is bounded above (resp., below), i.e., the set of upper (resp., lower) bounds ofs
is nonempty;is_least s a
,is_greatest s a
:a
is a least (resp., greatest) element ofs
; for a partial order, it is unique if exists;is_lub s a
,is_glb s a
:a
is a least upper bound (resp., a greatest lower bound) ofs
; for a partial order, it is unique if exists.
We also prove various lemmas about monotonicity, behaviour under ∪
, ∩
, insert
, and provide
formulas for ∅
, univ
, and intervals.
Definitions
The set of upper bounds of a set.
Equations
- upper_bounds s = {x : α | ∀ ⦃a : α⦄, a ∈ s → a ≤ x}
The set of lower bounds of a set.
Equations
- lower_bounds s = {x : α | ∀ ⦃a : α⦄, a ∈ s → x ≤ a}
a
is a greatest element of a set s
; for a partial order, it is unique if exists
Equations
- is_greatest s a = (a ∈ s ∧ a ∈ upper_bounds s)
a
is a greatest lower bound of a set s
; for a partial order, it is unique if exists.
Equations
- is_glb s = is_greatest (lower_bounds s)
A set s
is not bounded above if and only if for each x
there exists y ∈ s
such that x
is not greater than or equal to y
. This version only assumes preorder
structure and uses
¬(y ≤ x)
. A version for linear orders is called not_bdd_above_iff
.
A set s
is not bounded below if and only if for each x
there exists y ∈ s
such that x
is not less than or equal to y
. This version only assumes preorder
structure and uses
¬(x ≤ y)
. A version for linear orders is called not_bdd_below_iff
.
A set s
is not bounded above if and only if for each x
there exists y ∈ s
that is greater
than x
. A version for preorders is called not_bdd_above_iff'
.
A set s
is not bounded below if and only if for each x
there exists y ∈ s
that is less
than x
. A version for preorders is called not_bdd_below_iff'
.
Monotonicity
Conversions
If s
has a greatest element, then it is bounded above.
Union and intersection
If s
and t
are bounded above sets in a semilattice_sup
, then so is s ∪ t
.
The union of two sets is bounded above if and only if each of the sets is.
The union of two sets is bounded above if and only if each of the sets is.
If a
is the least upper bound of s
and b
is the least upper bound of t
,
then a ⊔ b
is the least upper bound of s ∪ t
.
If a
is the greatest lower bound of s
and b
is the greatest lower bound of t
,
then a ⊓ b
is the greatest lower bound of s ∪ t
.
If a
is the least element of s
and b
is the least element of t
,
then min a b
is the least element of s ∪ t
.
If a
is the greatest element of s
and b
is the greatest element of t
,
then max a b
is the greatest element of s ∪ t
.
Specific sets
Unbounded intervals
Singleton
Bounded intervals
Univ
Empty set
insert
Adding a point to a set preserves its boundedness above.
Adding a point to a set preserves its boundedness below.
When there is a global maximum, every set is bounded above.
When there is a global minimum, every set is bounded below.
Pair
(In)equalities with the least upper bound and the greatest lower bound
Images of upper/lower bounds under monotone functions
A monotone map sends a greatest element of a set to a greatest element of its image.