summaryrefslogtreecommitdiff
path: root/BFF.agda
diff options
context:
space:
mode:
authorHelmut Grohne <helmut@subdivi.de>2012-10-05 12:47:09 +0200
committerHelmut Grohne <helmut@subdivi.de>2012-10-05 12:47:09 +0200
commit7ba21759412a8b356f7790ac5f5e413302331183 (patch)
tree58b2f83f1abe029596071e0b151470b122e72102 /BFF.agda
parent96e45ecbf31c5685fa914882ec4b21b1392c49fc (diff)
downloadbidiragda-7ba21759412a8b356f7790ac5f5e413302331183.tar.gz
move all postulates to one module
This should make it easier to see what is assumed.
Diffstat (limited to 'BFF.agda')
-rw-r--r--BFF.agda7
1 files changed, 3 insertions, 4 deletions
diff --git a/BFF.agda b/BFF.agda
index 546782d..612c2c3 100644
--- a/BFF.agda
+++ b/BFF.agda
@@ -9,6 +9,7 @@ open import Function using (id ; _∘_ ; flip)
open import FinMap
open import CheckInsert
+import FreeTheorems
_>>=_ : {A B : Set} → Maybe A → (A → Maybe B) → Maybe B
_>>=_ = flip (flip maybe′ nothing)
@@ -17,8 +18,7 @@ fmap : {A B : Set} → (A → B) → Maybe A → Maybe B
fmap f = maybe′ (λ a → just (f a)) nothing
module ListBFF where
- get-type : Set₁
- get-type = {A : Set} → List A → List A
+ open FreeTheorems.ListList public using (get-type)
assoc : {A : Set} {n : ℕ} → EqInst A → List (Fin n) → List A → Maybe (FinMapMaybe n A)
assoc _ [] [] = just empty
@@ -39,8 +39,7 @@ module ListBFF where
in fmap (flip map s′ ∘ flip lookup) h′
module VecBFF where
- get-type : (ℕ → ℕ) → Set₁
- get-type getlen = {A : Set} {n : ℕ} → Vec A n → Vec A (getlen n)
+ open FreeTheorems.VecVec public using (get-type)
assoc : {A : Set} {n m : ℕ} → EqInst A → Vec (Fin n) m → Vec A m → Maybe (FinMapMaybe n A)
assoc _ []V []V = just empty