File tree Expand file tree Collapse file tree 2 files changed +5
-11
lines changed
src/Data/List/Relation/Unary/Unique Expand file tree Collapse file tree 2 files changed +5
-11
lines changed Original file line number Diff line number Diff line change 9
9
module Data.List.Relation.Unary.Unique.Propositional {a} {A : Set a} where
10
10
11
11
open import Relation.Binary.PropositionalEquality.Properties using (setoid)
12
- open import Data.List.Relation.Unary.Unique.Setoid as SetoidUnique
13
12
14
13
------------------------------------------------------------------------
15
14
-- Re-export the contents of setoid uniqueness
16
15
17
- open SetoidUnique (setoid A) public
16
+ open import Data.List.Relation.Unary.Unique.Setoid (setoid A) public
17
+
Original file line number Diff line number Diff line change 6
6
7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
- open import Relation.Binary.Core using (Rel)
10
9
open import Relation.Binary.Bundles using (Setoid)
11
- open import Relation.Nullary.Negation using (¬_)
12
10
13
11
module Data.List.Relation.Unary.Unique.Setoid {a ℓ} (S : Setoid a ℓ) where
14
12
15
- open Setoid S renaming (Carrier to A )
13
+ open Setoid S using (_≉_ )
16
14
17
15
------------------------------------------------------------------------
18
16
-- Definition
19
17
20
- private
21
- Distinct : Rel A ℓ
22
- Distinct x y = ¬ (x ≈ y)
23
-
24
- open import Data.List.Relation.Unary.AllPairs.Core Distinct public
18
+ open import Data.List.Relation.Unary.AllPairs.Core _≉_ public
25
19
renaming (AllPairs to Unique)
26
20
27
- open import Data.List.Relation.Unary.AllPairs {R = Distinct } public
21
+ open import Data.List.Relation.Unary.AllPairs {R = _≉_ } public
28
22
using (head; tail)
You can’t perform that action at this time.
0 commit comments