diff --git a/CHANGELOG.md b/CHANGELOG.md index 494cfbb6a5..8795b734a6 100644 --- a/CHANGELOG.md +++ b/CHANGELOG.md @@ -460,6 +460,11 @@ Backwards compatible changes All₂-concat⁻ : All₂ _~_ (concat xss) (concat yss) → All₂ (All₂ _~_) xss yss ``` +* Added proofs to `Relation.Binary.Consequences` + ```agda + P-resp⟶¬P-resp : Symmetric _≈_ → P Respects _≈_ → (¬_ ∘ P) Respects _≈_ + ``` + Version 0.13 ============ diff --git a/src/Relation/Binary/Consequences.agda b/src/Relation/Binary/Consequences.agda index 4b0f071eae..dafdc88161 100644 --- a/src/Relation/Binary/Consequences.agda +++ b/src/Relation/Binary/Consequences.agda @@ -114,6 +114,11 @@ trans∧tri⟶resp≈ {_≈_ = _≈_} {_<_} sym trans <-trans tri = ... | tri≈ _ y≈z _ = ⊥-elim (tri⟶irr tri (trans x≈y y≈z) x _ _ z