File tree 1 file changed +3
-2
lines changed
1 file changed +3
-2
lines changed Original file line number Diff line number Diff line change @@ -13,7 +13,7 @@ module Data.List.Membership.Setoid {c ℓ} (S : Setoid c ℓ) where
13
13
14
14
open import Function.Base using (_∘_; id; flip)
15
15
open import Data.List.Base as List using (List; []; _∷_; length; lookup)
16
- open import Data.List.Relation.Unary.Any
16
+ open import Data.List.Relation.Unary.Any as Any
17
17
using (Any; index; map; here; there)
18
18
open import Data.Product.Base as Prod using (∃; _×_; _,_)
19
19
open import Relation.Unary using (Pred)
@@ -35,7 +35,8 @@ x ∉ xs = ¬ x ∈ xs
35
35
------------------------------------------------------------------------
36
36
-- Operations
37
37
38
- open Data.List.Relation.Unary.Any using (_∷=_; _─_) public
38
+ _∷=_ = Any._∷=_ {A = A}
39
+ _─_ = Any._─_ {A = A}
39
40
40
41
mapWith∈ : ∀ {b} {B : Set b}
41
42
(xs : List A) → (∀ {x} → x ∈ xs → B) → List B
You can’t perform that action at this time.
0 commit comments