Morphisms of finite species
Content created by Fredrik Bakke, Egbert Rijke and Victor Blanchi.
Created on 2023-03-21.
Last modified on 2025-02-11.
module species.morphisms-finite-species where
Imports
open import foundation.dependent-pair-types open import foundation.equality-dependent-function-types open import foundation.equivalences open import foundation.function-types open import foundation.fundamental-theorem-of-identity-types open import foundation.homotopies open import foundation.homotopy-induction open import foundation.identity-types open import foundation.propositions open import foundation.sets open import foundation.torsorial-type-families open import foundation.universe-levels open import species.species-of-finite-types open import univalent-combinatorics.finite-types
Idea
A homomorphism between two finite species is a pointwise family of maps.
Definitions
The type of morphisms between finite species
hom-finite-species : {l1 l2 l3 : Level} → finite-species l1 l2 → finite-species l1 l3 → UU (lsuc l1 ⊔ l2 ⊔ l3) hom-finite-species {l1} F G = (X : Finite-Type l1) → type-Finite-Type (F X) → type-Finite-Type (G X)
The identity morphisms of finite species
id-hom-finite-species : {l1 l2 : Level} (F : finite-species l1 l2) → hom-finite-species F F id-hom-finite-species F = λ X x → x
Composition of morphisms of finite species
comp-hom-finite-species : {l1 l2 l3 l4 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (H : finite-species l1 l4) → hom-finite-species G H → hom-finite-species F G → hom-finite-species F H comp-hom-finite-species F G H f g X = (f X) ∘ (g X)
Homotopies of morphisms of finite species
htpy-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) → (hom-finite-species F G) → (hom-finite-species F G) → UU (lsuc l1 ⊔ l2 ⊔ l3) htpy-hom-finite-species {l1} F G f g = (X : Finite-Type l1) → (f X) ~ (g X) refl-htpy-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) → (f : hom-finite-species F G) → htpy-hom-finite-species F G f f refl-htpy-hom-finite-species F G f X = refl-htpy
Properties
Associativity of composition of homomorphisms of finite species
module _ {l1 l2 l3 l4 l5 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (H : finite-species l1 l4) (K : finite-species l1 l5) where associative-comp-hom-finite-species : (h : hom-finite-species H K) (g : hom-finite-species G H) (f : hom-finite-species F G) → comp-hom-finite-species F G K (comp-hom-finite-species G H K h g) f = comp-hom-finite-species F H K h (comp-hom-finite-species F G H g f) associative-comp-hom-finite-species h g f = refl
The unit laws for composition of homomorphisms of finite species
left-unit-law-comp-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (f : hom-finite-species F G) → Id (comp-hom-finite-species F G G (id-hom-finite-species G) f) f left-unit-law-comp-hom-finite-species F G f = refl right-unit-law-comp-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (f : hom-finite-species F G) → Id (comp-hom-finite-species F F G f (id-hom-finite-species F)) f right-unit-law-comp-hom-finite-species F G f = refl
Characterization of the identity type of homomorphisms of finite species
htpy-eq-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (f g : hom-finite-species F G) → Id f g → htpy-hom-finite-species F G f g htpy-eq-hom-finite-species F G f g refl X y = refl is-torsorial-htpy-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (f : hom-finite-species F G) → is-torsorial (htpy-hom-finite-species F G f) is-torsorial-htpy-hom-finite-species F G f = is-torsorial-Eq-Π (λ X → is-torsorial-htpy (f X)) is-equiv-htpy-eq-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (f g : hom-finite-species F G) → is-equiv (htpy-eq-hom-finite-species F G f g) is-equiv-htpy-eq-hom-finite-species F G f = fundamental-theorem-id ( is-torsorial-htpy-hom-finite-species F G f) ( λ g → htpy-eq-hom-finite-species F G f g) extensionality-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) (f g : hom-finite-species F G) → Id f g ≃ htpy-hom-finite-species F G f g pr1 (extensionality-hom-finite-species F G f g) = htpy-eq-hom-finite-species F G f g pr2 (extensionality-hom-finite-species F G f g) = is-equiv-htpy-eq-hom-finite-species F G f g
The type of homomorphisms of finite species is a set
is-set-hom-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) → is-set (hom-finite-species F G) is-set-hom-finite-species F G f g = is-prop-equiv ( extensionality-hom-finite-species F G f g) ( is-prop-Π ( λ X → is-prop-Π ( λ x → is-set-is-finite ( is-finite-type-Finite-Type (G X)) ( f X x) ( g X x)))) hom-set-finite-species : {l1 l2 l3 : Level} (F : finite-species l1 l2) (G : finite-species l1 l3) → Set (lsuc l1 ⊔ l2 ⊔ l3) pr1 (hom-set-finite-species F G) = hom-finite-species F G pr2 (hom-set-finite-species F G) = is-set-hom-finite-species F G
Recent changes
- 2025-02-11. Fredrik Bakke. Switch from
𝔽
toFinite-*
(#1312). - 2024-03-11. Fredrik Bakke. Refactor category theory to use strictly involutive identity types (#1052).
- 2024-01-11. Fredrik Bakke. Make type family implicit for
is-torsorial-Eq-structure
andis-torsorial-Eq-Π
(#995). - 2023-11-27. Fredrik Bakke. Refactor categories to carry a bidirectional witness of associativity (#945).
- 2023-11-24. Egbert Rijke. Refactor precomposition (#937).