mathlib3 documentation

order.bounds.basic

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:

We also prove various lemmas about monotonicity, behaviour under , , insert, and provide formulas for , univ, and intervals.

Definitions #

def upper_bounds {α : Type u} [preorder α] (s : set α) :
set α

The set of upper bounds of a set.

Equations
def lower_bounds {α : Type u} [preorder α] (s : set α) :
set α

The set of lower bounds of a set.

Equations
def bdd_above {α : Type u} [preorder α] (s : set α) :
Prop

A set is bounded above if there exists an upper bound.

Equations
def bdd_below {α : Type u} [preorder α] (s : set α) :
Prop

A set is bounded below if there exists a lower bound.

Equations
def is_least {α : Type u} [preorder α] (s : set α) (a : α) :
Prop

a is a least element of a set s; for a partial order, it is unique if exists.

Equations
def is_greatest {α : Type u} [preorder α] (s : set α) (a : α) :
Prop

a is a greatest element of a set s; for a partial order, it is unique if exists

Equations
def is_lub {α : Type u} [preorder α] (s : set α) :
α Prop

a is a least upper bound of a set s; for a partial order, it is unique if exists.

Equations
def is_glb {α : Type u} [preorder α] (s : set α) :
α Prop

a is a greatest lower bound of a set s; for a partial order, it is unique if exists.

Equations
theorem mem_upper_bounds {α : Type u} [preorder α] {s : set α} {a : α} :
a upper_bounds s (x : α), x s x a
theorem mem_lower_bounds {α : Type u} [preorder α] {s : set α} {a : α} :
a lower_bounds s (x : α), x s a x
theorem mem_upper_bounds_iff_subset_Iic {α : Type u} [preorder α] {s : set α} {a : α} :
theorem mem_lower_bounds_iff_subset_Ici {α : Type u} [preorder α] {s : set α} {a : α} :
theorem bdd_above_def {α : Type u} [preorder α] {s : set α} :
bdd_above s (x : α), (y : α), y s y x
theorem bdd_below_def {α : Type u} [preorder α] {s : set α} :
bdd_below s (x : α), (y : α), y s x y
theorem bot_mem_lower_bounds {α : Type u} [preorder α] [order_bot α] (s : set α) :
theorem top_mem_upper_bounds {α : Type u} [preorder α] [order_top α] (s : set α) :
@[simp]
theorem is_least_bot_iff {α : Type u} [preorder α] {s : set α} [order_bot α] :
@[simp]
theorem is_greatest_top_iff {α : Type u} [preorder α] {s : set α} [order_top α] :
theorem not_bdd_above_iff' {α : Type u} [preorder α] {s : set α} :
¬bdd_above s (x : α), (y : α) (H : y s), ¬y x

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.

theorem not_bdd_below_iff' {α : Type u} [preorder α] {s : set α} :
¬bdd_below s (x : α), (y : α) (H : y s), ¬x y

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.

theorem not_bdd_above_iff {α : Type u_1} [linear_order α] {s : set α} :
¬bdd_above s (x : α), (y : α) (H : y s), x < y

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'.

theorem not_bdd_below_iff {α : Type u_1} [linear_order α] {s : set α} :
¬bdd_below s (x : α), (y : α) (H : y s), y < x

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'.

theorem bdd_above.dual {α : Type u} [preorder α] {s : set α} (h : bdd_above s) :
theorem bdd_below.dual {α : Type u} [preorder α] {s : set α} (h : bdd_below s) :
theorem is_least.dual {α : Type u} [preorder α] {s : set α} {a : α} (h : is_least s a) :
theorem is_greatest.dual {α : Type u} [preorder α] {s : set α} {a : α} (h : is_greatest s a) :
theorem is_lub.dual {α : Type u} [preorder α] {s : set α} {a : α} (h : is_lub s a) :
theorem is_glb.dual {α : Type u} [preorder α] {s : set α} {a : α} (h : is_glb s a) :
@[reducible]
def is_least.order_bot {α : Type u} [preorder α] {s : set α} {a : α} (h : is_least s a) :

If a is the least element of a set s, then subtype s is an order with bottom element.

Equations
@[reducible]
def is_greatest.order_top {α : Type u} [preorder α] {s : set α} {a : α} (h : is_greatest s a) :

If a is the greatest element of a set s, then subtype s is an order with top element.

Equations

Monotonicity #

