|
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 | 10 |
|
12 |
| -module Data.List.Fresh.Membership.Setoid.Properties {c ℓ} (S : Setoid c ℓ) where |
| 11 | +module Data.List.Fresh.Membership.Setoid.Properties {c ℓ} (S : Setoid c ℓ) |
| 12 | + where |
13 | 13 |
|
14 | 14 | open import Level using (Level; _⊔_)
|
15 |
| -open import Data.Empty |
16 |
| -open import Data.Nat.Base |
17 |
| -open import Data.Nat.Properties |
| 15 | +open import Data.List.Fresh |
| 16 | +open import Data.List.Fresh.Properties using (fresh-respectsˡ) |
| 17 | +open import Data.List.Fresh.Membership.Setoid S using (_∈_; _∉_) |
| 18 | +open import Data.List.Fresh.Relation.Unary.Any using (Any; here; there; _─_) |
| 19 | +import Data.List.Fresh.Relation.Unary.Any.Properties as List# |
| 20 | + using (length-remove) |
| 21 | +open import Data.Empty using (⊥; ⊥-elim) |
| 22 | +open import Data.Nat.Base using (ℕ; suc; zero; _≤_; _<_; z≤n; s≤s; z<s; s<s) |
| 23 | +open import Data.Nat.Properties using (module ≤-Reasoning) |
18 | 24 | open import Data.Product.Base using (∃; _×_; _,_)
|
19 | 25 | open import Data.Sum.Base as Sum using (_⊎_; inj₁; inj₂; fromInj₂)
|
20 |
| - |
21 | 26 | open import Function.Base using (id; _∘′_; _$_)
|
22 |
| -open import Relation.Nullary |
| 27 | +open import Relation.Binary.Core using (Rel) |
| 28 | +open import Relation.Nullary.Negation.Core using (¬_) |
| 29 | +open import Relation.Nullary using (Irrelevant) |
23 | 30 | open import Relation.Unary as Unary using (Pred)
|
24 |
| -import Relation.Binary.Definitions as Binary |
| 31 | +import Relation.Binary.Definitions as Binary using (_Respectsˡ_; Irrelevant) |
25 | 32 | import Relation.Binary.PropositionalEquality.Core as ≡
|
26 |
| -open import Relation.Nary |
27 |
| - |
28 |
| -open import Data.List.Fresh |
29 |
| -open import Data.List.Fresh.Properties |
30 |
| -open import Data.List.Fresh.Membership.Setoid S |
31 |
| -open import Data.List.Fresh.Relation.Unary.Any using (Any; here; there; _─_) |
32 |
| -import Data.List.Fresh.Relation.Unary.Any.Properties as List# |
| 33 | + using (_≡_; cong; sym; subst) |
| 34 | +open import Relation.Nary using (∀[_]; _⇒_) |
33 | 35 |
|
34 | 36 | open Setoid S renaming (Carrier to A)
|
35 | 37 |
|
|
0 commit comments