summaryrefslogtreecommitdiff
path: root/Bidir.agda
diff options
context:
space:
mode:
authorHelmut Grohne <helmut@subdivi.de>2012-02-09 15:56:29 +0100
committerHelmut Grohne <helmut@subdivi.de>2012-02-09 15:56:29 +0100
commitdf9a08b332fff377d06d973535017d891f5a3416 (patch)
tree0345db8eb53106f5aad3e82062252192e8600943 /Bidir.agda
parentab5bd5693f85750462418566e0310cb42a6cf6b0 (diff)
downloadbidiragda-df9a08b332fff377d06d973535017d891f5a3416.tar.gz
rephrase free-theorem-list-list using pointwise equality
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 23381d0..57b77db 100644
--- a/Bidir.agda
+++ b/Bidir.agda
@@ -11,7 +11,7 @@ open import Function using (id ; _∘_ ; flip)
open import Relation.Nullary using (Dec ; yes ; no)
open import Relation.Nullary.Negation using (contradiction)
open import Relation.Binary.Core using (_≡_ ; refl)
-open import Relation.Binary.PropositionalEquality using (cong ; sym ; inspect ; Reveal_is_)
+open import Relation.Binary.PropositionalEquality using (cong ; sym ; inspect ; Reveal_is_ ; _≗_)
open Relation.Binary.PropositionalEquality.≡-Reasoning using (begin_ ; _≡⟨_⟩_ ; _∎)
open import FinMap
@@ -109,7 +109,7 @@ bff get eq s v = let s′ = enumerate s
in fmap (flip map s′ ∘ flip lookup) h′
postulate
- free-theorem-list-list : {β γ : Set} → (get : {α : Set} → List α → List α) → (f : β → γ) → (l : List β) → get (map f l) ≡ map f (get l)
+ free-theorem-list-list : {β γ : Set} → (get : {α : Set} → List α → List α) → (f : β → γ) → get ∘ map f ≗ map f ∘ get
toList-map-commutes : {A B : Set} {n : ℕ} → (f : A → B) → (v : Data.Vec.Vec A n) → (toList (Data.Vec.map f v)) ≡ map f (toList v)
toList-map-commutes f Data.Vec.[] = refl