theorem upper_bounds_mono_set {α : Type u} [preorder α] ⦃s t : set α⦄ (hst : s t) :
theorem lower_bounds_mono_set {α : Type u} [preorder α] ⦃s t : set α⦄ (hst : s t) :
theorem upper_bounds_mono_mem {α : Type u} [preorder α] {s : set α} ⦃a b : α⦄ (hab : a b) :
theorem lower_bounds_mono_mem {α : Type u} [preorder α] {s : set α} ⦃a b : α⦄ (hab : a b) :
theorem upper_bounds_mono {α : Type u} [preorder α] ⦃s t : set α⦄ (hst : s t) ⦃a b : α⦄ (hab : a b) :
theorem lower_bounds_mono {α : Type u} [preorder α] ⦃s t : set α⦄ (hst : s t) ⦃a b : α⦄ (hab : a b) :
theorem bdd_above.mono {α : Type u} [preorder α] ⦃s t : set α⦄ (h : s t) :

If s ⊆ t and t is bounded above, then so is s.

theorem bdd_below.mono {α : Type u} [preorder α] ⦃s t : set α⦄ (h : s t) :

If s ⊆ t and t is bounded below, then so is s.

theorem is_lub.of_subset_of_superset {α : Type u} [preorder α] {a : α} {s t p : set α} (hs : is_lub s a) (hp : is_lub p a) (hst : s t) (htp : t p) :
is_lub t a

If a is a least upper bound for sets s and p, then it is a least upper bound for any set t, s ⊆ t ⊆ p.

theorem is_glb.of_subset_of_superset {α : Type u} [preorder α] {a : α} {s t p : set α} (hs : is_glb s a) (hp : is_glb p a) (hst : s t) (htp : t p) :
is_glb t a

If a is a greatest lower bound for sets s and p, then it is a greater lower bound for any set t, s ⊆ t ⊆ p.

theorem is_least.mono {α : Type u} [preorder α] {s t : set α} {a b : α} (ha : is_least s a) (hb : is_least t b) (hst : s t) :
b a
theorem is_greatest.mono {α : Type u} [preorder α] {s t : set α} {a b : α} (ha : is_greatest s a) (hb : is_greatest t b) (hst : s t) :
a b
theorem is_lub.mono {α : Type u} [preorder α] {s t : set α} {a b : α} (ha : is_lub s a) (hb : is_lub t b) (hst : s t) :
a b
theorem is_glb.mono {α : Type u} [preorder α] {s t : set α} {a b : α} (ha : is_glb s a) (hb : is_glb t b) (hst : s t) :
b a

Conversions #

theorem is_least.is_glb {α : Type u} [preorder α] {s : set α} {a : α} (h : is_least s a) :
is_glb s a
theorem is_greatest.is_lub {α : Type u} [preorder α] {s : set α} {a : α} (h : is_greatest s a) :
is_lub s a
theorem is_lub.upper_bounds_eq {α : Type u} [preorder α] {s : set α} {a : α} (h : is_lub s a) :
theorem is_glb.lower_bounds_eq {α : Type u} [preorder α] {s : set α} {a : α} (h : is_glb s a) :
theorem is_least.lower_bounds_eq {α : Type u} [preorder α] {s : set α} {a : α} (h : is_least s a) :
theorem is_greatest.upper_bounds_eq {α : Type u} [preorder α] {s : set α} {a : α} (h : is_greatest s a) :
theorem is_lub_le_iff {α : Type u} [preorder α] {s : set α} {a b : α} (h : is_lub s a) :
theorem le_is_glb_iff {α : Type u} [preorder α] {s : set α} {a b : α} (h : is_glb s a) :
theorem is_lub_iff_le_iff {α : Type u} [preorder α] {s : set α} {a : α} :
is_lub s a (b : α), a b b upper_bounds s
theorem is_glb_iff_le_iff {α : Type u} [preorder α] {s : set α} {a : α} :
is_glb s a (b : α), b a b lower_bounds s
theorem is_lub.bdd_above {α : Type u} [preorder α] {s : set α} {a : α} (h : is_lub s a) :

If s has a least upper bound, then it is bounded above.

theorem is_glb.bdd_below {α : Type u} [preorder α] {s : set α} {a : α} (h : is_glb s a) :

If s has a greatest lower bound, then it is bounded below.

theorem is_greatest.bdd_above {α : Type u} [preorder α] {s : set α} {a : α} (h : is_greatest s a) :

If s has a greatest element, then it is bounded above.

theorem is_least.bdd_below {α : Type u} [preorder α] {s : set α} {a : α} (h : is_least s a) :

If s has a least element, then it is bounded below.

theorem is_least.nonempty {α : Type u} [preorder α] {s : set α} {a : α} (h : is_least s a) :
theorem is_greatest.nonempty {α : Type u} [preorder α] {s : set α} {a : α} (h : is_greatest s a) :

Union and intersection #

