summaryrefslogtreecommitdiff
path: root/CheckInsert.agda
diff options
context:
space:
mode:
authorHelmut Grohne <helmut@subdivi.de>2019-09-29 13:54:46 +0200
committerHelmut Grohne <helmut@subdivi.de>2019-09-29 13:54:46 +0200
commit6ce567bf63a61bce4ccf71e3ec402d94d1da2fb1 (patch)
treeb8fcf765afd7da6f300221f02da215696e2be4a2 /CheckInsert.agda
parent8435606d98e418394edbe5104b3f425e56a5a207 (diff)
downloadbidiragda-6ce567bf63a61bce4ccf71e3ec402d94d1da2fb1.tar.gz
port to agda/2.6.0.1 and agda-stdlib/1.1
* Data.Vec.lookup changed parameter order. * A number of symbols were moved from Data.Maybe to submodules. * In a number of occasions, agda no longer figures implicit arguments and they had to be made explicit. * We can no longer use heterogeneous proofs inside equational reasoning for propositional equality. Use heterogeneous equational reasoning. * Stop importing proof-irrelevance as that would require K.
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 ; ¬_)