summaryrefslogtreecommitdiff
path: root/Precond.agda
diff options
context:
space:
mode:
authorHelmut Grohne <grohne@cs.uni-bonn.de>2014-01-23 13:19:02 +0100
committerHelmut Grohne <grohne@cs.uni-bonn.de>2014-01-23 13:19:02 +0100
commitaf1ea86b6e817a85d4d160833fc5d4bb89e2df7b (patch)
tree1a634eae43fb1656bda3f5a3bb856b744131c73d /Precond.agda
parent9cb635bb49c1846da7f9c00cc475b0fac9a2fa42 (diff)
downloadbidiragda-af1ea86b6e817a85d4d160833fc5d4bb89e2df7b.tar.gz
generalize BFF and theorem-2 to arbitrary Setoids
Since the generalization of lemma-checkInsert-restrict there is nothing to show for theorem-1. So everything works with Setoids now yielding the same results as the paper proofs.
Diffstat (limited to 'Precond.agda')
-rw-r--r--Precond.agda2
1 files changed, 1 insertions, 1 deletions
diff --git a/Precond.agda b/Precond.agda
index 41e3407..9bae83b 100644
--- a/Precond.agda
+++ b/Precond.agda
@@ -26,7 +26,7 @@ open CheckInsert (decSetoid deq) using (checkInsert ; lemma-checkInsert-new ; le
import BFF
import Bidir
-open BFF.VecBFF Carrier deq using (get-type ; assoc ; enumerate ; denumerate ; bff)
+open BFF.VecBFF (decSetoid deq) using (get-type ; assoc ; enumerate ; denumerate ; bff)
assoc-enough : {getlen : ℕ → ℕ} (get : get-type getlen) → {m : ℕ} → (s : Vec Carrier m) → (v : Vec Carrier (getlen m)) → ∃ (λ h → assoc (get (enumerate s)) v ≡ just h) → ∃ λ u → bff get s v ≡ just u
assoc-enough get s v (h , p) = u , cong (_<$>_ (flip map s′ ∘ flip lookup) ∘ (_<$>_ (flip union g))) p