@[simp]
theorem upper_bounds_union {α : Type u} [preorder α] {s t : set α} :
@[simp]
theorem lower_bounds_union {α : Type u} [preorder α] {s t : set α} :
theorem is_least_union_iff {α : Type u} [preorder α] {a : α} {s t : set α} :
theorem is_greatest_union_iff {α : Type u} [preorder α] {s t : set α} {a : α} :
theorem bdd_above.inter_of_left {α : Type u} [preorder α] {s t : set α} (h : bdd_above s) :

If s is bounded, then so is s ∩ t

theorem bdd_above.inter_of_right {α : Type u} [preorder α] {s t : set α} (h : bdd_above t) :

If t is bounded, then so is s ∩ t

theorem bdd_below.inter_of_left {α : Type u} [preorder α] {s t : set α} (h : bdd_below s) :

If s is bounded, then so is s ∩ t

theorem bdd_below.inter_of_right {α : Type u} [preorder α] {s t : set α} (h : bdd_below t) :

If t is bounded, then so is s ∩ t

theorem bdd_above.union {α : Type u} [preorder α] [is_directed α has_le.le] {s t : set α} :

In a directed order, the union of bounded above sets is bounded above.

theorem bdd_above_union {α : Type u} [preorder α] [is_directed α has_le.le] {s t : set α} :

In a directed order, the union of two sets is bounded above if and only if both sets are.

theorem bdd_below.union {α : Type u} [preorder α] [is_directed α ge] {s t : set α} :

In a codirected order, the union of bounded below sets is bounded below.

theorem bdd_below_union {α : Type u} [preorder α] [is_directed α ge] {s t : set α} :

In a codirected order, the union of two sets is bounded below if and only if both sets are.

theorem is_lub.union {γ : Type w} [semilattice_sup γ] {a b : γ} {s t : set γ} (hs : is_lub s a) (ht : is_lub t b) :
is_lub (s t) (a b)

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.

theorem is_glb.union {γ : Type w} [semilattice_inf γ] {a₁ a₂ : γ} {s t : set γ} (hs : is_glb s a₁) (ht : is_glb t a₂) :
is_glb (s t) (a₁ a₂)

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.

theorem is_least.union {γ : Type w} [linear_order γ] {a b : γ} {s t : set γ} (ha : is_least s a) (hb : is_least t b) :

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.

theorem is_greatest.union {γ : Type w} [linear_order γ] {a b : γ} {s t : set γ} (ha : is_greatest s a) (hb : is_greatest t b) :

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.

theorem is_lub.inter_Ici_of_mem {γ : Type w} [linear_order γ] {s : set γ} {a b : γ} (ha : is_lub s a) (hb : b s) :
theorem is_glb.inter_Iic_of_mem {γ : Type w} [linear_order γ] {s : set γ} {a b : γ} (ha : is_glb s a) (hb : b s) :
theorem bdd_above_iff_exists_ge {γ : Type w} [semilattice_sup γ] {s : set γ} (x₀ : γ) :
bdd_above s (x : γ), x₀ x (y : γ), y s y x
theorem bdd_below_iff_exists_le {γ : Type w} [semilattice_inf γ] {s : set γ} (x₀ : γ) :
bdd_below s (x : γ), x x₀ (y : γ), y s x y
theorem bdd_above.exists_ge {γ : Type w} [semilattice_sup γ] {s : set γ} (hs : bdd_above s) (x₀ : γ) :
(x : γ), x₀ x (y : γ), y s y x
theorem bdd_below.exists_le {γ : Type w} [semilattice_inf γ] {s : set γ} (hs : bdd_below s) (x₀ : γ) :
(x : γ), x x₀ (y : γ), y s x y

Specific sets #

Unbounded intervals #

