File tree Expand file tree Collapse file tree 3 files changed +11
-8
lines changed Expand file tree Collapse file tree 3 files changed +11
-8
lines changed Original file line number Diff line number Diff line change @@ -784,6 +784,9 @@ Non-backwards compatible changes
784
784
properties about the orderings themselves the second index must be provided
785
785
explicitly.
786
786
787
+ * The argument ` xs ` in ` xs≮[] ` in ` Data.{List|Vec}.Relation.Binary.Lex.Strict `
788
+ introduced in PRs #1648 and #1672 has now been made implicit.
789
+
787
790
* Issue #2075 (Johannes Waldmann): wellfoundedness of the lexicographic ordering
788
791
on products, defined in ` Data.Product.Relation.Binary.Lex.Strict ` , no longer
789
792
requires the assumption of symmetry for the first equality relation ` _≈₁_ ` ,
@@ -2705,7 +2708,7 @@ Other minor changes
2705
2708
2706
2709
* Added new proofs in ` Data.Vec.Relation.Binary.Lex.Strict ` :
2707
2710
``` agda
2708
- xs≮[] : ∀ {n} ( xs : Vec A n) → ¬ xs < []
2711
+ xs≮[] : { xs : Vec A n} → ¬ xs < []
2709
2712
<-respectsˡ : IsPartialEquivalence _≈_ → _≺_ Respectsˡ _≈_ →
2710
2713
∀ {m n} → _Respectsˡ_ (_<_ {m} {n}) _≋_
2711
2714
<-respectsʳ : IsPartialEquivalence _≈_ → _≺_ Respectsʳ _≈_ →
Original file line number Diff line number Diff line change @@ -51,11 +51,11 @@ module _ {a ℓ₁ ℓ₂} {A : Set a} where
51
51
_≋_ = Pointwise _≈_
52
52
_<_ = Lex-< _≈_ _≺_
53
53
54
- xs≮[] : ∀ xs → ¬ xs < []
55
- xs≮[] _ (base ())
54
+ xs≮[] : ∀ {xs} → ¬ xs < []
55
+ xs≮[] (base ())
56
56
57
57
¬[]<[] : ¬ [] < []
58
- ¬[]<[] = xs≮[] []
58
+ ¬[]<[] = xs≮[]
59
59
60
60
<-irreflexive : Irreflexive _≈_ _≺_ → Irreflexive _≋_ _<_
61
61
<-irreflexive irr (x≈y ∷ xs≋ys) (this x<y) = irr x≈y x<y
Original file line number Diff line number Diff line change @@ -69,11 +69,11 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
69
69
_≋_ = Pointwise _≈_
70
70
_<_ = Lex-< _≈_ _≺_
71
71
72
- xs≮[] : ∀ {n} ( xs : Vec A n) → ¬ xs < []
73
- xs≮[] _ (base ())
72
+ xs≮[] : ∀ {n} { xs : Vec A n} → ¬ xs < []
73
+ xs≮[] (base ())
74
74
75
75
¬[]<[] : ¬ [] < []
76
- ¬[]<[] = xs≮[] []
76
+ ¬[]<[] = xs≮[]
77
77
78
78
module _ (≺-irrefl : Irreflexive _≈_ _≺_) where
79
79
@@ -134,7 +134,7 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
134
134
where
135
135
136
136
<-wellFounded : ∀ {n} → WellFounded (_<_ {n})
137
- <-wellFounded {0 } [] = acc λ ys ys<[] → ⊥-elim (xs≮[] ys ys <[])
137
+ <-wellFounded {0 } [] = acc λ ys ys<[] → ⊥-elim (xs≮[] ys<[])
138
138
<-wellFounded {suc n} xs = Subrelation.wellFounded <⇒uncons-Lex uncons-Lex-wellFounded xs
139
139
where
140
140
<⇒uncons-Lex : {xs ys : Vec A (suc n)} → xs < ys → (×-Lex _≈_ _≺_ _<_ on uncons) xs ys
You can’t perform that action at this time.
0 commit comments