summaryrefslogtreecommitdiff
path: root/Bidir.agda
diff options
context:
space:
mode:
authorHelmut Grohne <grohne@cs.uni-bonn.de>2014-02-10 15:50:27 +0100
committerHelmut Grohne <grohne@cs.uni-bonn.de>2014-02-10 15:50:27 +0100
commit6cc566c46889c5e7aafc8d75c6627137e56ab30f (patch)
tree092dce779785d17f572dfd1880baa23c69cd1a33 /Bidir.agda
parent586d72e18898311d975f5748bca397c403b6a83b (diff)
parent04b7bf8fabf64a2414d64cfb385f6a397da0a0fb (diff)
downloadbidiragda-6cc566c46889c5e7aafc8d75c6627137e56ab30f.tar.gz
Merge branch master into feature-shape-update
For building on the sieve example.
Diffstat (limited to 'Bidir.agda')
-rw-r--r--Bidir.agda4
1 files changed, 2 insertions, 2 deletions
diff --git a/Bidir.agda b/Bidir.agda
index 9765392..f0b7bc1 100644
--- a/Bidir.agda
+++ b/Bidir.agda
@@ -178,8 +178,8 @@ lemma->>=-just (just a) p = a , refl
lemma->>=-just nothing ()
lemma-just-sequence : {A : Set} {n : ℕ} → (v : Vec A n) → sequenceV (map just v) ≡ just v
-lemma-just-sequence [] = refl
-lemma-just-sequence (x ∷ xs) rewrite lemma-just-sequence xs = refl
+lemma-just-sequence [] = refl
+lemma-just-sequence (x ∷ xs) = cong (_<$>_ (_∷_ x)) (lemma-just-sequence xs)
lemma-mapM-successful : {A B : Set} {f : A → Maybe B} {n : ℕ} → (v : Vec A n) → {r : Vec B n} → mapMV f v ≡ just r → ∃ λ w → map f v ≡ map just w
lemma-mapM-successful [] p = [] , refl