Skip to content

Commit

Permalink
fix Categories.Monad.Strong
Browse files Browse the repository at this point in the history
  • Loading branch information
4e554c4c committed Mar 13, 2024
1 parent e0f3c4f commit 5050aa0
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/Categories/Monad/Strong.agda
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,7 @@ open import Categories.Functor renaming (id to idF)
open import Categories.Category.Monoidal
open import Categories.Category.Product
open import Categories.NaturalTransformation hiding (id)
open import Categories.Monad
open import Categories.Monad hiding (id)

private
variable
Expand Down Expand Up @@ -96,4 +96,4 @@ record RightStrongMonad {C : Category o ℓ e} (V : Monoidal C) : Set (o ⊔ ℓ
rightStrength : RightStrength V M

module M = Monad M
open RightStrength rightStrength public
open RightStrength rightStrength public

0 comments on commit 5050aa0

Please sign in to comment.