Documentation

Mathlib.Topology.Category.LightProfinite.Sequence

The light profinite set classifying convergent sequences #

This files defines the light profinite set ℕ∪{∞}, defined as the one point compactification of .

The continuous map from ℕ∪{∞} to  sending n to 1/(n+1) and to 0.

Equations
  • One or more equations did not get rendered due to their size.
Instances For

    The continuous map from ℕ∪{∞} to  sending n to 1/(n+1) and to 0 is a closed embedding.

    @[reducible, inline]

    The one point compactification of the natural numbers as a light profinite set.

    Equations
    Instances For

      The one point compactification of the natural numbers as a light profinite set.

      Equations
      Instances For
        theorem LightProfinite.continuous_iff_convergent {Y : Type u_1} [TopologicalSpace Y] (f : LightProfinite.NatUnionInfty.toCompHaus.toTopY) :
        Continuous f Filter.Tendsto (fun (x : ) => f (some x)) Filter.atTop (nhds (f OnePoint.infty))