summaryrefslogtreecommitdiff
path: root/BFF.agda
diff options
context:
space:
mode:
authorHelmut Grohne <grohne@cs.uni-bonn.de>2014-02-04 11:12:42 +0100
committerHelmut Grohne <grohne@cs.uni-bonn.de>2014-02-04 11:12:42 +0100
commitce4bbcc0c06b088a10881fcd66da5422571e7995 (patch)
treec87b21f7ed50c335dd093700050ce94b134d44fb /BFF.agda
parent20c176d383e59a0345f7425c5f14679906159a59 (diff)
downloadbidiragda-ce4bbcc0c06b088a10881fcd66da5422571e7995.tar.gz
remove unused imports
Most of the became unused by using the convenience functions introduced in the parent commit.
Diffstat (limited to 'BFF.agda')
-rw-r--r--BFF.agda4
1 files changed, 0 insertions, 4 deletions
diff --git a/BFF.agda b/BFF.agda
index f5573ba..ced6ebf 100644
--- a/BFF.agda
+++ b/BFF.agda
@@ -11,11 +11,7 @@ open Category.Functor.RawFunctor {Level.zero} Data.Maybe.functor using (_<$>_)
open import Data.List using (List ; [] ; _∷_ ; map ; length)
open import Data.Vec using (Vec ; toList ; fromList ; tabulate ; allFin) renaming (lookup to lookupV ; map to mapV ; [] to []V ; _∷_ to _∷V_)
open import Function using (id ; _∘_ ; flip)
-open import Function.Equality using (_⟶_ ; _⟨$⟩_)
-open import Function.Injection using (module Injection) renaming (Injection to _↪_ ; id to id↪)
open import Relation.Binary using (Setoid ; DecSetoid ; module DecSetoid)
-open import Relation.Binary.PropositionalEquality using (cong) renaming (setoid to EqSetoid)
-open Injection using (to)
open import FinMap
open import Generic using (mapMV ; ≡-to-Π)