Skip to content

Commit

Permalink
moving Fst functor to Base.More
Browse files Browse the repository at this point in the history
  • Loading branch information
GenericMonkey committed Jul 19, 2023
1 parent 6f973e4 commit dbacb50
Show file tree
Hide file tree
Showing 2 changed files with 28 additions and 13 deletions.
25 changes: 25 additions & 0 deletions Cubical/Categories/Displayed/Base/More.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,25 @@
{-# OPTIONS --safe #-}
--
module Cubical.Categories.Displayed.Base.More where


open import Cubical.Foundations.Prelude

open import Cubical.Categories.Category.Base
open import Cubical.Categories.Functor

open import Cubical.Categories.Displayed.Base

private
variable
ℓC ℓC' ℓCᴰ ℓCᴰ' : Level

module _ {C : Category ℓC ℓC'} {Cᴰ : Categoryᴰ C ℓCᴰ ℓCᴰ'} where
open Functor

Fst : Functor (∫C Cᴰ) C
Fst .F-ob = fst
Fst .F-hom = fst
Fst .F-id = refl
Fst .F-seq =
λ f g cong {x = f ⋆⟨ ∫C Cᴰ ⟩ g} fst refl
16 changes: 3 additions & 13 deletions Cubical/Categories/Displayed/Preorder.agda
Original file line number Diff line number Diff line change
Expand Up @@ -10,6 +10,7 @@ open import Cubical.Categories.Category.Base
open import Cubical.Categories.Functor

open import Cubical.Categories.Displayed.Base
open import Cubical.Categories.Displayed.Base.More

private
variable
Expand Down Expand Up @@ -44,19 +45,8 @@ module _ {C : Category ℓC ℓC'} (Pᴰ : Preorderᴰ C ℓCᴰ ℓCᴰ') where
; isSetHomᴰ = isProp→isSet (Pᴰ .isPropHomᴰ)
}

module _ {C : Category ℓC ℓC'} where
open Functor

Fst : {Cᴰ : Categoryᴰ C ℓCᴰ ℓCᴰ'} Functor (∫C Cᴰ) C
Fst .F-ob = fst
Fst .F-hom = fst
Fst .F-id = refl
Fst {Cᴰ = Cᴰ} .F-seq =
λ f g cong {x = f ⋆⟨ ∫C Cᴰ ⟩ g} fst refl

open Preorderᴰ

Preorderᴰ→FstFaithful : (Pᴰ : Preorderᴰ C ℓCᴰ ℓCᴰ')
isFaithful (Fst {Cᴰ = Preorderᴰ→Catᴰ Pᴰ})
Preorderᴰ→FstFaithful Pᴰ x y f g p =
Preorderᴰ→FstFaithful : isFaithful (Fst {Cᴰ = Preorderᴰ→Catᴰ})
Preorderᴰ→FstFaithful x y f g p =
ΣPathP (p , isProp→PathP (λ i Pᴰ .isPropHomᴰ {f = p i}) (f .snd) (g .snd))

0 comments on commit dbacb50

Please sign in to comment.