diff options
author | Helmut Grohne <helmut@subdivi.de> | 2019-09-29 13:54:46 +0200 |
---|---|---|
committer | Helmut Grohne <helmut@subdivi.de> | 2019-09-29 13:54:46 +0200 |
commit | 6ce567bf63a61bce4ccf71e3ec402d94d1da2fb1 (patch) | |
tree | b8fcf765afd7da6f300221f02da215696e2be4a2 /Bidir.agda | |
parent | 8435606d98e418394edbe5104b3f425e56a5a207 (diff) | |
download | bidiragda-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 'Bidir.agda')
-rw-r--r-- | Bidir.agda | 8 |
1 files changed, 5 insertions, 3 deletions
@@ -8,8 +8,10 @@ open import Data.Fin using (Fin) import Level import Category.Monad import Category.Functor -open import Data.Maybe using (Maybe ; nothing ; just ; maybe′ ; drop-just ; just-injective) renaming (setoid to MaybeSetoid ; Eq to MaybeEq) +open import Data.Maybe using (Maybe ; nothing ; just ; maybe′) import Data.Maybe.Categorical +open import Data.Maybe.Properties using (just-injective) +open import Data.Maybe.Relation.Binary.Pointwise using (just ; nothing ; drop-just) renaming (setoid to MaybeSetoid ; Pointwise to MaybeEq) open Category.Monad.RawMonad {Level.zero} Data.Maybe.Categorical.monad using (_>>=_) open Category.Functor.RawFunctor {Level.zero} Data.Maybe.Categorical.functor using (_<$>_) open import Data.List using (List) @@ -100,7 +102,7 @@ lemma-fmap-denumerate-enumerate : {S : Set} {C : Set → S → Set} → (ShapeT lemma-fmap-denumerate-enumerate {S} {C} ShapeT {s = s} c = begin fmap (denumerate ShapeT c) (fill s (allFin (arity s))) ≡⟨ fill-fmap (denumerate ShapeT c) s (allFin (arity s)) ⟩ - fill s (map (flip lookupVec (content c)) (allFin (arity s))) + fill s (map (lookupVec (content c)) (allFin (arity s))) ≡⟨ P.cong (fill s) (map-lookup-allFin (content c)) ⟩ fill s (content c) ≡⟨ content-fill c ⟩ @@ -275,7 +277,7 @@ module _ (G : Get) where contentV (fmapV (flip lookupM (h↦h′ h)) (get t)) ≡⟨ Shaped.fmap-content ViewShapeT (flip lookupM (h↦h′ h)) (get t) ⟩ map (flip lookupM (h↦h′ h)) (contentV (get t)) - ≡⟨ lemma-exchange-maps (lemma-union-not-used h (reshape g′ (arityS (gl₁ j)))) (lemma-assoc-domain (contentV (get t)) (contentV v) ph) ⟩ + ≡⟨ lemma-exchange-maps (h↦h′ h) h (lemma-union-not-used h (reshape g′ (arityS (gl₁ j)))) (lemma-assoc-domain (contentV (get t)) (contentV v) ph) ⟩ map (flip lookupM h) (contentV (get t)) ≈⟨ lemma-2 (contentV (get t)) (contentV v) h ph ⟩ map just (contentV v) |