theorem is_least_Ici {α : Type u} [preorder α] {a : α} :
theorem is_greatest_Iic {α : Type u} [preorder α] {a : α} :
theorem is_lub_Iic {α : Type u} [preorder α] {a : α} :
theorem is_glb_Ici {α : Type u} [preorder α] {a : α} :
theorem upper_bounds_Iic {α : Type u} [preorder α] {a : α} :
theorem lower_bounds_Ici {α : Type u} [preorder α] {a : α} :
theorem bdd_above_Iic {α : Type u} [preorder α] {a : α} :
theorem bdd_below_Ici {α : Type u} [preorder α] {a : α} :
theorem bdd_above_Iio {α : Type u} [preorder α] {a : α} :
theorem bdd_below_Ioi {α : Type u} [preorder α] {a : α} :
theorem lub_Iio_le {α : Type u} [preorder α] {b : α} (a : α) (hb : is_lub (set.Iio a) b) :
b a
theorem le_glb_Ioi {α : Type u} [preorder α] {b : α} (a : α) (hb : is_glb (set.Ioi a) b) :
a b
theorem lub_Iio_eq_self_or_Iio_eq_Iic {γ : Type w} [partial_order γ] {j : γ} (i : γ) (hj : is_lub (set.Iio i) j) :
theorem glb_Ioi_eq_self_or_Ioi_eq_Ici {γ : Type w} [partial_order γ] {j : γ} (i : γ) (hj : is_glb (set.Ioi i) j) :
theorem exists_lub_Iio {γ : Type w} [linear_order γ] (i : γ) :
(j : γ), is_lub (set.Iio i) j
theorem exists_glb_Ioi {γ : Type w} [linear_order γ] (i : γ) :
(j : γ), is_glb (set.Ioi i) j
theorem is_lub_Iio {γ : Type w} [linear_order γ] [densely_ordered γ] {a : γ} :
theorem is_glb_Ioi {γ : Type w} [linear_order γ] [densely_ordered γ] {a : γ} :
theorem upper_bounds_Iio {γ : Type w} [linear_order γ] [densely_ordered γ] {a : γ} :
theorem lower_bounds_Ioi {γ : Type w} [linear_order γ] [densely_ordered γ] {a : γ} :

Singleton #

theorem is_greatest_singleton {α : Type u} [preorder α] {a : α} :
theorem is_least_singleton {α : Type u} [preorder α] {a : α} :
is_least {a} a
theorem is_lub_singleton {α : Type u} [preorder α] {a : α} :
is_lub {a} a
theorem is_glb_singleton {α : Type u} [preorder α] {a : α} :
is_glb {a} a
theorem bdd_above_singleton {α : Type u} [preorder α] {a : α} :
theorem bdd_below_singleton {α : Type u} [preorder α] {a : α} :
@[simp]
theorem upper_bounds_singleton {α : Type u} [preorder α] {a : α} :
@[simp]
theorem lower_bounds_singleton {α : Type u} [preorder α] {a : α} :

Bounded intervals #

theorem bdd_above_Icc {α : Type u} [preorder α] {a b : α} :
theorem bdd_below_Icc {α : Type u} [preorder α] {a b : α} :
theorem bdd_above_Ico {α : Type u} [preorder α] {a b : α} :
theorem bdd_below_Ico {α : Type u} [preorder α] {a b : α} :
theorem bdd_above_Ioc {α : Type u} [preorder α] {a b : α} :
theorem bdd_below_Ioc {α : Type u} [preorder α] {a b : α} :
theorem bdd_above_Ioo {α : Type u} [preorder α] {a b : α} :
theorem bdd_below_Ioo {α : Type u} [preorder α] {a b : α} :
theorem is_greatest_Icc {α : Type u} [preorder α] {a b : α} (h : a b) :
theorem is_lub_Icc {α : Type u} [preorder α] {a b : α} (h : a b) :
is_lub (set.Icc a b) b
theorem upper_bounds_Icc {α : Type u} [preorder α] {a b : α} (h : a b) :
theorem is_least_Icc {α : Type u} [preorder α] {a b : α} (h : a b) :
theorem is_glb_Icc {α : Type u} [preorder α] {a b : α} (h : a b) :
is_glb (set.Icc a b) a
theorem lower_bounds_Icc {α : Type u} [preorder α] {a b : α} (h : a b) :
theorem is_greatest_Ioc {α : Type u} [preorder α] {a b : α} (h : a < b) :
theorem is_lub_Ioc {α : Type u} [preorder α] {a b : α} (h : a < b) :
is_lub (set.Ioc a b) b
theorem upper_bounds_Ioc {α : Type u} [preorder α] {a b : α} (h : a < b) :
theorem is_least_Ico {α : Type u} [preorder α] {a b : α} (h : a < b) :
theorem is_glb_Ico {α : Type u} [preorder α] {a b : α} (h : a < b) :
is_glb (set.Ico a b) a
theorem lower_bounds_Ico {α : Type u} [preorder α] {a b : α} (h : a < b) :
theorem is_glb_Ioo {γ : Type w} [semilattice_sup γ] [densely_ordered γ] {a b : γ} (h : a < b) :
is_glb (set.Ioo a b) a
theorem lower_bounds_Ioo {γ : Type w} [semilattice_sup γ] [densely_ordered γ] {a b : γ} (hab : a < b) :
theorem is_glb_Ioc {γ : Type w} [semilattice_sup γ] [densely_ordered γ] {a b : γ} (hab : a < b) :
is_glb (set.Ioc a b) a
theorem lower_bound_Ioc {γ : Type w} [semilattice_sup γ] [densely_ordered γ] {a b : γ} (hab : a < b) :
theorem is_lub_Ioo {γ : Type w} [semilattice_inf γ] [densely_ordered γ] {a b : γ} (hab : a < b) :
is_lub (set.Ioo a b) b
theorem upper_bounds_Ioo {γ : Type w} [semilattice_inf γ] [densely_ordered γ] {a b : γ} (hab : a < b) :
theorem is_lub_Ico {γ : Type w} [semilattice_inf γ] [densely_ordered γ] {a b : γ} (hab : a < b) :
is_lub (set.Ico a b) b
theorem upper_bounds_Ico {γ : Type w} [semilattice_inf γ] [densely_ordered γ] {a b : γ} (hab : a < b) :
theorem bdd_below_iff_subset_Ici {α : Type u} [preorder α] {s : set α} :
bdd_below s (a : α), s set.Ici a
theorem bdd_above_iff_subset_Iic {α : Type u} [preorder α] {s : set α} :
bdd_above s (a : α), s set.Iic a
theorem bdd_below_bdd_above_iff_subset_Icc {α : Type u} [preorder α] {s : set α} :
bdd_below s bdd_above s (a b : α), s set.Icc a b

