IndexedMap.agda 426 B

12345678910111213
  1. open import Relation.Binary
  2. open import Relation.Binary.PropositionalEquality
  3. open import Data.Product
  4. open import Level
  5. module IndexedMap
  6. {Index : Set} {Key : Index → Set} {_≈_ _<_ : Rel (∃ Key) zero}
  7. (isOrderedKeySet : IsStrictTotalOrder _≈_ _<_)
  8. -- Equal keys must have equal indices.
  9. (indicesEqual : _≈_ =[ proj₁ ]⇒ _≡_)
  10. (Value : Index → Set)
  11. where