Documentation

Counterexamples.TopologistsSineCurve

The "topologist's sine curve" is connected but not path-connected #

We give an example of a closed subset T of ℝ × ℝ which is connected but not path-connected: the closure of the set { (x, sin x⁻¹) | x ∈ Ioi 0 }.

Main results #

This formalization is part of the UniDistance Switzerland bachelor thesis of Daniele Bolla. A similar result has also been independently formalized by Vlad Tsyrklevich (https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/golf.20request.3A.20Topologist's.20sine.20curve).

The topologist's sine curve, i.e. the graph of y = sin (x⁻¹) for 0 < x.

Equations
Instances For

    The vertical line segment { (0, y) | -1 ≤ y ≤ 1 }, which is the set of limit points of S not contained in S itself.

    Equations
    Instances For

      The union of S and Z (which we will show is the closure of S).

      Equations
      Instances For
        noncomputable def TopologistsSineCurve.xSeq (y : ) (k : ) :

        A sequence of x-values tending to 0 at which the sine curve has a given y-coordinate.

        Equations
        Instances For
          theorem TopologistsSineCurve.xSeq_pos (y : ) (k : ) :
          0 < xSeq y k
          theorem TopologistsSineCurve.sin_inv_xSeq {y : } (hy : y Set.Icc (-1) 1) (k : ) :

          T is closed #

          The closure of the topologist's sine curve S is the set T.

          T is connected #

          T is connected, being the closure of the set S (which is obviously connected since it is a continuous image of the positive real line).

          T is not path-connected #

          noncomputable def TopologistsSineCurve.w :

          A point in the body of the topologist's sine curve.

          Equations
          Instances For
            theorem TopologistsSineCurve.exists_mem_Ioc_of_y {y : } (hy : y Set.Icc (-1) 1) {a : } (ha : 0 < a) :
            xSet.Ioc 0 a, Real.sin x⁻¹ = y

            For any 0 < a and any y ∈ Icc (-1) 1, we can find x ∈ Ioc a 0 with sin x⁻¹ = y.