summaryrefslogtreecommitdiff
path: root/CheckInsert.agda
diff options
context:
space:
mode:
Diffstat (limited to 'CheckInsert.agda')
-rw-r--r--CheckInsert.agda3
1 files changed, 2 insertions, 1 deletions
diff --git a/CheckInsert.agda b/CheckInsert.agda
index 9447b04..dbba6e6 100644
--- a/CheckInsert.agda
+++ b/CheckInsert.agda
@@ -6,7 +6,8 @@ module CheckInsert (A : DecSetoid ℓ₀ ℓ₀) where
open import Data.Nat using (ℕ)
open import Data.Fin using (Fin)
open import Data.Fin.Properties using (_≟_)
-open import Data.Maybe using (Maybe ; nothing ; just) renaming (setoid to MaybeSetoid ; Eq to MaybeEq)
+open import Data.Maybe using (Maybe ; nothing ; just)
+open import Data.Maybe.Relation.Binary.Pointwise using () renaming (setoid to MaybeSetoid)
open import Data.Vec using (Vec) renaming (_∷_ to _∷V_)
open import Data.Vec.Properties using (lookup∘update′)
open import Relation.Nullary using (Dec ; yes ; no ; ¬_)