Left and right limits #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define the (strict) left and right limits of a function.
left_lim f x
is the strict left limit off
atx
(usingf x
as a garbage value ifx
is isolated to its left).right_lim f x
is the strict right limit off
atx
(usingf x
as a garbage value ifx
is isolated to its right).
We develop a comprehensive API for monotone functions. Notably,
monotone.continuous_at_iff_left_lim_eq_right_lim
states that a monotone function is continuous at a point if and only if its left and right limits coincide.monotone.countable_not_continuous_at
asserts that a monotone function taking values in a second-countable space has at most countably many discontinuity points.
We also port the API to antitone functions.
TODO #
Prove corresponding stronger results for strict_mono and strict_anti functions.
Let f : α → β
be a function from a linear order α
to a topological_space β
, and
let a : α
. The limit strictly to the left of f
at a
, denoted with left_lim f a
, is defined
by using the order topology on α
. If a
is isolated to its left or the function has no left
limit, we use f a
instead to guarantee a good behavior in most cases.
Equations
- function.left_lim f a = let _inst_3 : topological_space α := preorder.topology α in ite (nhds_within a (set.Iio a) = ⊥ ∨ ¬∃ (y : β), filter.tendsto f (nhds_within a (set.Iio a)) (nhds y)) (f a) (lim (nhds_within a (set.Iio a)) f)
Let f : α → β
be a function from a linear order α
to a topological_space β
, and
let a : α
. The limit strictly to the right of f
at a
, denoted with right_lim f a
, is defined
by using the order topology on α
. If a
is isolated to its right or the function has no right
limit, , we use f a
instead to guarantee a good behavior in most cases.
Equations
- function.right_lim f a = function.left_lim f a
A monotone function is continuous to the left at a point if and only if its left limit coincides with the value of the function.
A monotone function is continuous to the right at a point if and only if its right limit coincides with the value of the function.
A monotone function is continuous at a point if and only if its left and right limits coincide.
In a second countable space, the set of points where a monotone function is not right-continuous
is at most countable. Superseded by countable_not_continuous_at
which gives the two-sided
version.
In a second countable space, the set of points where a monotone function is not left-continuous
is at most countable. Superseded by countable_not_continuous_at
which gives the two-sided
version.
In a second countable space, the set of points where a monotone function is not continuous is at most countable.
An antitone function is continuous to the left at a point if and only if its left limit coincides with the value of the function.
An antitone function is continuous to the right at a point if and only if its right limit coincides with the value of the function.
An antitone function is continuous at a point if and only if its left and right limits coincide.
In a second countable space, the set of points where an antitone function is not continuous is at most countable.