summaryrefslogtreecommitdiff
path: root/BFF.agda
diff options
context:
space:
mode:
authorHelmut Grohne <helmut@subdivi.de>2018-11-25 11:29:53 +0100
committerHelmut Grohne <helmut@subdivi.de>2018-11-25 11:29:53 +0100
commit25d4df9182c92ef26979566f06c7c9f17746f0fb (patch)
tree9fb198f637098799730a4f2fd1f30afcfe8182e1 /BFF.agda
parent7fcd0fde85d545abbdae2265e173650c12d9b4c2 (diff)
downloadbidiragda-25d4df9182c92ef26979566f06c7c9f17746f0fb.tar.gz
port to agda/2.5.4.1 and agda-stdlib/0.17
Diffstat (limited to 'BFF.agda')
-rw-r--r--BFF.agda5
1 files changed, 3 insertions, 2 deletions
diff --git a/BFF.agda b/BFF.agda
index e9b459a..06744f6 100644
--- a/BFF.agda
+++ b/BFF.agda
@@ -6,8 +6,9 @@ open import Level using () renaming (zero to ℓ₀)
import Category.Monad
import Category.Functor
open import Data.Maybe using (Maybe ; just ; nothing ; maybe′)
-open Category.Monad.RawMonad {Level.zero} Data.Maybe.monad using (_>>=_)
-open Category.Functor.RawFunctor {Level.zero} Data.Maybe.functor using (_<$>_)
+import Data.Maybe.Categorical
+open Category.Monad.RawMonad {Level.zero} Data.Maybe.Categorical.monad using (_>>=_)
+open Category.Functor.RawFunctor {Level.zero} Data.Maybe.Categorical.functor using (_<$>_)
open import Data.List using (List ; [] ; _∷_ ; map ; length)
open import Data.Vec using (Vec ; toList ; fromList ; allFin) renaming (lookup to lookupV ; map to mapV ; [] to []V ; _∷_ to _∷V_)
open import Function using (_∘_ ; flip)