Univ #

@[simp]
theorem is_greatest_univ_iff {α : Type u} [preorder α] {a : α} :
theorem is_lub_univ {α : Type u} [preorder α] [order_top α] :
@[simp]
theorem is_least_univ_iff {α : Type u} [preorder α] {a : α} :
theorem is_glb_univ {α : Type u} [preorder α] [order_bot α] :
@[simp]
@[simp]

Empty set #

@[simp]
@[simp]
@[simp]
theorem bdd_above_empty {α : Type u} [preorder α] [nonempty α] :
@[simp]
theorem bdd_below_empty {α : Type u} [preorder α] [nonempty α] :
@[simp]
theorem is_glb_empty_iff {α : Type u} [preorder α] {a : α} :
@[simp]
theorem is_lub_empty_iff {α : Type u} [preorder α] {a : α} :
theorem is_glb_empty {α : Type u} [preorder α] [order_top α] :
theorem is_lub_empty {α : Type u} [preorder α] [order_bot α] :
theorem is_lub.nonempty {α : Type u} [preorder α] {s : set α} {a : α} [no_min_order α] (hs : is_lub s a) :
theorem is_glb.nonempty {α : Type u} [preorder α] {s : set α} {a : α} [no_max_order α] (hs : is_glb s a) :
theorem nonempty_of_not_bdd_above {α : Type u} [preorder α] {s : set α} [ha : nonempty α] (h : ¬bdd_above s) :
theorem nonempty_of_not_bdd_below {α : Type u} [preorder α] {s : set α} [ha : nonempty α] (h : ¬bdd_below s) :

insert #

@[simp]
theorem bdd_above_insert {α : Type u} [preorder α] [is_directed α has_le.le] {s : set α} {a : α} :

Adding a point to a set preserves its boundedness above.

@[protected]
theorem bdd_above.insert {α : Type u} [preorder α] [is_directed α has_le.le] {s : set α} (a : α) :
@[simp]
theorem bdd_below_insert {α : Type u} [preorder α] [is_directed α ge] {s : set α} {a : α} :

Adding a point to a set preserves its boundedness below.

theorem bdd_below.insert {α : Type u} [preorder α] [is_directed α ge] {s : set α} (a : α) :
theorem is_lub.insert {γ : Type w} [semilattice_sup γ] (a : γ) {b : γ} {s : set γ} (hs : is_lub s b) :
theorem is_glb.insert {γ : Type w} [semilattice_inf γ] (a : γ) {b : γ} {s : set γ} (hs : is_glb s b) :
theorem is_greatest.insert {γ : Type w} [linear_order γ] (a : γ) {b : γ} {s : set γ} (hs : is_greatest s b) :
theorem is_least.insert {γ : Type w} [linear_order γ] (a : γ) {b : γ} {s : set γ} (hs : is_least s b) :
@[simp]
theorem upper_bounds_insert {α : Type u} [preorder α] (a : α) (s : set α) :
@[simp]
theorem lower_bounds_insert {α : Type u} [preorder α] (a : α) (s : set α) :
@[protected, simp]
theorem order_top.bdd_above {α : Type u} [preorder α] [order_top α] (s : set α) :

When there is a global maximum, every set is bounded above.

@[protected, simp]
theorem order_bot.bdd_below {α : Type u} [preorder α] [order_bot α] (s : set α) :

When there is a global minimum, every set is bounded below.

Pair #

