module Algebra.Group.Concrete where

Concrete groupsπŸ”—

In homotopy type theory, we can give an alternative definition of groups: they are the pointed, connected groupoids. The idea is that those groupoids contain exactly the same information as their fundamental group.

Such groups are dubbed concrete, because they represent the groups of symmetries of a given object (the base point); by opposition, β€œalgebraic” Groups are called abstract.

record ConcreteGroup β„“ : Type (lsuc β„“) where
  no-eta-equality
  constructor concrete-group
  field
    B                : Typeβˆ™ β„“
    has-is-connected : is-connectedβˆ™ B
    has-is-groupoid  : is-groupoid ⌞ B ⌟

  pt : ⌞ B ⌟
  pt = B .snd

Given a concrete group the underlying pointed type is denoted by analogy with the delooping of an abstract group; note that, here, the delooping is the chosen representation of so B is just a record field. We write for the base point.

Concrete groups are pointed connected types, so they enjoy the following elimination principle, which will be useful later:

  B-elim-contr : {P : ⌞ B ⌟ β†’ Type β„“'}
               β†’ is-contr (P pt)
               β†’ βˆ€ x β†’ P x
  B-elim-contr {P = P} c = connectedβˆ™-elim-prop {P = P} has-is-connected
    (is-contr→is-prop c) (c .centre)

The delooping of a group is a concrete group. In fact, we will prove later that all concrete groups arise as deloopings.

Concrete : βˆ€ {β„“} β†’ Group β„“ β†’ ConcreteGroup β„“
Concrete G .B = Deloopβˆ™ G
Concrete G .has-is-connected = Deloop-is-connected
Concrete G .has-is-groupoid = squash

Another important example of a concrete group is the circle: the delooping of the integers.

opaque
  SΒΉ-is-connected : is-connectedβˆ™ SΒΉβˆ™
  SΒΉ-is-connected = SΒΉ-elim (inc refl) prop!

SΒΉ-concrete : ConcreteGroup lzero
SΒΉ-concrete .B = SΒΉβˆ™
SΒΉ-concrete .has-is-connected = SΒΉ-is-connected
SΒΉ-concrete .has-is-groupoid = hlevel 3

The category of concrete groupsπŸ”—

The notion of group homomorphism between two groups and gets translated to, on the β€œconcrete” side, pointed maps

The pointedness condition ensures that these maps behave like abstract group homomorphisms; in particular, that they form a set.

ConcreteGroups-Hom-set
  : (G : ConcreteGroup β„“) (H : ConcreteGroup β„“')
  β†’ is-set (B G β†’βˆ™ B H)
ConcreteGroups-Hom-set G H (f , ptf) (g , ptg) p q =
  Ξ£-set-square (Ξ» _ β†’ hlevel 2) (funext-square (B-elim-contr G square))
  where
    open ConcreteGroup H using (H-Level-B)
    square : is-contr ((Ξ» j β†’ p j .fst (pt G)) ≑ (Ξ» j β†’ q j .fst (pt G)))
    square .centre i j = hcomp (βˆ‚ i ∨ βˆ‚ j) Ξ» where
      k (k = i0) β†’ pt H
      k (i = i0) β†’ p j .snd (~ k)
      k (i = i1) β†’ q j .snd (~ k)
      k (j = i0) β†’ ptf (~ k)
      k (j = i1) β†’ ptg (~ k)
    square .paths _ = H .has-is-groupoid _ _ _ _ _ _

These naturally assemble into a category.

ConcreteGroups : βˆ€ β„“ β†’ Precategory (lsuc β„“) β„“
ConcreteGroups β„“ .Ob = ConcreteGroup β„“
ConcreteGroups _ .Hom G H = B G β†’βˆ™ B H
ConcreteGroups _ .Hom-set = ConcreteGroups-Hom-set
The rest of the categorical structure is inherited from pointed functions, and univalence follows from the univalence of the universe of groupoids.
ConcreteGroups _ .id = idβˆ™
ConcreteGroups _ ._∘_ = _βˆ˜βˆ™_
ConcreteGroups _ .idr f = Ξ£-pathp refl (βˆ™-idl _)
ConcreteGroups _ .idl f = Ξ£-pathp refl (βˆ™-idr _)
ConcreteGroups _ .assoc (f , ptf) (g , ptg) (h , pth) = Ξ£-pathp refl $
  ⌜ ap f (ap g pth βˆ™ ptg) ⌝ βˆ™ ptf   β‰‘βŸ¨ ap! (ap-βˆ™ f _ _) βŸ©β‰‘
  (ap (f βŠ™ g) pth βˆ™ ap f ptg) βˆ™ ptf β‰‘βŸ¨ sym (βˆ™-assoc _ _ _) βŸ©β‰‘
  ap (f βŠ™ g) pth βˆ™ ap f ptg βˆ™ ptf   ∎

private
  isoβ†’equiv : βˆ€ {a b} β†’ Isomorphism (ConcreteGroups β„“) a b β†’ ⌞ a ⌟ ≃ ⌞ b ⌟
  iso→equiv im = Iso→Equiv (im .to .fst ,
    iso (im .from .fst) (happly (ap fst (im .invl))) (happly (ap fst (im .invr))))

ConcreteGroups-is-category : is-category (ConcreteGroups β„“)
ConcreteGroups-is-category .to-path im = ConcreteGroup-path $
  Σ-pathp (ua (iso→equiv im)) (path→ua-pathp _ (im .to .snd))
ConcreteGroups-is-category {β„“} .to-path-over im = β‰…-pathp (ConcreteGroups β„“) _ _ $
  Σ-pathp (funextP λ _ → path→ua-pathp _ refl)
    (Ξ» i j β†’ pathβ†’ua-pathp (isoβ†’equiv im) (Ξ» i β†’ im .to .snd (i ∧ j)) i)

Concrete vs.Β abstractπŸ”—

Our goal is now to prove that concrete groups and abstract groups are equivalent, in the sense that there is an equivalence of categories between ConcreteGroups and Groups.

Since we’re dealing with groupoids, we can use the alternative definition of the fundamental group that avoids set truncations.

module _ (G : ConcreteGroup β„“) where
  open π₁Groupoid (B G) (G .has-is-groupoid)
    renaming (π₁ to π₁B; Ο€β‚β‰‘Ο€β‚€β‚Šβ‚ to π₁Bβ‰‘Ο€β‚€β‚Šβ‚)
    public

We define a functor from concrete groups to abstract groups. The object mapping is given by taking the fundamental group. Given a pointed map we can apply it to a loop on to get a loop on then, we use the fact that is pointed to get a loop on by conjugation.

π₁F : Functor (ConcreteGroups β„“) (Groups β„“)
π₁F .Fβ‚€ = π₁B
π₁F .F₁ (f , ptf) .hom x = conj ptf (ap f x)

By some simple path yoga, this preserves multiplication, and the construction is functorial:

π₁F .F₁ (f , ptf) .preserves .pres-⋆ x y =
  conj ptf ⌜ ap f (x βˆ™ y) ⌝             β‰‘βŸ¨ ap! (ap-βˆ™ f _ _) βŸ©β‰‘
  conj ptf (ap f x βˆ™ ap f y)            β‰‘βŸ¨ conj-of-βˆ™ _ _ _ βŸ©β‰‘
  conj ptf (ap f x) βˆ™ conj ptf (ap f y) ∎

π₁F .F-id = ext conj-refl
π₁F .F-∘ (f , ptf) (g , ptg) = ext Ξ» x β†’
  conj (ap f ptg βˆ™ ptf) (ap (f βŠ™ g) x)        β‰‘Λ˜βŸ¨ conj-βˆ™ _ _ _ βŸ©β‰‘Λ˜
  conj ptf ⌜ conj (ap f ptg) (ap (f βŠ™ g) x) ⌝ β‰‘Λ˜βŸ¨ apΒ‘ (ap-conj f _ _) βŸ©β‰‘Λ˜
  conj ptf (ap f (conj ptg (ap g x)))         ∎

We start by showing that π₁F is split essentially surjective. This is the easy part: to build a concrete group out of an abstract group, we simply take its Delooping, and use the fact that the fundamental group of the delooping recovers the original group.

π₁F-is-split-eso : is-split-eso (π₁F {β„“})
π₁F-is-split-eso G .fst = Concrete G
π₁F-is-split-eso G .snd = pathβ†’iso (π₁Bβ‰‘Ο€β‚€β‚Šβ‚ (Concrete G) βˆ™ sym (G≑π₁B G))

We now tackle the hard part: to prove that π₁F is fully faithful. In order to show that the action on morphisms is an equivalence, we need a way of β€œdelooping” a group homomorphism into a pointed map

module Deloop-Hom {G H : ConcreteGroup β„“} (f : Groups β„“ .Hom (π₁B G) (π₁B H)) where
  open ConcreteGroup H using (H-Level-B)

How can we build such a map? All we know about is that it is a pointed connected groupoid, and thus that it comes with the elimination principle B-elim-contr. This suggests that we need to define a type family such that is contractible, conclude that holds and extract a map from that. The following construction is adapted from (Bezem et al. 2023, sec. 4.10):

  record C (x : ⌞ G ⌟) : Type β„“ where
    constructor mk
    field
      y : ⌞ H ⌟
      p : pt G ≑ x β†’ pt H ≑ y
      f-p : (Ο‰ : pt G ≑ pt G) (Ξ± : pt G ≑ x) β†’ p (Ο‰ βˆ™ Ξ±) ≑ f # Ο‰ βˆ™ p Ξ±

Our family sends a point to a point with a function that sends based paths ending at to based paths ending at with the additional constraint that must β€œextend” in the sense that a loop on the left can be factored out using

For the centre of contraction, we simply pick to be sending loops on to loops on

  C-contr : is-contr (C (pt G))
  C-contr .centre .C.y = pt H
  C-contr .centre .C.p = f .hom
  C-contr .centre .C.f-p = f .preserves .pres-⋆

As it turns out, such a structure is entirely determined by the pair which means it is contractible.

  C-contr .paths (mk y p f-p) i = mk (pt≑y i) (funextP f≑p i) (░≑░ i) where
    pt≑y : pt H ≑ y
    pt≑y = p refl

    f≑p : βˆ€ Ο‰ β†’ Square refl (f # Ο‰) (p Ο‰) (p refl)
    f≑p Ο‰ = βˆ™-filler (f # Ο‰) (p refl) β–· (sym (f-p Ο‰ refl) βˆ™ ap p (βˆ™-idr Ο‰))

    ░≑░ : PathP (Ξ» i β†’ βˆ€ Ο‰ Ξ± β†’ f≑p (Ο‰ βˆ™ Ξ±) i ≑ f # Ο‰ βˆ™ f≑p Ξ± i) (f .preserves .pres-⋆) f-p
    ░≑░ = is-propβ†’pathp (Ξ» i β†’ hlevel 1) _ _

We can now apply the elimination principle and unpack our data:

  c : βˆ€ x β†’ C x
  c = B-elim-contr G C-contr

  g : B G β†’βˆ™ B H
  p : {x : ⌞ G ⌟} β†’ pt G ≑ x β†’ pt H ≑ g .fst x

  g .fst x = c x .C.y
  g .snd = sym (p refl)

  p {x} = c x .C.p

  f-p : (Ο‰ : pt G ≑ pt G) (Ξ± : pt G ≑ pt G) β†’ p (Ο‰ βˆ™ Ξ±) ≑ f # Ο‰ βˆ™ p Ξ±
  f-p = c (pt G) .C.f-p

In order to show that this is a delooping of (i.e.Β that we need one more thing: that extends on the right. We get this essentially for free, by path induction, because ends at by definition.

  p-g : (Ξ± : pt G ≑ pt G) {x' : ⌞ G ⌟} (l : pt G ≑ x')
      β†’ p (Ξ± βˆ™ l) ≑ p Ξ± βˆ™ ap (g .fst) l
  p-g Ξ± = J (Ξ» _ l β†’ p (Ξ± βˆ™ l) ≑ p Ξ± βˆ™ ap (g .fst) l)
    (ap p (βˆ™-idr _) βˆ™ sym (βˆ™-idr _))

Since is pointed by this lets us conclude that we have found a right inverse to

  f≑apg : (Ο‰ : pt G ≑ pt G) β†’ Square (p refl) (f # Ο‰) (ap (g .fst) Ο‰) (p refl)
  f≑apg Ο‰ = commutesβ†’square $
    p refl βˆ™ ap (g .fst) Ο‰ β‰‘Λ˜βŸ¨ p-g refl Ο‰ βŸ©β‰‘Λ˜
    p (refl βˆ™ Ο‰)           β‰‘Λ˜βŸ¨ ap p βˆ™-id-comm βŸ©β‰‘Λ˜
    p (Ο‰ βˆ™ refl)           β‰‘βŸ¨ f-p Ο‰ refl βŸ©β‰‘
    f # Ο‰ βˆ™ p refl         ∎

  rinv : π₁F .F₁ {G} {H} g ≑ f
  rinv = ext Ξ» Ο‰ β†’ pathpβ†’conj (symP (f≑apg Ο‰))

We are most of the way there. In order to get a proper equivalence, we must check that delooping gives us back the same pointed map

We use the same trick, building upon what we’ve done before: start by defining a family that asserts that agrees with all the way, not just on loops:

module Deloop-Hom-π₁F {G H : ConcreteGroup β„“} (f : B G β†’βˆ™ B H) where
  open Deloop-Hom {G = G} {H} (π₁F .F₁ {G} {H} f) public
  open ConcreteGroup H using (H-Level-B)

  C' : βˆ€ x β†’ Type _
  C' x = Ξ£ (f .fst x ≑ g .fst x) Ξ» eq
       β†’ (Ξ± : pt G ≑ x) β†’ Square (f .snd) (ap (f .fst) Ξ±) (p Ξ±) eq

This is a property, and has it:

  C'-contr : is-contr (C' (pt G))
  C'-contr .centre .fst = f .snd βˆ™ sym (g .snd)
  C'-contr .centre .snd α = commutes→square $
    f .snd βˆ™ p ⌜ Ξ± ⌝                                β‰‘Λ˜βŸ¨ apΒ‘ (βˆ™-idr _) βŸ©β‰‘Λ˜
    f .snd βˆ™ ⌜ p (Ξ± βˆ™ refl) ⌝                       β‰‘βŸ¨ ap! (f-p Ξ± refl) βŸ©β‰‘
    f .snd βˆ™ conj (f .snd) (ap (f .fst) Ξ±) βˆ™ p refl β‰‘Λ˜βŸ¨ βˆ™-extendl (βˆ™-swapl (sym (conj-defn _ _))) βŸ©β‰‘Λ˜
    ap (f .fst) Ξ± βˆ™ f .snd βˆ™ p refl                 ∎
  C'-contr .paths (eq , eq-paths) = Ξ£-prop-path! $
    sym (βˆ™-unique _ (transpose (eq-paths refl)))

Using the elimination principle again, we get enough information about g to conclude that it is equal to f, so that we have a left inverse.

  c' : βˆ€ x β†’ C' x
  c' = B-elim-contr G C'-contr

  g≑f : βˆ€ x β†’ g .fst x ≑ f .fst x
  g≑f x = sym (c' x .fst)

The homotopy g≑f is pointed by definition, but we need to bend the path into a Square:

  Ξ² : g≑f (pt G) ≑ sym (f .snd βˆ™ sym (g .snd))
  Ξ² = ap (sym βŠ™ fst) (sym (C'-contr .paths (c' (pt G))))

  ptg≑ptf : Square (g≑f (pt G)) (g .snd) (f .snd) refl
  ptg≑ptf i j = hcomp (βˆ‚ i ∨ βˆ‚ j) Ξ» where
    k (k = i0) β†’ βˆ™-filler (f .snd) (sym (g .snd)) (~ j) (~ i)
    k (i = i0) β†’ g .snd j
    k (i = i1) β†’ f .snd (j ∧ k)
    k (j = i0) β†’ Ξ² (~ k) i
    k (j = i1) β†’ f .snd (~ i ∨ k)

  linv : g ≑ f
  linv = funextβˆ™ g≑f ptg≑ptf

Phew. At last, π₁F is fully faithful.

π₁F-is-ff : is-fully-faithful (π₁F {β„“})
π₁F-is-ff {β„“} {G} {H} = is-isoβ†’is-equiv $ iso
  (Deloop-Hom.g {G = G} {H})
  (Deloop-Hom.rinv {G = G} {H})
  (Deloop-Hom-π₁F.linv {G = G} {H})

We’ve shown that π₁F is fully faithful and essentially surjective; this lets us conclude with the desired equivalence.

π₁F-is-equivalence : is-equivalence (π₁F {β„“})
π₁F-is-equivalence = ff+split-esoβ†’is-equivalence
  (Ξ» {G} {H} β†’ π₁F-is-ff {_} {G} {H})
  π₁F-is-split-eso

π₁B-is-equiv : is-equiv (π₁B {β„“})
π₁B-is-equiv = is-cat-equivalenceβ†’equiv-on-objects
  ConcreteGroups-is-category
  Groups-is-category
  π₁F-is-equivalence

module Concrete≃Abstract {β„“} = Equiv (_ , π₁B-is-equiv {β„“})

References