Structured type duality
Content created by Egbert Rijke, Fredrik Bakke, Jonathan Prieto-Cubides and Victor Blanchi.
Created on 2023-04-27.
Last modified on 2023-11-24.
module foundation.structured-type-duality where
Imports
open import foundation.dependent-pair-types open import foundation.equivalences open import foundation.structure open import foundation.type-arithmetic-dependent-pair-types open import foundation.type-duality open import foundation.univalence open import foundation.universe-levels open import foundation-core.fibers-of-maps open import foundation-core.function-types open import foundation-core.functoriality-dependent-function-types open import foundation-core.functoriality-dependent-pair-types open import foundation-core.type-theoretic-principle-of-choice
Theorem
Structured type duality
Slice-structure : {l1 l2 : Level} (l : Level) (P : UU (l1 ⊔ l) → UU l2) (B : UU l1) → UU (l1 ⊔ l2 ⊔ lsuc l) Slice-structure l P B = Σ (UU l) (λ A → hom-structure P A B) equiv-Fiber-structure : {l1 l2 : Level} (l : Level) (P : UU (l1 ⊔ l) → UU l2) (B : UU l1) → Slice-structure (l1 ⊔ l) P B ≃ fam-structure P B equiv-Fiber-structure {l1} {l3} l P B = ( ( inv-distributive-Π-Σ) ∘e ( equiv-Σ ( λ C → (b : B) → P (C b)) ( equiv-Fiber l B) ( λ f → equiv-Π-equiv-family (λ b → id-equiv)))) ∘e ( inv-associative-Σ ( UU (l1 ⊔ l)) ( λ A → A → B) ( λ f → structure-map P (pr2 f)))
equiv-fixed-Slice-structure : {l : Level} (P : UU l → UU l) (X : UU l) (A : UU l) → ( hom-structure P X A) ≃ ( Σ (A → Σ (UU l) (λ Z → P (Z))) ( λ Y → X ≃ (Σ A (pr1 ∘ Y)))) equiv-fixed-Slice-structure {l} P X A = ( ( equiv-Σ ( λ Y → X ≃ Σ A (pr1 ∘ Y)) ( equiv-Fiber-structure l P A) ( λ s → inv-equiv ( equiv-postcomp-equiv (equiv-total-fiber (pr1 (pr2 s))) X))) ∘e ( ( equiv-right-swap-Σ) ∘e ( ( inv-left-unit-law-Σ-is-contr ( is-torsorial-equiv X) ( X , id-equiv)))))
Recent changes
- 2023-11-24. Egbert Rijke. Refactor precomposition (#937).
- 2023-10-21. Egbert Rijke. Rename
is-contr-total
tois-torsorial
(#871). - 2023-09-11. Fredrik Bakke and Egbert Rijke. Some computations for different notions of equivalence (#711).
- 2023-09-06. Egbert Rijke. Rename fib to fiber (#722).
- 2023-06-10. Egbert Rijke. cleaning up transport and dependent identifications files (#650).