at_top and at_bot filters on preorded sets, monoids and groups.
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 : α), 𝓟 {b : α | a ≤ b}
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 : α), 𝓟 {b : α | b ≤ 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.
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'.
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.
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.
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.