File tree Expand file tree Collapse file tree 4 files changed +214
-106
lines changed
List/Relation/Binary/Permutation Expand file tree Collapse file tree 4 files changed +214
-106
lines changed Original file line number Diff line number Diff line change @@ -271,11 +271,6 @@ attached to all deprecated names to discourage their use.
271
271
decSetoid ↦ ≡-decSetoid
272
272
```
273
273
274
- * In ` Data.Integer.Properties ` :
275
- ``` agda
276
- [1+m]*n≡n+m*n ↦ suc-*
277
- ```
278
-
279
274
* In ` Data.List.Relation.Unary.All.Properties ` :
280
275
``` agda
281
276
Any¬→¬All ↦ Any¬⇒¬All
@@ -615,6 +610,12 @@ Other minor additions
615
610
∣p∣⊔∣q∣≤∣p∪q∣ : ∣ p ∣ ⊔ ∣ q ∣ ≤ ∣ p ∪ q ∣
616
611
```
617
612
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
+
618
619
* Added new functions to ` Data.List ` :
619
620
``` agda
620
621
derun : B.Decidable R → List A → List A
@@ -671,6 +672,10 @@ Other minor additions
671
672
deduplicate⁻ : Any P (deduplicate Q? xs) → Any P xs
672
673
```
673
674
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
+
674
679
* Added new functions to ` Data.List.Relation.Binary.Permutation.Setoid ` :
675
680
``` agda
676
681
↭-prep : xs ↭ ys → x ∷ xs ↭ x ∷ ys
You can’t perform that action at this time.
0 commit comments