Asymptotics
We introduce these relations:
- is_O_with c f g l: "f is big O of g along l with constant c";
- is_O f g l: "f is big O of g along l";
- is_o f g l: "f is little o of g along l".
Here l is any filter on the domain of f and g, which are assumed to be the same. The codomains
of f and g do not need to be the same; all that is needed that there is a norm associated with
these types, and it is the norm that is compared asymptotically.
The relation is_O_with c is introduced to factor out common algebraic arguments in the proofs of
similar properties of is_O and is_o. Usually proofs outside of this file should use is_O
instead.
Often the ranges of f and g will be the real numbers, in which case the norm is the absolute
value. In general, we have
is_O f g l ↔ is_O (λ x, ∥f x∥) (λ x, ∥g x∥) l,
and similarly for is_o. But our setup allows us to use the notions e.g. with functions
to the integers, rationals, complex numbers, or any normed vector space without mentioning the
norm explicitly.
If f and g are functions to a normed field like the reals or complex numbers and g is always
nonzero, we have
is_o f g l ↔ tendsto (λ x, f x / (g x)) l (𝓝 0).
In fact, the right-to-left direction holds without the hypothesis on g, and in the other direction
it suffices to assume that f is zero wherever g is. (This generalization is useful in defining
the Fréchet derivative.)
Definitions
This version of the Landau notation is_O_with C f g l where f and g are two functions on
a type α and l is a filter on α, means that eventually for l, ∥f∥ is bounded by C * ∥g∥.
In other words, ∥f∥ / ∥g∥ is eventually bounded by C, modulo division by zero issues that are
avoided by this definition. Probably you want to use is_O instead of this relation.
Definition of is_O_with. We record it in a lemma as we will set is_O_with to be irreducible
at the end of this file.
The Landau notation is_O f g l where f and g are two functions on a type α and l is
a filter on α, means that eventually for l, ∥f∥ is bounded by a constant multiple of ∥g∥.
In other words, ∥f∥ / ∥g∥ is eventually bounded, modulo division by zero issues that are avoided
by this definition.
Equations
- asymptotics.is_O f g l = ∃ (c : ℝ), asymptotics.is_O_with c f g l
Definition of is_O in terms of is_O_with. We record it in a lemma as we will set
is_O to be irreducible at the end of this file.
Definition of is_O in terms of filters. We record it in a lemma as we will set
is_O to be irreducible at the end of this file.
The Landau notation is_o f g l where f and g are two functions on a type α and l is
a filter on α, means that eventually for l, ∥f∥ is bounded by an arbitrarily small constant
multiple of ∥g∥. In other words, ∥f∥ / ∥g∥ tends to 0 along l, modulo division by zero
issues that are avoided by this definition.
Equations
- asymptotics.is_o f g l = ∀ ⦃c : ℝ⦄, 0 < c → asymptotics.is_O_with c f g l
Definition of is_o in terms of is_O_with. We record it in a lemma as we will set
is_o to be irreducible at the end of this file.
Definition of is_o in terms of filters. We record it in a lemma as we will set
is_o to be irreducible at the end of this file.
Conversions
Congruence
Filter operations and transitivity
Simplification : norm
Simplification: negate
Product of functions (right)
Addition and subtraction
Lemmas about is_O (f₁ - f₂) g l / is_o (f₁ - f₂) g l treated as a binary relation
        Zero, one, and other constants
Multiplication by a constant
Multiplication
Scalar multiplication
Sum
Relation between f = o(g) and f / g → 0
        Miscellanous lemmas
Transfer is_O_with over a local_homeomorph.
Transfer is_O over a local_homeomorph.
Transfer is_o over a local_homeomorph.
Transfer is_O_with over a homeomorph.
Transfer is_O over a homeomorph.
Transfer is_o over a homeomorph.