We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent d3c5037 commit 2d9f276Copy full SHA for 2d9f276
src/Relation/Binary/Reasoning/Base/Apartness.agda
@@ -20,7 +20,7 @@ open import Relation.Binary.Reasoning.Syntax
20
module Relation.Binary.Reasoning.Base.Apartness {a ℓ₁ ℓ₂} {A : Set a}
21
{_≈_ : Rel A ℓ₁} {_#_ : Rel A ℓ₂}
22
(≈-equiv : IsEquivalence _≈_)
23
- (#-trans : Transitive _#_) (#-sym : Symmetric _#_)
+ (#-sym : Symmetric _#_)
24
(#-≈-trans : Trans _#_ _≈_ _#_) (≈-#-trans : Trans _≈_ _#_ _#_)
25
where
26
0 commit comments