summaryrefslogtreecommitdiff
path: root/Bidir.agda
diff options
context:
space:
mode:
authorHelmut Grohne <helmut@subdivi.de>2012-02-09 15:08:36 +0100
committerHelmut Grohne <helmut@subdivi.de>2012-02-09 15:08:36 +0100
commitaf1cc6bc8685515ffbf269e420449219a105301c (patch)
treedc54387a8776c06bbcf10e7670653586cc5649a0 /Bidir.agda
parente0f83c9ca1816a4c0b3c030bb2cd562156311ecd (diff)
downloadbidiragda-af1cc6bc8685515ffbf269e420449219a105301c.tar.gz
prove lemma-union-generate
Diffstat (limited to 'Bidir.agda')
-rw-r--r--Bidir.agda3
1 files changed, 0 insertions, 3 deletions
diff --git a/Bidir.agda b/Bidir.agda
index 4e7d46e..332cc55 100644
--- a/Bidir.agda
+++ b/Bidir.agda
@@ -130,9 +130,6 @@ lemma-map-denumerate-enumerate (a ∷ as) = cong (_∷_ a) (begin
≡⟨ lemma-map-denumerate-enumerate as ⟩
as ∎)
-lemma-union-generate : {A : Set} {n : ℕ} → (f : Fin n → A) → (is : List (Fin n)) → union (generate f is) (fromFunc f) ≡ fromFunc f
-lemma-union-generate f is = {!!}
-
theorem-1 : (get : {α : Set} → List α → List α) → {τ : Set} → (eq : EqInst τ) → (s : List τ) → bff get eq s (get s) ≡ just s
theorem-1 get eq s = begin
bff get eq s (get s)