at_top
and at_bot
filters on preorded sets, monoids and groups. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define the filters
at_top
: corresponds ton → +∞
;at_bot
: corresponds ton → -∞
.
Then we prove many lemmas like “if f → +∞
, then f ± c → +∞
”.
at_top
is the filter representing the limit → ∞
on an ordered set.
It is generated by the collection of up-sets {b | a ≤ b}
.
(The preorder need not have a top element for this to be well defined,
and indeed is trivial when a top element exists.)
Equations
- filter.at_top = ⨅ (a : α), filter.principal (set.Ici a)
at_bot
is the filter representing the limit → -∞
on an ordered set.
It is generated by the collection of down-sets {b | b ≤ a}
.
(The preorder need not have a bottom element for this to be well defined,
and indeed is trivial when a bottom element exists.)
Equations
- filter.at_bot = ⨅ (a : α), filter.principal (set.Iic a)
Sequences #
If u
is a sequence which is unbounded above,
then after any point, it reaches a value strictly greater than all previous values.
If u
is a sequence which is unbounded below,
then after any point, it reaches a value strictly smaller than all previous values.
If u
is a sequence which is unbounded above,
then it frequently
reaches a value strictly greater than all previous values.
If u
is a sequence which is unbounded below,
then it frequently
reaches a value strictly smaller than all previous values.
The monomial function x^n
tends to +∞
at +∞
for any positive natural n
.
A version for positive real powers exists as tendsto_rpow_at_top
.
$\lim_{x\to+\infty}|x|=+\infty$
$\lim_{x\to-\infty}|x|=+\infty$
Multiplication by constant: iff lemmas #
If r
is a positive constant, then λ x, r * f x
tends to infinity along a filter if and only
if f
tends to infinity along the same filter.
If r
is a positive constant, then λ x, f x * r
tends to infinity along a filter if and only
if f
tends to infinity along the same filter.
If f
tends to infinity along a nontrivial filter l
, then λ x, r * f x
tends to infinity
if and only if 0 < r.
If f
tends to infinity along a nontrivial filter l
, then λ x, f x * r
tends to infinity
if and only if 0 < r.
If a function tends to infinity along a filter, then this function multiplied by a positive
constant (on the left) also tends to infinity. For a version working in ℕ
or ℤ
, use
filter.tendsto.const_mul_at_top'
instead.
If a function tends to infinity along a filter, then this function multiplied by a positive
constant (on the right) also tends to infinity. For a version working in ℕ
or ℤ
, use
filter.tendsto.at_top_mul_const'
instead.
If a function tends to infinity along a filter, then this function divided by a positive constant also tends to infinity.
If r
is a positive constant, then λ x, r * f x
tends to negative infinity along a filter if
and only if f
tends to negative infinity along the same filter.
If r
is a positive constant, then λ x, f x * r
tends to negative infinity along a filter if
and only if f
tends to negative infinity along the same filter.
If r
is a negative constant, then λ x, r * f x
tends to infinity along a filter if and only
if f
tends to negative infinity along the same filter.
If r
is a negative constant, then λ x, f x * r
tends to infinity along a filter if and only
if f
tends to negative infinity along the same filter.
If r
is a negative constant, then λ x, r * f x
tends to negative infinity along a filter if
and only if f
tends to infinity along the same filter.
If r
is a negative constant, then λ x, f x * r
tends to negative infinity along a filter if
and only if f
tends to infinity along the same filter.
The function λ x, r * f x
tends to infinity along a nontrivial filter if and only if r > 0
and f
tends to infinity or r < 0
and f
tends to negative infinity.
The function λ x, f x * r
tends to infinity along a nontrivial filter if and only if r > 0
and f
tends to infinity or r < 0
and f
tends to negative infinity.
The function λ x, r * f x
tends to negative infinity along a nontrivial filter if and only if
r > 0
and f
tends to negative infinity or r < 0
and f
tends to infinity.
The function λ x, f x * r
tends to negative infinity along a nontrivial filter if and only if
r > 0
and f
tends to negative infinity or r < 0
and f
tends to infinity.
If f
tends to negative infinity along a nontrivial filter l
, then λ x, r * f x
tends to
infinity if and only if r < 0.
If f
tends to negative infinity along a nontrivial filter l
, then λ x, f x * r
tends to
infinity if and only if r < 0.
If f
tends to negative infinity along a nontrivial filter l
, then λ x, r * f x
tends to
negative infinity if and only if 0 < r.
If f
tends to negative infinity along a nontrivial filter l
, then λ x, f x * r
tends to
negative infinity if and only if 0 < r.
If f
tends to infinity along a nontrivial filter l
, then λ x, r * f x
tends to negative
infinity if and only if r < 0.
If f
tends to infinity along a nontrivial filter l
, then λ x, f x * r
tends to negative
infinity if and only if r < 0.
If a function tends to infinity along a filter, then this function multiplied by a negative constant (on the left) tends to negative infinity.
If a function tends to infinity along a filter, then this function multiplied by a negative constant (on the right) tends to negative infinity.
If a function tends to negative infinity along a filter, then this function multiplied by a positive constant (on the left) also tends to negative infinity.
If a function tends to negative infinity along a filter, then this function multiplied by a positive constant (on the right) also tends to negative infinity.
If a function tends to negative infinity along a filter, then this function divided by a positive constant also tends to negative infinity.
If a function tends to negative infinity along a filter, then this function multiplied by a negative constant (on the left) tends to positive infinity.
If a function tends to negative infinity along a filter, then this function multiplied by a negative constant (on the right) tends to positive infinity.
A function f
grows to +∞
independent of an order-preserving embedding e
.
A function f
goes to -∞
independent of an order-preserving embedding e
.
A function f
maps upwards closed sets (at_top sets) to upwards closed sets when it is a
Galois insertion. The Galois "insertion" and "connection" is weakened to only require it to be an
insertion and a connetion above b'
.
The image of the filter at_top
on Ici a
under the coercion equals at_top
.
The image of the filter at_top
on Ioi a
under the coercion equals at_top
.
The at_top
filter for an open interval Ioi a
comes from the at_top
filter in the ambient
order.
The at_top
filter for an open interval Ici a
comes from the at_top
filter in the ambient
order.
The at_bot
filter for an open interval Iio a
comes from the at_bot
filter in the ambient
order.
The at_bot
filter for an open interval Iio a
comes from the at_bot
filter in the ambient
order.
The at_bot
filter for an open interval Iic a
comes from the at_bot
filter in the ambient
order.
The at_bot
filter for an open interval Iic a
comes from the at_bot
filter in the ambient
order.
If u
is a monotone function with linear ordered codomain and the range of u
is not bounded
above, then tendsto u at_top at_top
.
If u
is a monotone function with linear ordered codomain and the range of u
is not bounded
below, then tendsto u at_bot at_bot
.
If a monotone function u : ι → α
tends to at_top
along some non-trivial filter l
, then
it tends to at_top
along at_top
.
If a monotone function u : ι → α
tends to at_bot
along some non-trivial filter l
, then
it tends to at_bot
along at_bot
.
Let f
and g
be two maps to the same commutative monoid. This lemma gives a sufficient
condition for comparison of the filter at_top.map (λ s, ∏ b in s, f b)
with
at_top.map (λ s, ∏ b in s, g b)
. This is useful to compare the set of limit points of
Π b in s, f b
as s → at_top
with the similar set for g
.
Let f
and g
be two maps to the same commutative additive monoid. This lemma gives
a sufficient condition for comparison of the filter at_top.map (λ s, ∑ b in s, f b)
with
at_top.map (λ s, ∑ b in s, g b)
. This is useful to compare the set of limit points of
∑ b in s, f b
as s → at_top
with the similar set for g
.
Given an antitone basis s : ℕ → set α
of a filter, extract an antitone subbasis s ∘ φ
,
φ : ℕ → ℕ
, such that m < n
implies r (φ m) (φ n)
. This lemma can be used to extract an
antitone basis with basis sets decreasing "sufficiently fast".
If f
is a nontrivial countably generated filter, then there exists a sequence that converges
to f
.
An abstract version of continuity of sequentially continuous functions on metric spaces:
if a filter k
is countably generated then tendsto f k l
iff for every sequence u
converging to k
, f ∘ u
tends to l
.
A sequence converges if every subsequence has a convergent subsequence.
Let g : γ → β
be an injective function and f : β → α
be a function from the codomain of g
to an additive commutative monoid. Suppose that f x = 0
outside of the range of g
. Then the
filters at_top.map (λ s, ∑ i in s, f (g i))
and at_top.map (λ s, ∑ i in s, f i)
coincide.
This lemma is used to prove the equality ∑' x, f (g x) = ∑' y, f y
under
the same assumptions.
Let g : γ → β
be an injective function and f : β → α
be a function from the codomain of g
to a commutative monoid. Suppose that f x = 1
outside of the range of g
. Then the filters
at_top.map (λ s, ∏ i in s, f (g i))
and at_top.map (λ s, ∏ i in s, f i)
coincide.
The additive version of this lemma is used to prove the equality ∑' x, f (g x) = ∑' y, f y
under
the same assumptions.