Skip to content

Commit f7094cc

Browse files
authored
[ fix #2153 ] Properly re-export specialised combinators (#2161)
1 parent cdb11b8 commit f7094cc

File tree

2 files changed

+6
-2
lines changed

2 files changed

+6
-2
lines changed

CHANGELOG.md

+3
Original file line numberDiff line numberDiff line change
@@ -33,6 +33,9 @@ Bug-fixes
3333
in `Function.Construct.Composition` had their arguments in the wrong order. They have
3434
been flipped so they can actually be used as a composition operator.
3535

36+
* The operations `_∷=_` and `_─_` exported from `Data.List.Membership.Setoid`
37+
had an extraneous `{A : Set a}` parameter. This has been removed.
38+
3639
* The combinators `_≃⟨_⟩_` and `_≃˘⟨_⟩_` in `Data.Rational.Properties.≤-Reasoning`
3740
now correctly accepts proofs of type `_≃_` instead of the previous proofs of type `_≡_`.
3841

src/Data/List/Membership/Setoid.agda

+3-2
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ module Data.List.Membership.Setoid {c ℓ} (S : Setoid c ℓ) where
1313

1414
open import Function.Base using (_∘_; id; flip)
1515
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
1717
using (Any; index; map; here; there)
1818
open import Data.Product.Base as Prod using (∃; _×_; _,_)
1919
open import Relation.Unary using (Pred)
@@ -35,7 +35,8 @@ x ∉ xs = ¬ x ∈ xs
3535
------------------------------------------------------------------------
3636
-- Operations
3737

38-
open Data.List.Relation.Unary.Any using (_∷=_; _─_) public
38+
_∷=_ = Any._∷=_ {A = A}
39+
_─_ = Any._─_ {A = A}
3940

4041
mapWith∈ : {b} {B : Set b}
4142
(xs : List A) ( {x} x ∈ xs B) List B

0 commit comments

Comments
 (0)