Asymptotic equivalence #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file, we define the relation is_equivalent l u v
, which means that u-v
is little o of
v
along the filter l
.
Unlike is_[oO]
relations, this one requires u
and v
to have the same codomain β
. While the
definition only requires β
to be a normed_add_comm_group
, most interesting properties require it
to be a normed_field
.
Notations #
We introduce the notation u ~[l] v := is_equivalent l u v
, which you can use by opening the
asymptotics
locale.
Main results #
If β
is a normed_add_comm_group
:
_ ~[l] _
is an equivalence relation- Equivalent statements for
u ~[l] const _ c
:- If
c ≠ 0
, this is true ifftendsto u l (𝓝 c)
(seeis_equivalent_const_iff_tendsto
) - For
c = 0
, this is true iffu =ᶠ[l] 0
(seeis_equivalent_zero_iff_eventually_zero
)
- If
If β
is a normed_field
:
-
Alternative characterization of the relation (see
is_equivalent_iff_exists_eq_mul
) :u ~[l] v ↔ ∃ (φ : α → β) (hφ : tendsto φ l (𝓝 1)), u =ᶠ[l] φ * v
-
Provided some non-vanishing hypothesis, this can be seen as
u ~[l] v ↔ tendsto (u/v) l (𝓝 1)
(seeis_equivalent_iff_tendsto_one
) -
For any constant
c
,u ~[l] v
impliestendsto u l (𝓝 c) ↔ tendsto v l (𝓝 c)
(seeis_equivalent.tendsto_nhds_iff
) -
*
and/
are compatible with_ ~[l] _
(seeis_equivalent.mul
andis_equivalent.div
)
If β
is a normed_linear_ordered_field
:
- If
u ~[l] v
, we havetendsto u l at_top ↔ tendsto v l at_top
(seeis_equivalent.tendsto_at_top_iff
)
Implementation Notes #
Note that is_equivalent
takes the parameters (l : filter α) (u v : α → β)
in that order.
This is to enable calc
support, as calc
requires that the last two explicit arguments are u v
.
Two functions u
and v
are said to be asymptotically equivalent along a filter l
when
u x - v x = o(v x)
as x converges along l
.
Equations
- asymptotics.is_equivalent l u v = (u - v) =o[l] v