diff options
author | Helmut Grohne <helmut@subdivi.de> | 2012-02-09 15:08:36 +0100 |
---|---|---|
committer | Helmut Grohne <helmut@subdivi.de> | 2012-02-09 15:08:36 +0100 |
commit | af1cc6bc8685515ffbf269e420449219a105301c (patch) | |
tree | dc54387a8776c06bbcf10e7670653586cc5649a0 /Bidir.agda | |
parent | e0f83c9ca1816a4c0b3c030bb2cd562156311ecd (diff) | |
download | bidiragda-af1cc6bc8685515ffbf269e420449219a105301c.tar.gz |
prove lemma-union-generate
Diffstat (limited to 'Bidir.agda')
-rw-r--r-- | Bidir.agda | 3 |
1 files changed, 0 insertions, 3 deletions
@@ -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) |