Skip to content

Commit

Permalink
Category of dagger categories
Browse files Browse the repository at this point in the history
  • Loading branch information
Taneb committed May 27, 2024
1 parent fe9b960 commit 9730fd3
Showing 1 changed file with 31 additions and 0 deletions.
31 changes: 31 additions & 0 deletions src/Categories/Category/Instance/DagCats.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,31 @@
{-# OPTIONS --safe --without-K #-}

module Categories.Category.Instance.DagCats where

open import Categories.Category.Core
open import Categories.Category.Dagger
open import Categories.Functor.Dagger
open import Categories.NaturalTransformation.NaturalIsomorphism

open import Function.Base using (_on_)
open import Level

DagCats : o ℓ e Category (suc (o ⊔ ℓ ⊔ e)) (o ⊔ ℓ ⊔ e) (o ⊔ ℓ ⊔ e)
DagCats o ℓ e = record
{ Obj = DaggerCategory o ℓ e
; _⇒_ = DaggerFunctor
; _≈_ = NaturalIsomorphism on DaggerFunctor.functor
; id = id
; _∘_ = _∘F†_
; assoc = λ {_ _ _ _ F G H} associator (DaggerFunctor.functor F) (DaggerFunctor.functor G) (DaggerFunctor.functor H)
; sym-assoc = λ {_ _ _ _ F G H} sym (associator (DaggerFunctor.functor F) (DaggerFunctor.functor G) (DaggerFunctor.functor H))
; identityˡ = unitorˡ
; identityʳ = unitorʳ
; identity² = unitor²
; equiv = record
{ refl = refl
; sym = sym
; trans = trans
}
; ∘-resp-≈ = _ⓘₕ_
}

0 comments on commit 9730fd3

Please sign in to comment.