Skip to content

Commit

Permalink
Fix typos in comments
Browse files Browse the repository at this point in the history
  • Loading branch information
epost committed Mar 22, 2023
1 parent 452ec48 commit ef4b9fa
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/Categories/Category.agda
Original file line number Diff line number Diff line change
Expand Up @@ -10,10 +10,10 @@ private
variable
o ℓ e : Level

-- Convenience functions for working over mupliple categories at once:
-- Convenience functions for working over multiple categories at once:
-- C [ x , y ] (for x y objects of C) - Hom_C(x , y)
-- C [ f ≈ g ] (for f g arrows of C) - that f and g are equivalent arrows
-- C [ f ∘ g ] (for f g composables arrows of C) - composition in C
-- C [ f ∘ g ] (for f g composable arrows of C) - composition in C
infix 10 _[_,_] _[_≈_] _[_∘_]

_[_,_] : (C : Category o ℓ e) (X : Category.Obj C) (Y : Category.Obj C) Set
Expand Down

0 comments on commit ef4b9fa

Please sign in to comment.