------------------------------------------------------------------------ -- The Agda standard library -- -- Vectors made up entirely of unique elements (setoid equality) ------------------------------------------------------------------------ {-# OPTIONS --cubical-compatible --safe #-} open import Relation.Binary.Core using (Rel) open import Relation.Binary.Bundles using (Setoid) module Data.Vec.Relation.Unary.Unique.Setoid {a ℓ} (S : Setoid a ℓ) where open Setoid S renaming (Carrier to A) open import Data.Vec.Base import Data.Vec.Relation.Unary.AllPairs as AllPairsM open import Level using (_⊔_) open import Relation.Unary using (Pred) open import Relation.Nullary.Negation using (¬_) ------------------------------------------------------------------------ -- Definition private Distinct : Rel A ℓ Distinct x y = ¬ (x ≈ y) open import Data.Vec.Relation.Unary.AllPairs.Core Distinct public renaming (AllPairs to Unique) open import Data.Vec.Relation.Unary.AllPairs {R = Distinct} public using (head; tail)
RetroSearch is an open source project built by @garambo | Open a GitHub Issue
Search and Browse the WWW like it's 1997 | Search results from DuckDuckGo
HTML:
3.2
| Encoding:
UTF-8
| Version:
0.7.4