summaryrefslogtreecommitdiff
path: root/BFF.agda
diff options
context:
space:
mode:
authorHelmut Grohne <helmut@subdivi.de>2019-09-29 13:54:46 +0200
committerHelmut Grohne <helmut@subdivi.de>2019-09-29 13:54:46 +0200
commit6ce567bf63a61bce4ccf71e3ec402d94d1da2fb1 (patch)
treeb8fcf765afd7da6f300221f02da215696e2be4a2 /BFF.agda
parent8435606d98e418394edbe5104b3f425e56a5a207 (diff)
downloadbidiragda-6ce567bf63a61bce4ccf71e3ec402d94d1da2fb1.tar.gz
port to agda/2.6.0.1 and agda-stdlib/1.1
* Data.Vec.lookup changed parameter order. * A number of symbols were moved from Data.Maybe to submodules. * In a number of occasions, agda no longer figures implicit arguments and they had to be made explicit. * We can no longer use heterogeneous proofs inside equational reasoning for propositional equality. Use heterogeneous equational reasoning. * Stop importing proof-irrelevance as that would require K.
Diffstat (limited to 'BFF.agda')
-rw-r--r--BFF.agda2
1 files changed, 1 insertions, 1 deletions
diff --git a/BFF.agda b/BFF.agda
index 06744f6..74380a9 100644
--- a/BFF.agda
+++ b/BFF.agda
@@ -35,7 +35,7 @@ module PartialShapeBFF (A : DecSetoid ℓ₀ ℓ₀) where
where open Shaped ShapeT
denumerate : {S : Set} {C : Set → S → Set} → (ShapeT : Shaped S C) → {α : Set} {s : S} → (c : C α s) → Fin (Shaped.arity ShapeT s) → α
- denumerate ShapeT c = flip lookupV (Shaped.content ShapeT c)
+ denumerate ShapeT c = lookupV (Shaped.content ShapeT c)
bff : (G : Get) → {i : Get.I G} → (j : Get.I G) → Get.SourceContainer G Carrier (Get.gl₁ G i) → Get.ViewContainer G Carrier (Get.gl₂ G j) → Maybe (Get.SourceContainer G (Maybe Carrier) (Get.gl₁ G j))
bff G {i} j s v = let s′ = enumerate SourceShapeT (gl₁ i)