theorem is_lub_pair {γ : Type w} [semilattice_sup γ] {a b : γ} :
is_lub {a, b} (a b)
theorem is_glb_pair {γ : Type w} [semilattice_inf γ] {a b : γ} :
is_glb {a, b} (a b)
theorem is_least_pair {γ : Type w} [linear_order γ] {a b : γ} :
theorem is_greatest_pair {γ : Type w} [linear_order γ] {a b : γ} :

Lower/upper bounds #

@[simp]
theorem is_lub_lower_bounds {α : Type u} [preorder α] {s : set α} {a : α} :
@[simp]
theorem is_glb_upper_bounds {α : Type u} [preorder α] {s : set α} {a : α} :

(In)equalities with the least upper bound and the greatest lower bound #

theorem lower_bounds_le_upper_bounds {α : Type u} [preorder α] {s : set α} {a b : α} (ha : a lower_bounds s) (hb : b upper_bounds s) :
theorem is_glb_le_is_lub {α : Type u} [preorder α] {s : set α} {a b : α} (ha : is_glb s a) (hb : is_lub s b) (hs : s.nonempty) :
a b
theorem is_lub_lt_iff {α : Type u} [preorder α] {s : set α} {a b : α} (ha : is_lub s a) :
a < b (c : α) (H : c upper_bounds s), c < b
theorem lt_is_glb_iff {α : Type u} [preorder α] {s : set α} {a b : α} (ha : is_glb s a) :
b < a (c : α) (H : c lower_bounds s), b < c
theorem le_of_is_lub_le_is_glb {α : Type u} [preorder α] {s : set α} {a b x y : α} (ha : is_glb s a) (hb : is_lub s b) (hab : b a) (hx : x s) (hy : y s) :
x y
theorem is_least.unique {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_least s a) (Hb : is_least s b) :
a = b
theorem is_least.is_least_iff_eq {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_least s a) :
is_least s b a = b
theorem is_greatest.unique {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_greatest s a) (Hb : is_greatest s b) :
a = b
theorem is_greatest.is_greatest_iff_eq {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_greatest s a) :
is_greatest s b a = b
theorem is_lub.unique {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_lub s a) (Hb : is_lub s b) :
a = b
theorem is_glb.unique {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_glb s a) (Hb : is_glb s b) :
a = b
theorem set.subsingleton_of_is_lub_le_is_glb {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_glb s a) (Hb : is_lub s b) (hab : b a) :
theorem is_glb_lt_is_lub_of_ne {α : Type u} [partial_order α] {s : set α} {a b : α} (Ha : is_glb s a) (Hb : is_lub s b) {x y : α} (Hx : x s) (Hy : y s) (Hxy : x y) :
a < b
theorem lt_is_lub_iff {α : Type u} [linear_order α] {s : set α} {a b : α} (h : is_lub s a) :
b < a (c : α) (H : c s), b < c
theorem is_glb_lt_iff {α : Type u} [linear_order α] {s : set α} {a b : α} (h : is_glb s a) :
a < b (c : α) (H : c s), c < b
theorem is_lub.exists_between {α : Type u} [linear_order α] {s : set α} {a b : α} (h : is_lub s a) (hb : b < a) :
(c : α) (H : c s), b < c c a
theorem is_lub.exists_between' {α : Type u} [linear_order α] {s : set α} {a b : α} (h : is_lub s a) (h' : a s) (hb : b < a) :
(c : α) (H : c s), b < c c < a
theorem is_glb.exists_between {α : Type u} [linear_order α] {s : set α} {a b : α} (h : is_glb s a) (hb : a < b) :
(c : α) (H : c s), a c c < b
theorem is_glb.exists_between' {α : Type u} [linear_order α] {s : set α} {a b : α} (h : is_glb s a) (h' : a s) (hb : a < b) :
(c : α) (H : c s), a < c c < b

Images of upper/lower bounds under monotone functions #

theorem monotone_on.mem_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : monotone_on f t) {a : α} (Hst : s t) (Has : a upper_bounds s) (Hat : a t) :
f a upper_bounds (f '' s)
theorem monotone_on.mem_upper_bounds_image_self {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : monotone_on f t) {a : α} :
theorem monotone_on.mem_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : monotone_on f t) {a : α} (Hst : s t) (Has : a lower_bounds s) (Hat : a t) :
f a lower_bounds (f '' s)
theorem monotone_on.mem_lower_bounds_image_self {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : monotone_on f t) {a : α} :
theorem monotone_on.image_upper_bounds_subset_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : monotone_on f t) (Hst : s t) :
theorem monotone_on.image_lower_bounds_subset_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : monotone_on f t) (Hst : s t) :
theorem monotone_on.map_bdd_above {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : monotone_on f t) (Hst : s t) :

