File tree 2 files changed +9
-5
lines changed
2 files changed +9
-5
lines changed Original file line number Diff line number Diff line change @@ -11,6 +11,10 @@ Bug-fixes
11
11
12
12
* Removed unnecessary parameter ` #-trans : Transitive _#_ ` from
13
13
` Relation.Binary.Reasoning.Base.Apartness ` .
14
+ * Relax the types for ` ≡-syntax ` in ` Relation.Binary.HeterogeneousEquality ` .
15
+ These operators are used for equational reasoning of heterogeneous equality
16
+ ` x ≅ y ` , but previously the three operators in ` ≡-syntax ` unnecessarily require
17
+ ` x ` and ` y ` to have the same type, making them unusable in most situations.
14
18
15
19
Non-backwards compatible changes
16
20
--------------------------------
Original file line number Diff line number Diff line change @@ -234,22 +234,22 @@ module ≅-Reasoning where
234
234
235
235
infix 4 _IsRelatedTo_
236
236
237
- data _IsRelatedTo_ {A : Set ℓ } {B : Set ℓ } (x : A) (y : B) : Set ℓ where
237
+ data _IsRelatedTo_ {A : Set a } {B : Set b } (x : A) (y : B) : Set a where
238
238
relTo : (x≅y : x ≅ y) → x IsRelatedTo y
239
239
240
240
start : ∀ {x : A} {y : B} → x IsRelatedTo y → x ≅ y
241
241
start (relTo x≅y) = x≅y
242
242
243
- ≡-go : ∀ {A : Set a} → Trans {A = A} {C = A } _≡_ _IsRelatedTo_ _IsRelatedTo_
243
+ ≡-go : ∀ {A : Set a} {B : Set b} → Trans {A = A} {C = B } _≡_ _IsRelatedTo_ _IsRelatedTo_
244
244
≡-go x≡y (relTo y≅z) = relTo (trans (reflexive x≡y) y≅z)
245
245
246
246
-- Combinators with one heterogeneous relation
247
- module _ {A : Set ℓ } {B : Set ℓ } where
247
+ module _ {A : Set a } {B : Set b } where
248
248
open begin-syntax (_IsRelatedTo_ {A = A} {B}) start public
249
+ open ≡-syntax (_IsRelatedTo_ {A = A} {B}) ≡-go public
249
250
250
251
-- Combinators with homogeneous relations
251
- module _ {A : Set ℓ} where
252
- open ≡-syntax (_IsRelatedTo_ {A = A}) ≡-go public
252
+ module _ {A : Set a} where
253
253
open end-syntax (_IsRelatedTo_ {A = A}) (relTo refl) public
254
254
255
255
-- Can't create syntax in the standard `Syntax` module for
You can’t perform that action at this time.
0 commit comments