Documentation

Mathlib.AlgebraicTopology.FundamentalGroupoid.SimplyConnected

Simply connected spaces #

This file defines simply connected spaces. A topological space is simply connected if its fundamental groupoid is equivalent to Unit.

We also define the corresponding predicate for sets.

Main theorems #

A simply connected space is one whose fundamental groupoid is equivalent to Discrete Unit

Instances
    @[deprecated simplyConnectedSpace_iff (since := "2026-01-08")]

    Alias of simplyConnectedSpace_iff.

    theorem SimplyConnectedSpace.paths_homotopic {X : Type u_3} [TopologicalSpace X] [SimplyConnectedSpace X] {x y : X} (p₁ p₂ : Path x y) :
    p₁.Homotopic p₂

    In a simply connected space, any two paths are homotopic

    A space is simply connected iff it is path connected, and there is at most one path up to homotopy between any two points.

    A space is simply connected if and only if it is path-connected and every loop at any basepoint is null-homotopic (i.e., homotopic to the constant loop).

    Simply connected sets #

    def IsSimplyConnected {X : Type u_1} [TopologicalSpace X] (s : Set X) :

    We say that a set is simply connected if it's a simply connected topological space in the induced topology.

    Equations
    Instances For
      theorem isSimplyConnected_iff_exists_homotopy_refl_forall_mem {X : Type u_1} [TopologicalSpace X] {s : Set X} :
      IsSimplyConnected s IsPathConnected s ∀ (x : X) (p : Path x x), (∀ (t : unitInterval), p t s)∃ (F : p.Homotopy (Path.refl x)), ∀ (t : unitInterval × unitInterval), F t s

      A set is simply connected iff it's path connected and any loop is homotopic to the constant path within s.

      @[simp]
      @[simp]
      theorem isSimplyConnected_smul_set₀_iff {X : Type u_1} [TopologicalSpace X] {G : Type u_3} [GroupWithZero G] [MulAction G X] [ContinuousConstSMul G X] {c : G} {s : Set X} (hc : c 0) :