The image under a monotone function on a set t of a subset which has an upper bound in t is bounded above.

theorem monotone_on.map_bdd_below {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : monotone_on f t) (Hst : s t) :

The image under a monotone function on a set t of a subset which has a lower bound in t is bounded below.

theorem monotone_on.map_is_least {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : monotone_on f t) {a : α} (Ha : is_least t a) :
is_least (f '' t) (f a)

A monotone map sends a least element of a set to a least element of its image.

theorem monotone_on.map_is_greatest {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : monotone_on f t) {a : α} (Ha : is_greatest t a) :
is_greatest (f '' t) (f a)

A monotone map sends a greatest element of a set to a greatest element of its image.

theorem antitone_on.mem_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : antitone_on f t) {a : α} (Hst : s t) (Has : a lower_bounds s) :
a t f a upper_bounds (f '' s)
theorem antitone_on.mem_upper_bounds_image_self {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : antitone_on f t) {a : α} :
theorem antitone_on.mem_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : antitone_on f t) {a : α} (Hst : s t) :
theorem antitone_on.mem_lower_bounds_image_self {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : antitone_on f t) {a : α} :
theorem antitone_on.image_lower_bounds_subset_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : antitone_on f t) (Hst : s t) :
theorem antitone_on.image_upper_bounds_subset_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : antitone_on f t) (Hst : s t) :
theorem antitone_on.map_bdd_above {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : antitone_on f t) (Hst : s t) :

The image under an antitone function of a set which is bounded above is bounded below.

