Skip to content

Commit 63128f9

Browse files
Merge branch 'master' of https://github.com/agda/agda-stdlib
2 parents 4bd69b4 + 99319e8 commit 63128f9

File tree

4 files changed

+214
-106
lines changed

4 files changed

+214
-106
lines changed

CHANGELOG.md

Lines changed: 10 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -271,11 +271,6 @@ attached to all deprecated names to discourage their use.
271271
decSetoid ↦ ≡-decSetoid
272272
```
273273

274-
* In `Data.Integer.Properties`:
275-
```agda
276-
[1+m]*n≡n+m*n ↦ suc-*
277-
```
278-
279274
* In `Data.List.Relation.Unary.All.Properties`:
280275
```agda
281276
Any¬→¬All ↦ Any¬⇒¬All
@@ -615,6 +610,12 @@ Other minor additions
615610
∣p∣⊔∣q∣≤∣p∪q∣ : ∣ p ∣ ⊔ ∣ q ∣ ≤ ∣ p ∪ q ∣
616611
```
617612

613+
* Added new proofs to `Data.Integer.Properties`:
614+
```agda
615+
suc[i]≤j⇒i<j : sucℤ i ≤ j → i < j
616+
i<j⇒suc[i]≤j : i < j → sucℤ i ≤ j
617+
```
618+
618619
* Added new functions to `Data.List`:
619620
```agda
620621
derun : B.Decidable R → List A → List A
@@ -671,6 +672,10 @@ Other minor additions
671672
deduplicate⁻ : Any P (deduplicate Q? xs) → Any P xs
672673
```
673674

675+
* The implementation of `↭-trans` has been altered in
676+
`Data.List.Relation.Binary.Permutation.Inductive` to avoid
677+
adding unnecessary `refl`s, hence improving it's performance.
678+
674679
* Added new functions to `Data.List.Relation.Binary.Permutation.Setoid`:
675680
```agda
676681
↭-prep : xs ↭ ys → x ∷ xs ↭ x ∷ ys

0 commit comments

Comments
 (0)