Skip to content

Commit

Permalink
remove unnecessary parameter from `Relation.Binary.Reasoning.Base.Apa…
Browse files Browse the repository at this point in the history
…rtness` (#2438)

Co-authored-by: MatthewDaggitt <matthewdaggitt@gmail.com>
  • Loading branch information
damhiya and MatthewDaggitt authored Aug 14, 2024
1 parent ab0038b commit b6cf220
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 1 deletion.
3 changes: 3 additions & 0 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,9 @@ Highlights
Bug-fixes
---------

* Removed unnecessary parameter `#-trans : Transitive _#_` from
`Relation.Binary.Reasoning.Base.Apartness`.

Non-backwards compatible changes
--------------------------------

Expand Down
2 changes: 1 addition & 1 deletion src/Relation/Binary/Reasoning/Base/Apartness.agda
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,7 @@ open import Relation.Binary.Reasoning.Syntax
module Relation.Binary.Reasoning.Base.Apartness {a ℓ₁ ℓ₂} {A : Set a}
{_≈_ : Rel A ℓ₁} {_#_ : Rel A ℓ₂}
(≈-equiv : IsEquivalence _≈_)
(#-trans : Transitive _#_) (#-sym : Symmetric _#_)
(#-sym : Symmetric _#_)
(#-≈-trans : Trans _#_ _≈_ _#_) (≈-#-trans : Trans _≈_ _#_ _#_)
where

Expand Down

0 comments on commit b6cf220

Please sign in to comment.