theorem antitone_on.map_bdd_below {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {s t : set α} (Hf : antitone_on f t) (Hst : s t) :

The image under an antitone function of a set which is bounded below is bounded above.

theorem antitone_on.map_is_greatest {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : antitone_on f t) {a : α} :
is_greatest t a is_least (f '' t) (f a)

An antitone map sends a greatest element of a set to a least element of its image.

theorem antitone_on.map_is_least {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} {t : set α} (Hf : antitone_on f t) {a : α} :
is_least t a is_greatest (f '' t) (f a)

An antitone map sends a least element of a set to a greatest element of its image.

theorem monotone.mem_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {a : α} {s : set α} (Ha : a upper_bounds s) :
f a upper_bounds (f '' s)
theorem monotone.mem_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {a : α} {s : set α} (Ha : a lower_bounds s) :
f a lower_bounds (f '' s)
theorem monotone.image_upper_bounds_subset_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {s : set α} :
theorem monotone.image_lower_bounds_subset_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {s : set α} :
theorem monotone.map_bdd_above {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {s : set α} :

The image under a monotone function of a set which is bounded above is bounded above. See also bdd_above.image2.

theorem monotone.map_bdd_below {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {s : set α} :

The image under a monotone function of a set which is bounded below is bounded below. See also bdd_below.image2.

theorem monotone.map_is_least {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {a : α} {s : set α} (Ha : is_least s a) :
is_least (f '' s) (f a)

A monotone map sends a least element of a set to a least element of its image.

theorem monotone.map_is_greatest {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (Hf : monotone f) {a : α} {s : set α} (Ha : is_greatest s a) :
is_greatest (f '' s) (f a)

A monotone map sends a greatest element of a set to a greatest element of its image.

theorem antitone.mem_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {a : α} {s : set α} :
theorem antitone.mem_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {a : α} {s : set α} :
theorem antitone.image_lower_bounds_subset_upper_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {s : set α} :
theorem antitone.image_upper_bounds_subset_lower_bounds_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {s : set α} :
theorem antitone.map_bdd_above {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {s : set α} :

The image under an antitone function of a set which is bounded above is bounded below.

theorem antitone.map_bdd_below {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {s : set α} :

The image under an antitone function of a set which is bounded below is bounded above.

theorem antitone.map_is_greatest {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {a : α} {s : set α} :
is_greatest s a is_least (f '' s) (f a)

An antitone map sends a greatest element of a set to a least element of its image.

theorem antitone.map_is_least {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : antitone f) {a : α} {s : set α} :
is_least s a is_greatest (f '' s) (f a)

An antitone map sends a least element of a set to a greatest element of its image.

theorem mem_upper_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : a upper_bounds s) (hb : b upper_bounds t) :
theorem mem_lower_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : a lower_bounds s) (hb : b lower_bounds t) :
theorem image2_upper_bounds_upper_bounds_subset {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :
theorem image2_lower_bounds_lower_bounds_subset {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :
theorem bdd_above.image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :

See also monotone.map_bdd_above.

theorem bdd_below.image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :

See also monotone.map_bdd_below.

theorem is_greatest.image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : is_greatest s a) (hb : is_greatest t b) :
is_greatest (set.image2 f s t) (f a b)
theorem is_least.image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : is_least s a) (hb : is_least t b) :
is_least (set.image2 f s t) (f a b)
theorem mem_upper_bounds_image2_of_mem_upper_bounds_of_mem_lower_bounds {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : a upper_bounds s) (hb : b lower_bounds t) :
theorem mem_lower_bounds_image2_of_mem_lower_bounds_of_mem_upper_bounds {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : a lower_bounds s) (hb : b upper_bounds t) :
theorem image2_upper_bounds_lower_bounds_subset_upper_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem image2_lower_bounds_upper_bounds_subset_lower_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem bdd_above.bdd_above_image2_of_bdd_below {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem bdd_below.bdd_below_image2_of_bdd_above {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem is_greatest.is_greatest_image2_of_is_least {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : is_greatest s a) (hb : is_least t b) :
is_greatest (set.image2 f s t) (f a b)
theorem is_least.is_least_image2_of_is_greatest {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), monotone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : is_least s a) (hb : is_greatest t b) :
is_least (set.image2 f s t) (f a b)
theorem mem_upper_bounds_image2_of_mem_lower_bounds {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : a lower_bounds s) (hb : b lower_bounds t) :
theorem mem_lower_bounds_image2_of_mem_upper_bounds {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : a upper_bounds s) (hb : b upper_bounds t) :
theorem image2_upper_bounds_upper_bounds_subset_upper_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem image2_lower_bounds_lower_bounds_subset_lower_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem bdd_below.image2_bdd_above {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem bdd_above.image2_bdd_below {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) :
theorem is_least.is_greatest_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : is_least s a) (hb : is_least t b) :
is_greatest (set.image2 f s t) (f a b)
theorem is_greatest.is_least_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), antitone (f a)) (ha : is_greatest s a) (hb : is_greatest t b) :
is_least (set.image2 f s t) (f a b)
theorem mem_upper_bounds_image2_of_mem_upper_bounds_of_mem_upper_bounds {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : a lower_bounds s) (hb : b upper_bounds t) :
theorem mem_lower_bounds_image2_of_mem_lower_bounds_of_mem_lower_bounds {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : a upper_bounds s) (hb : b lower_bounds t) :
theorem image2_lower_bounds_upper_bounds_subset_upper_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :
theorem image2_upper_bounds_lower_bounds_subset_lower_bounds_image2 {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :
theorem bdd_below.bdd_above_image2_of_bdd_above {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :
theorem bdd_above.bdd_below_image2_of_bdd_above {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) :
theorem is_least.is_greatest_image2_of_is_greatest {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : is_least s a) (hb : is_greatest t b) :
is_greatest (set.image2 f s t) (f a b)
theorem is_greatest.is_least_image2_of_is_least {α : Type u} {β : Type v} {γ : Type w} [preorder α] [preorder β] [preorder γ] {f : α β γ} {s : set α} {t : set β} {a : α} {b : β} (h₀ : (b : β), antitone (function.swap f b)) (h₁ : (a : α), monotone (f a)) (ha : is_greatest s a) (hb : is_least t b) :
is_least (set.image2 f s t) (f a b)
theorem is_glb.of_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : {x y : α}, f x f y x y) {s : set α} {x : α} (hx : is_glb (f '' s) (f x)) :
is_glb s x
theorem is_lub.of_image {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (hf : {x y : α}, f x f y x y) {s : set α} {x : α} (hx : is_lub (f '' s) (f x)) :
is_lub s x
theorem is_lub_pi {α : Type u} {π : α Type u_1} [Π (a : α), preorder (π a)] {s : set (Π (a : α), π a)} {f : Π (a : α), π a} :
is_lub s f (a : α), is_lub (function.eval a '' s) (f a)
theorem is_glb_pi {α : Type u} {π : α Type u_1} [Π (a : α), preorder (π a)] {s : set (Π (a : α), π a)} {f : Π (a : α), π a} :
is_glb s f (a : α), is_glb (function.eval a '' s) (f a)
theorem is_lub_prod {α : Type u} {β : Type v} [preorder α] [preorder β] {s : set × β)} (p : α × β) :
theorem is_glb_prod {α : Type u} {β : Type v} [preorder α] [preorder β] {s : set × β)} (p : α × β) :
def scott_continuous {α : Type u} {β : Type v} [preorder α] [preorder β] (f : α β) :
Prop

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.

Equations
@[protected]
theorem scott_continuous.monotone {α : Type u} {β : Type v} [preorder α] [preorder β] {f : α β} (h : scott_continuous f) :