Fundamental group of a space #
Given a topological space X
and a basepoint x
, the fundamental group is the automorphism group
of x
i.e. the group with elements being loops based at x
(quotiented by homotopy equivalence).
The fundamental group is the automorphism group (vertex group) of the basepoint in the fundamental groupoid.
Equations
- FundamentalGroup X x = CategoryTheory.Aut { as := x }
Instances For
instance
instGroupFundamentalGroup
(X : Type u)
[TopologicalSpace X]
(x : X)
:
Group (FundamentalGroup X x)
Equations
instance
instInhabitedFundamentalGroup
(X : Type u)
[TopologicalSpace X]
(x : X)
:
Inhabited (FundamentalGroup X x)
Equations
def
FundamentalGroup.fundamentalGroupMulEquivOfPath
{X : Type u}
[TopologicalSpace X]
{x₀ x₁ : X}
(p : Path x₀ x₁)
:
Get an isomorphism between the fundamental groups at two points given a path
Equations
Instances For
def
FundamentalGroup.fundamentalGroupMulEquivOfPathConnected
{X : Type u}
[TopologicalSpace X]
(x₀ x₁ : X)
[PathConnectedSpace X]
:
The fundamental group of a path connected space is independent of the choice of basepoint.
Equations
Instances For
@[reducible, inline]
An element of the fundamental group as a quotient of homotopic paths.
Instances For
@[reducible, inline]
abbrev
FundamentalGroup.fromArrow
{X : TopCat}
{x : ↑X}
(p : { as := x } ⟶ { as := x })
:
FundamentalGroup (↑X) x
An element of the fundamental group, constructed from an arrow in the fundamental groupoid.
Equations
- FundamentalGroup.fromArrow p = { hom := p, inv := CategoryTheory.Groupoid.inv p, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
@[reducible, inline]
abbrev
FundamentalGroup.fromPath
{X : TopCat}
{x : ↑X}
(p : Path.Homotopic.Quotient x x)
:
FundamentalGroup (↑X) x
An element of the fundamental group, constructed from a quotient of homotopic paths.