Convergence in terms of filters #
The general notion of limit of a map with respect to filters on the source and target types
is Filter.Tendsto
. It is defined in terms of the order and the push-forward operation.
For instance, anticipating on Topology.Basic, the statement: "if a sequence u
converges to
some x
and u n
belongs to a set M
for n
large enough then x
is in the closure of
M
" is formalized as: Tendsto u atTop (𝓝 x) → (∀ᶠ n in atTop, u n ∈ M) → x ∈ closure M
,
which is a special case of mem_closure_of_tendsto
from Topology/Basic
.
theorem
Filter.Tendsto.le_comap
{α : Type u_1}
{β : Type u_2}
{f : α → β}
{l₁ : Filter α}
{l₂ : Filter β}
:
Alias of the forward direction of Filter.tendsto_iff_comap
.
theorem
Set.MapsTo.tendsto
{α : Type u_1}
{β : Type u_2}
{s : Set α}
{t : Set β}
{f : α → β}
(h : MapsTo f s t)
:
Filter.Tendsto f (Filter.principal s) (Filter.principal t)
theorem
Filter.Tendsto.map_mapsTo_Iic
{α : Type u_1}
{β : Type u_2}
{F : Filter α}
{G : Filter β}
{m : α → β}
:
Tendsto m F G → Set.MapsTo (map m) (Set.Iic F) (Set.Iic G)
Alias of the reverse direction of Filter.map_mapsTo_Iic_iff_tendsto
.
theorem
Filter.map_mapsTo_Iic_iff_mapsTo
{α : Type u_1}
{β : Type u_2}
{s : Set α}
{t : Set β}
{m : α → β}
:
theorem
Set.MapsTo.filter_map_Iic
{α : Type u_1}
{β : Type u_2}
{s : Set α}
{t : Set β}
{m : α → β}
:
MapsTo m s t → MapsTo (Filter.map m) (Iic (Filter.principal s)) (Iic (Filter.principal t))
Alias of the reverse direction of Filter.map_mapsTo_Iic_iff_mapsTo
.