Prove that maps are functional assuming uniqueness
This commit is contained in:
@@ -76,7 +76,6 @@ module IsEquivalenceInstances where
|
||||
|
||||
open import Map A B ≡-dec-A using (Map; lift; subset; insert)
|
||||
open import Data.List using (_∷_; []) -- TODO: re-export these with nicer names from map
|
||||
open import Data.List.Relation.Unary.Any using (Any; here; there) -- TODO: re-export these with nicer names from map
|
||||
|
||||
open IsEquivalence eB renaming
|
||||
( ≈-refl to ≈₂-refl
|
||||
|
||||
Reference in New Issue
Block a user