Cavallo’s trick
Content created by Egbert Rijke and Fredrik Bakke.
Created on 2023-05-03.
Last modified on 2024-03-13.
module synthetic-homotopy-theory.cavallos-trick where
Imports
open import foundation.action-on-identifications-functions open import foundation.dependent-pair-types open import foundation.function-types open import foundation.homotopies open import foundation.identity-types open import foundation.sections open import foundation.universe-levels open import foundation.whiskering-identifications-concatenation open import structured-types.pointed-homotopies open import structured-types.pointed-maps open import structured-types.pointed-types
Idea
Cavallo’s trick is a way of upgrading an unpointed homotopy between pointed maps to a pointed homotopy.
Originally, this trick was formulated by Evan Cavallo for homogeneous spaces,
but it works as soon as the evaluation map (id ~ id) → Ω B
has a section.
Theorem
module _ {l1 l2 : Level} {A : Pointed-Type l1} {B : Pointed-Type l2} where htpy-cavallos-trick : (f g : A →∗ B) → section (λ (H : id ~ id) → H (point-Pointed-Type B)) → (map-pointed-map f ~ map-pointed-map g) → unpointed-htpy-pointed-map f g htpy-cavallos-trick (f , refl) (g , q) (K , α) H a = K (inv q ∙ inv (H (point-Pointed-Type A))) (f a) ∙ H a coherence-point-cavallos-trick : (f g : A →∗ B) (s : section (λ (H : id ~ id) → H (point-Pointed-Type B))) → (H : map-pointed-map f ~ map-pointed-map g) → coherence-point-unpointed-htpy-pointed-Π f g ( htpy-cavallos-trick f g s H) coherence-point-cavallos-trick (f , refl) (g , q) (K , α) H = inv ( ( right-whisker-concat ( ( right-whisker-concat (α _) (H _)) ∙ ( is-section-inv-concat' (H _) (inv q))) ( q)) ∙ ( left-inv q)) cavallos-trick : (f g : A →∗ B) → section (λ (H : id ~ id) → H (point-Pointed-Type B)) → (map-pointed-map f ~ map-pointed-map g) → f ~∗ g pr1 (cavallos-trick f g s H) = htpy-cavallos-trick f g s H pr2 (cavallos-trick f g s H) = coherence-point-cavallos-trick f g s H
References
- Cavallo’s trick was originally formalized in the cubical agda library.
- The above generalization was found by Buchholtz, Christensen, Rijke, and Taxerås Flaten, in [BCFR23].
- [BCFR23]
- Ulrik Buchholtz, J. Daniel Christensen, Jarl G. Taxerås Flaten, and Egbert Rijke. Central H-spaces and banded types. 02 2023. arXiv:2301.02636.
Recent changes
- 2024-03-13. Egbert Rijke. Refactoring pointed types (#1056).
- 2024-03-12. Fredrik Bakke. Bibliographies (#1058).
- 2023-10-22. Egbert Rijke and Fredrik Bakke. Refactor synthetic homotopy theory (#654).
- 2023-07-19. Egbert Rijke. refactoring pointed maps (#682).
- 2023-06-15. Egbert Rijke. Replace
isretr
withis-retraction
andissec
withis-section
(#659).