summaryrefslogtreecommitdiff
path: root/src/Data/BoundedVec.agda
diff options
context:
space:
mode:
Diffstat (limited to 'src/Data/BoundedVec.agda')
-rw-r--r--src/Data/BoundedVec.agda4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Data/BoundedVec.agda b/src/Data/BoundedVec.agda
index 6359af2..cd88d6d 100644
--- a/src/Data/BoundedVec.agda
+++ b/src/Data/BoundedVec.agda
@@ -13,8 +13,8 @@ open import Data.List.Base as List using (List)
open import Data.Vec as Vec using (Vec)
import Data.BoundedVec.Inefficient as Ineff
open import Relation.Binary.PropositionalEquality
-open import Data.Nat.Properties
-open SemiringSolver
+open import Data.Nat.Solver
+open +-*-Solver
------------------------------------------------------------------------
-- The type