summaryrefslogtreecommitdiff
path: root/FinMap.agda
diff options
context:
space:
mode:
authorHelmut Grohne <helmut@subdivi.de>2012-04-19 11:58:40 +0200
committerHelmut Grohne <helmut@subdivi.de>2012-04-19 11:58:40 +0200
commitfcf8bd5d0530dd6b05ba5c2931a66171b823e651 (patch)
treeb0e7bb8582dc2c46a80f3417c5572e81deb39008 /FinMap.agda
parent7c3e2c61e55aa876f88fbd34c94ccfb0a8c715d4 (diff)
downloadbidiragda-fcf8bd5d0530dd6b05ba5c2931a66171b823e651.tar.gz
FinMap: lemma-lookupM-restrict drop useless implicit
Diffstat (limited to 'FinMap.agda')
-rw-r--r--FinMap.agda2
1 files changed, 1 insertions, 1 deletions
diff --git a/FinMap.agda b/FinMap.agda
index 81862f6..ff5dda7 100644
--- a/FinMap.agda
+++ b/FinMap.agda
@@ -72,7 +72,7 @@ lemma-from-just : {A : Set} → {x y : A} → _≡_ {_} {Maybe A} (just x) (just
lemma-from-just refl = refl
lemma-lookupM-restrict : {A : Set} {n : ℕ} → (i : Fin n) → (f : Fin n → A) → (is : List (Fin n)) → (a : A) → lookupM i (restrict f is) ≡ just a → f i ≡ a
-lemma-lookupM-restrict {A} i f [] a p = lemma-just≢nothing (trans (sym p) (lemma-lookupM-empty i))
+lemma-lookupM-restrict i f [] a p = lemma-just≢nothing (trans (sym p) (lemma-lookupM-empty i))
lemma-lookupM-restrict i f (i' ∷ is) a p with i ≟ i'
lemma-lookupM-restrict i f (.i ∷ is) a p | yes refl = lemma-from-just (begin
just (f i)