Library HoTT.Homotopy.CayleyDickson

Require Import Types.Paths.
Require Import Classes.interfaces.abstract_algebra.
Require Import Cubical.DPath Cubical.PathSquare.
Require Import Pointed.Core Pointed.pSusp.
Require Import Homotopy.HSpace.Core.
Require Import Homotopy.Suspension.
Require Import Homotopy.Join.Core.

Local Open Scope pointed_scope.
Local Open Scope mc_mult_scope.

The Cayley-Dickson Construction
The Cayley-Dickson construction in homotopy type theory due to Buchholtz and Rijke https://arxiv.org/abs/1610.01134 is a method to construct an H-space structure on the join of two suspensions of a type A. As a special case, this gives a way to construct an H-space structure on S^3 leading to the quarternionic Hopf fibration.
The construction works by replicating the classical Cayley-Dickson construction on convolution algebras (×-algebras), which can produce the complex numbers, quaternions, octonions, etc. starting with the real numbers. We cannot replicate this directly in HoTT since such algebras have a contractible underlying vector space, therefore the construction here attempts to axiomatize the properties of the units of those algebras instead.
This is done by postulating a structure called a "Cayley-Dickson imaginaroid" on a type A and showing that Join (Susp A) (Susp A) is an H-space. An open problem is to show that this space itself is also an imaginaroid given further, yet unspecified, coherences on A.

Cayley-Dickson spheroids

A Cayley-Dickson Spheroid is a pointed type X which is an H-space, with two operations called negation and conjugation, satisfying the following seven laws: 1. --x = x 2. x** = x 3. 1* = 1 4. (-x)* = -x× 5. x(-y) = -(xy) 6. (xy)* = y× x× 7. x× x = 1 Note that the above laws are written in pseudocode since we cannot define multiplication by juxtaposition in Coq, and * is used to denote conjugation.
Class CayleyDicksonSpheroid (X : pType) := {
  cds_hspace : IsHSpace X;
  cds_negate : Negate X;
  cds_conjug : Conjugate X;
  cds_negate_inv : Involutive cds_negate;
  cds_conjug_inv : Involutive cds_conjug;
  cds_conjug_unit_pres : IsUnitPreserving cds_conjug;
  cds_conjug_left_inv : LeftInverse (.*.) cds_conjug mon_unit;
  cds_conjug_distr : DistrOpp (.*.) cds_conjug;
  cds_swapop : SwapOp (-) cds_conjug;
  cds_factorneg_r : FactorNegRight (-) (.*.);
}.
#[export] Existing Instances
  cds_hspace
  cds_negate
  cds_conjug
  cds_negate_inv
  cds_conjug_inv
  cds_conjug_unit_pres
  cds_conjug_left_inv
  cds_conjug_distr
  cds_swapop
  cds_factorneg_r.

Section CayleyDicksonSpheroid_Properties.

  Context {X : pType} `(CayleyDicksonSpheroid X).

  Local Instance isequiv_cds_conjug : IsEquiv cds_conjug
    := isequiv_adjointify cds_conjug cds_conjug cds_conjug_inv cds_conjug_inv.

  #[export] Instance cds_factorneg_l : FactorNegLeft (-) (.*.).
  Proof.
    intros x y.
    rapply (equiv_inj conj).
    lhs rapply distropp.
    rhs rapply swapop.
    rhs rapply (ap _ (distropp _ _)).
    rhs_V rapply factorneg_r.
    napply ap.
    apply swapop.
  Defined.

  #[export] Instance cds_conjug_right_inv : RightInverse (.*.) cds_conjug mon_unit.
  Proof.
    intro x.
    lhs_V exact (ap (.* conj x) (involutive x)).
    rapply left_inverse.
  Defined.

End CayleyDicksonSpheroid_Properties.

Negation and conjugation on suspensions


Instance conjugate_susp (A : Type) `(Negate A) : Conjugate (Susp A)
  := functor_susp (-).

Instance negate_susp (A : Type) `(Negate A) : Negate (Susp A)
  := susp_neg _ o conjugate_susp A (-).

conjugate_susp A and negate_susp A commute.
Instance swapop_conjugate_susp {A} `(Negate A)
  : SwapOp (negate_susp A (-)) (conjugate_susp A (-)).
Proof.
  intros x.
  symmetry.
  napply susp_neg_natural.
Defined.

conjugate_susp A is involutive, since any functor applied to an involution gives an involution.
Instance involutive_conjugate_susp {A} `(Negate A, !Involutive (-))
  : Involutive (conjugate_susp A (-)).
Proof.
  intros x.
  lhs_V napply functor_susp_compose.
  rhs_V napply functor_susp_idmap.
  napply functor2_susp.
  exact involutive.
Defined.

conjugate_susp A is involutive as any composite of commuting involutions is an involution.
Instance involutive_negate_susp {A} `(Negate A, !Involutive (-))
  : Involutive (negate_susp A (-)).
Proof.
  intros x.
  unfold negate_susp.
  lhs napply ap.
  1: napply swapop_conjugate_susp.
  lhs rapply susp_neg_inv.
  rapply involutive.
