9 lines
169 B
Agda
9 lines
169 B
Agda
|
{-# OPTIONS --cubical #-}
|
||
|
module Cat.Category.Monad where
|
||
|
|
||
|
open import Cubical
|
||
|
|
||
|
open import Cat.Category
|
||
|
open import Cat.Category.Functor
|
||
|
open import Cat.Categories.Fun
|