diff options
author | Helmut Grohne <grohne@cs.uni-bonn.de> | 2014-01-28 09:16:26 +0100 |
---|---|---|
committer | Helmut Grohne <grohne@cs.uni-bonn.de> | 2014-01-28 09:16:26 +0100 |
commit | 8cc43c2c7e5ab40394a1e6a23470edb3d2d6b909 (patch) | |
tree | 563cd32156d9fd7eb63c072698b4608b14d64cf9 /Bidir.agda | |
parent | 09cf8a92e03a4cebffdf9bb58aaf1b01b55e73a3 (diff) | |
download | bidiragda-8cc43c2c7e5ab40394a1e6a23470edb3d2d6b909.tar.gz |
cleanup unused function and import
Diffstat (limited to 'Bidir.agda')
-rw-r--r-- | Bidir.agda | 6 |
1 files changed, 1 insertions, 5 deletions
@@ -25,7 +25,7 @@ import Relation.Binary.EqReasoning as EqR import FreeTheorems open FreeTheorems.VecVec using (get-type ; free-theorem) -open import Generic using (just-injective ; vecIsSetoid ; mapMV ; mapMV-cong ; mapMV-purity ; sequenceV ; sequence-map) +open import Generic using (vecIsSetoid ; mapMV ; mapMV-cong ; mapMV-purity ; sequenceV ; sequence-map) open import FinMap import CheckInsert open CheckInsert A @@ -170,10 +170,6 @@ lemma-union-not-used h h' (i β· is') (Data.List.All._β·_ (x , px) p') = congβ (lemma-union-not-used h h' is' p') where open β‘-Reasoning -map-just-β-injective : {n : β} {x y : Vec Carrier n} β Setoid._β_ (vecIsSetoid (MaybeSetoid A.setoid) n) (map just x) (map just y) β Setoid._β_ (vecIsSetoid A.setoid n) x y -map-just-β-injective {x = []} {y = []} VecEq.[]-cong = VecEq.[]-cong -map-just-β-injective {x = _ β· _} {y = _ β· _} (just xβy VecEq.β·-cong ps) = xβy VecEq.β·-cong map-just-β-injective ps - lemma->>=-just : {A B : Set} (ma : Maybe A) {f : A β Maybe B} {b : B} β (ma >>= f) β‘ just b β β Ξ» a β ma β‘ just a lemma->>=-just (just a) p = a , refl lemma->>=-just nothing () |