Defined.

Cayley-Dickson imaginaroids

Every suspension of a Cayley-Dickson imaginaroid gives a Cayley-Dickson spheroid.
A Cayley-Dickson imaginaroid A whose multiplication on the suspension is associative gives rise to an H-space structure on the join of the suspension of A with itself.
Let A be a Cayley-Dickson imaginaroid with associative H-space multiplication on Susp A.
Declaring these as local instances so that they can be found
  Local Instance hspace_op' : SgOp (Susp A) := hspace_op.
  Local Instance hspace_unit' : MonUnit (Susp A) := hspace_mon_unit.

First we make some observations with the context we have.
  Section Lemmata.

    Context (a b c d : Susp A).

    Local Definition f := (fun xa × (c × -x)).
    Local Definition g := (fun yc × (y × b)).

    Lemma lemma1 : f (- mon_unit) = a × c.
    Proof.
      unfold f; apply ap.
      exact (hspace_right_identity c).
    Defined.

    Lemma lemma2 : f (conj c × conj a × d × conj b) = (-d) × conj b.
    Proof.
      unfold f.
      rewrite 2 factorneg_r.
      rewrite 3 simple_associativity.
      rewrite <- distropp.
      rewrite (right_inverse (a × c)).
      rewrite (left_identity d).
      symmetry.
      apply factorneg_l.
    Defined.

    Lemma lemma3 : g mon_unit = c × b.
    Proof.
      unfold g; apply ap.
      apply left_identity.
    Defined.

    Lemma lemma4 : g (conj c × conj a × d × conj b) = conj a × d.
    Proof.
      unfold g.
      rewrite 2 simple_associativity.
      rewrite <- simple_associativity.
      rewrite left_inverse.
      rewrite right_identity.
      rewrite 2 simple_associativity.
      rewrite right_inverse.
      rewrite <- simple_associativity.
      apply left_identity.
    Defined.

  End Lemmata.

  Arguments f {_ _}.
  Arguments g {_ _}.

Here is the multiplication map in algebraic form: (a,b) × (c,d) = (a × c - d × b*, a× × d + c × b). The following is the spherical form.
  #[export] Instance cd_op : SgOp (pjoin (psusp A) (psusp A)).
  Proof.
    snapply Join_rec2.
    - exact (fun a bjoinl (a × b)).
    - exact (fun a bjoinr (conj a × b)).
    - exact (fun a bjoinr (b × a)).
    - exact (fun a bjoinl ((- b) × conj a)).
    - intros; apply jglue.
    - intros; symmetry; apply jglue.
    - intros; apply jglue.
    - intros; symmetry; apply jglue.
    - intros a b c d; cbn beta.
      symmetry.
      apply sq_path.
      rewrite <- (lemma1 a c).
      rewrite <- (lemma2 a b c d).
      rewrite <- (lemma3 b c).
      rewrite <- (lemma4 a b c d).
      refine (sq_GGGG _ _ _ _ _).
      2,4: apply ap.
      1,2,3,4: srapply (Join_rec_beta_jglue _ _ (fun a bjglue (f a) (g b))).
      refine (sq_cGcG _ _ _).
      1,2: exact (ap_V _ (jglue _ _ )).
      refine (@sq_ap _ _ _ _ _ _ _ (jglue _ _) (jglue _ _)^
        (jglue _ _) (jglue _ _)^ _).
      change (PathSquare
        (jglue (- mon_unit) mon_unit)
        (jglue (conj c × conj a × d × conj b) (conj c × conj a × d × conj b))^
        (jglue (- mon_unit) (conj c × conj a × d × conj b))
        (jglue (conj c × conj a × d × conj b) mon_unit)^).
      generalize (conj c × conj a × d × conj b).
      clear a b c d.
      change ( s : Susp A,
        Diamond (-mon_unit) s (mon_unit) s).
      srapply Susp_ind; hnf.
      1: by apply diamond_v_sq.
      1: by apply diamond_h_sq.
      intro a.
      apply diamond_twist.
  Defined.

  #[export] Instance cd_op_left_identity
    : LeftIdentity cd_op pt.
  Proof.
    snapply Join_ind_Flr.
    1,2: exact (fun _ap _ (hspace_left_identity _)).
    intros a b.
    lhs napply whiskerR.
    1: exact (Join_rec_beta_jglue _ _ _ a b).
    symmetry.
    apply join_natsq.
  Defined.

  #[export] Instance cd_op_right_identity
    : RightIdentity cd_op pt.
  Proof.
    snapply Join_ind_Flr.
    1: exact (fun _ap joinl (hspace_right_identity _)).
    1: exact (fun _ap joinr (hspace_left_identity _)).
    intros a b.
    lhs napply whiskerR.
    1: exact (Join_rec_beta_jglue _ _ _ a b).
    simpl; symmetry.
    apply join_natsq.
  Defined.

  #[export] Instance hspace_cdi_susp_assoc
    : IsHSpace (pjoin (psusp A) (psusp A))
    := {}.

End ImaginaroidHSpace.