summaryrefslogtreecommitdiff
path: root/BFF.agda
diff options
context:
space:
mode:
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)