Mercurial > hg > Members > kono > Proof > category
view src/category-ex.agda @ 1124:f683d96fbc93 default tip
safe fix done
author | Shinji KONO <kono@ie.u-ryukyu.ac.jp> |
---|---|
date | Sun, 07 Jul 2024 22:28:50 +0900 |
parents | 45de2b31bf02 |
children |
line wrap: on
line source
{-# OPTIONS --cubical-compatible --safe #-} module category-ex where open import Level open import Category module _ {c₁ c₂ ℓ : Level} (A : Category c₁ c₂ ℓ) (a b c : Obj A) (g : Hom A a b) (f : Hom A b c) where open Category.Category h = _o_ A f g i = A [ f o g ]