Upper / lower bounds #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
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 #
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
.
Monotonicity #
Conversions #
If s
has a greatest element, then it is bounded above.
Union and intersection #
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
.
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.
Pair #
Lower/upper bounds #
(In)equalities with the least upper bound and the greatest lower bound #
Images of upper/lower bounds under monotone functions #
The image under a monotone function on a set t
of a subset which has an upper bound in t
is bounded above.
The image under a monotone function on a set t
of a subset which has a lower bound in t
is bounded below.
A monotone map sends a greatest element of a set to a greatest element of its image.
An antitone map sends a greatest element of a set to a least element of its image.
An antitone map sends a least element of a set to a greatest element of its image.
A monotone map sends a greatest element of a set to a greatest element of its image.
A function between preorders is said to be Scott continuous if it preserves is_lub
on directed
sets. It can be shown that a function is Scott continuous if and only if it is continuous wrt the
Scott topology.
The dual notion
∀ ⦃d : set α⦄, d.nonempty → directed_on (≥) d → ∀ ⦃a⦄, is_glb d a → is_glb (f '' d) (f a)
does not appear to play a significant role in the literature, so is omitted here.