@@ -258,8 +258,8 @@ automated warnings will be attached to these modules to discourage their use.
258
258
modules to find in the library. Therefore the module ` Induction.Nat ` has been
259
259
split into two new modules: ` Data.Nat.Induction ` and ` Data.Fin.Induction ` .
260
260
This should improve findability and better matches the design of the rest of
261
- the library. The new modules also re-export ` Acc ` and ` acc ` meaning that users no
262
- longer need to import ` Data.Induction.WellFounded ` as well.
261
+ the library. The new modules also publicly re-export ` Acc ` and ` acc ` , meaning
262
+ that users no longer need to import ` Data.Induction.WellFounded ` as well.
263
263
264
264
* The module ` Record ` has been moved to ` Data.Record ` .
265
265
@@ -348,7 +348,7 @@ attached to all deprecated names to discourage their use.
348
348
map-repeat-commute ↦ map-repeat
349
349
```
350
350
351
- * In ` Data.Bool ` (new names in ` Data.Bool.Properties ` ):
351
+ * In ` Data.Bool ` (with the new name in ` Data.Bool.Properties ` ):
352
352
``` agda
353
353
decSetoid ↦ ≡-decSetoid
354
354
```
@@ -405,7 +405,7 @@ attached to all deprecated names to discourage their use.
405
405
Note that in the case of the last three proofs, the order of the
406
406
arguments will need to be swapped.
407
407
408
- * In ` Data.Unit ` (new names in ` Data.Unit.Properties ` ):
408
+ * In ` Data.Unit ` (with the new names in ` Data.Unit.Properties ` ):
409
409
``` agda
410
410
setoid ↦ ≡-setoid
411
411
decSetoid ↦ ≡-decSetoid
@@ -427,19 +427,18 @@ attached to all deprecated names to discourage their use.
427
427
returnTC ↦ return
428
428
```
429
429
430
- * Renamed functions in ` Data.Char.Base ` and the corresponding property
431
- in ` Data.Char.Properties ` :
430
+ * Renamed functions in ` Data.Char.Base ` :
432
431
``` agda
433
432
fromNat ↦ fromℕ
434
433
toNat ↦ toℕ
435
- toNat-injective ↦ toℕ-injective
436
434
```
437
435
438
436
* In ` Data.(Char/String).Properties ` :
439
437
``` agda
440
438
setoid ↦ ≡-setoid
441
439
decSetoid ↦ ≡-decSetoid
442
440
strictTotalOrder ↦ <-strictTotalOrder-≈
441
+ toNat-injective ↦ toℕ-injective
443
442
```
444
443
445
444
* In ` Data.Vec.Properties ` :
@@ -448,30 +447,31 @@ attached to all deprecated names to discourage their use.
448
447
lookup-++-+′ ↦ lookup-++ʳ
449
448
```
450
449
451
- * In ` Data.Product.Relation.Binary.Pointwise.NonDependent ` :
450
+ * In ` Data.Product.Relation.Binary.Pointwise.NonDependent ` (with the
451
+ new name in ` Data.Product.Properties ` ).:
452
452
``` agda
453
- ≡?×≡?⇒≡? ↦ Data.Product.Properties. ≡-dec
453
+ ≡?×≡?⇒≡? ↦ ≡-dec
454
454
```
455
455
456
456
Other minor additions
457
457
---------------------
458
458
459
459
* Added new proofs in Data.Fin.Substitution.Lemmas:
460
460
``` agda
461
- weaken-↑ : weaken t / (ρ ↑) ≡ weaken (t / ρ)
462
- wk-⊙-∷ : wk ⊙ (t ∷ ρ) ≡ ρ
461
+ weaken-↑ : weaken t / (ρ ↑) ≡ weaken (t / ρ)
463
462
weaken-∷ : weaken t₁ / (t₂ ∷ ρ) ≡ t₁ / ρ
464
- weaken-sub : weaken t₁ / sub t₂ ≡ t₁
463
+ weaken-sub : weaken t₁ / sub t₂ ≡ t₁
464
+ wk-⊙-∷ : wk ⊙ (t ∷ ρ) ≡ ρ
465
465
```
466
466
467
467
* Added new record to ` Algebra ` :
468
468
``` agda
469
- record SelectiveMagma c ℓ : Set (suc (c ⊔ ℓ))
469
+ SelectiveMagma c ℓ : Set (suc (c ⊔ ℓ))
470
470
```
471
471
472
472
* Added new record to ` Algebra.Structure ` :
473
473
``` agda
474
- record IsSelectiveMagma (∙ : Op₂ A) : Set (a ⊔ ℓ)
474
+ IsSelectiveMagma (∙ : Op₂ A) : Set (a ⊔ ℓ)
475
475
```
476
476
477
477
* Added new proof to ` Algebra.Properties.AbelianGroup ` :
@@ -520,25 +520,25 @@ Other minor additions
520
520
521
521
* Added new proofs to ` Data.Bool.Properties ` :
522
522
``` agda
523
- ≡-setoid : Setoid 0ℓ 0ℓ
524
-
525
- ≤-reflexive : _≡_ ⇒ _≤_
526
- ≤-refl : Reflexive _≤_
527
- ≤-antisym : Antisymmetric _≡_ _≤_
528
- ≤-trans : Transitive _≤_
529
- ≤-total : Total _≤_
530
- _≤?_ : Decidable _≤_
531
- ≤-minimum : Minimum _≤_ false
532
- ≤-maximum : Maximum _≤_ true
533
- ≤-irrelevant : B.Irrelevant _≤_
534
- ≤-isPreorder : IsPreorder _≡_ _≤_
535
- ≤-isPartialOrder : IsPartialOrder _≡_ _≤_
536
- ≤-isTotalOrder : IsTotalOrder _≡_ _≤_
537
- ≤-isDecTotalOrder : IsDecTotalOrder _≡_ _≤_
538
- ≤-poset : Poset 0ℓ 0ℓ 0ℓ
539
- ≤-preorder : Preorder 0ℓ 0ℓ 0ℓ
540
- ≤-totalOrder : TotalOrder 0ℓ 0ℓ 0ℓ
541
- ≤-decTotalOrder : DecTotalOrder 0ℓ 0ℓ 0ℓ
523
+ ≡-setoid : Setoid 0ℓ 0ℓ
524
+
525
+ ≤-reflexive : _≡_ ⇒ _≤_
526
+ ≤-refl : Reflexive _≤_
527
+ ≤-antisym : Antisymmetric _≡_ _≤_
528
+ ≤-trans : Transitive _≤_
529
+ ≤-total : Total _≤_
530
+ _≤?_ : Decidable _≤_
531
+ ≤-minimum : Minimum _≤_ false
532
+ ≤-maximum : Maximum _≤_ true
533
+ ≤-irrelevant : B.Irrelevant _≤_
534
+ ≤-isPreorder : IsPreorder _≡_ _≤_
535
+ ≤-isPartialOrder : IsPartialOrder _≡_ _≤_
536
+ ≤-isTotalOrder : IsTotalOrder _≡_ _≤_
537
+ ≤-isDecTotalOrder : IsDecTotalOrder _≡_ _≤_
538
+ ≤-poset : Poset 0ℓ 0ℓ 0ℓ
539
+ ≤-preorder : Preorder 0ℓ 0ℓ 0ℓ
540
+ ≤-totalOrder : TotalOrder 0ℓ 0ℓ 0ℓ
541
+ ≤-decTotalOrder : DecTotalOrder 0ℓ 0ℓ 0ℓ
542
542
543
543
<-irrefl : Irreflexive _≡_ _<_
544
544
<-asym : Asymmetric _<_
@@ -550,9 +550,9 @@ Other minor additions
550
550
<-resp₂-≡ : _<_ Respects₂ _≡_
551
551
<-irrelevant : B.Irrelevant _<_
552
552
<-isStrictPartialOrder : IsStrictPartialOrder _≡_ _<_
553
- <-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
553
+ <-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
554
554
<-strictPartialOrder : StrictPartialOrder 0ℓ 0ℓ 0ℓ
555
- <-strictTotalOrder : StrictTotalOrder 0ℓ 0ℓ 0ℓ
555
+ <-strictTotalOrder : StrictTotalOrder 0ℓ 0ℓ 0ℓ
556
556
```
557
557
558
558
* Added new definitions to ` Data.Char.Base ` :
@@ -610,26 +610,26 @@ Other minor additions
610
610
611
611
* Added new proofs to ` Data.Integer.Properties ` :
612
612
``` agda
613
- ≡-setoid : Setoid 0ℓ 0ℓ
614
- ≤-totalOrder : TotalOrder 0ℓ 0ℓ 0ℓ
615
- _<?_ : Decidable _<_
613
+ ≡-setoid : Setoid 0ℓ 0ℓ
614
+ ≤-totalOrder : TotalOrder 0ℓ 0ℓ 0ℓ
615
+ _<?_ : Decidable _<_
616
616
617
- +[1+-injective : +[1+ m ] ≡ +[1+ n ] → m ≡ n
618
- drop‿+<+ : + m < + n → m ℕ.< n
619
- drop‿-<- : -[1+ m ] < -[1+ n ] → n ℕ.< m
617
+ +[1+-injective : +[1+ m ] ≡ +[1+ n ] → m ≡ n
618
+ drop‿+<+ : + m < + n → m ℕ.< n
619
+ drop‿-<- : -[1+ m ] < -[1+ n ] → n ℕ.< m
620
620
621
- -◃<+◃ : 0 < m → Sign.- ◃ m < Sign.+ ◃ n
622
- +◃≮- : Sign.+ ◃ m ≮ -[1+ n ]
623
- +◃-mono-< : m ℕ.< n → Sign.+ ◃ m < Sign.+ ◃ n
624
- +◃-cancel-< : Sign.+ ◃ m < Sign.+ ◃ n → m ℕ.< n
625
- neg◃-cancel-< : Sign.- ◃ m < Sign.- ◃ n → n ℕ.< m
621
+ -◃<+◃ : 0 < m → Sign.- ◃ m < Sign.+ ◃ n
622
+ +◃≮- : Sign.+ ◃ m ≮ -[1+ n ]
623
+ +◃-mono-< : m ℕ.< n → Sign.+ ◃ m < Sign.+ ◃ n
624
+ +◃-cancel-< : Sign.+ ◃ m < Sign.+ ◃ n → m ℕ.< n
625
+ neg◃-cancel-< : Sign.- ◃ m < Sign.- ◃ n → n ℕ.< m
626
626
627
- m⊖n≤m : m ⊖ n ≤ + m
628
- m⊖n<1+m : m ⊖ n < +[1+ m ]
629
- m⊖1+n<m : m ⊖ suc n < + m
630
- -[1+m]≤n⊖m+1 : -[1+ m ] ≤ n ⊖ suc m
631
- ⊖-monoʳ->-< : (p ⊖_) Preserves ℕ._>_ ⟶ _<_
632
- ⊖-monoˡ-< : (_⊖ p) Preserves ℕ._<_ ⟶ _<_
627
+ m⊖n≤m : m ⊖ n ≤ + m
628
+ m⊖n<1+m : m ⊖ n < +[1+ m ]
629
+ m⊖1+n<m : m ⊖ suc n < + m
630
+ -[1+m]≤n⊖m+1 : -[1+ m ] ≤ n ⊖ suc m
631
+ ⊖-monoʳ->-< : (p ⊖_) Preserves ℕ._>_ ⟶ _<_
632
+ ⊖-monoˡ-< : (_⊖ p) Preserves ℕ._<_ ⟶ _<_
633
633
634
634
*-distrib-+ : _*_ DistributesOver _+_
635
635
*-monoˡ-<-pos : (+[1+ n ] *_) Preserves _<_ ⟶ _<_
@@ -732,22 +732,22 @@ Other minor additions
732
732
m<[1+n%d]⇒m≤[n%d] : m < suc n % d → m ≤ n % d
733
733
[1+m%d]≤1+n⇒[m%d]≤n : 0 < suc m % d → suc m % d ≤ suc n → m % d ≤ n
734
734
735
- 0/n≡0 : 0 / n ≡ 0
736
- n/1≡n : n / 1 ≡ n
737
- n/n≡1 : n / n ≡ 1
738
- m*n/n≡m : m * n / n ≡ m
739
- m/n*n≡m : n ∣ m → m / n * n ≡ m
740
- m*[n/m]≡n : m ∣ n → m * (n / m) ≡ n
741
- m/n*n≤m : m / n * n ≤ m
742
- m/n<m : m ≥ 1 → n ≥ 2 → m / n < m
743
- *-/-assoc : d ∣ n → (m * n) / d ≡ m * (n / d)
744
- +-distrib-/ : m % d + n % d < d → (m + n) / d ≡ m / d + n / d
745
- +-distrib-/-∣ˡ : d ∣ m → (m + n) / d ≡ m / d + n / d
746
- +-distrib-/-∣ʳ : d ∣ n → (m + n) / d ≡ m / d + n / d
735
+ 0/n≡0 : 0 / n ≡ 0
736
+ n/1≡n : n / 1 ≡ n
737
+ n/n≡1 : n / n ≡ 1
738
+ m*n/n≡m : m * n / n ≡ m
739
+ m/n*n≡m : n ∣ m → m / n * n ≡ m
740
+ m*[n/m]≡n : m ∣ n → m * (n / m) ≡ n
741
+ m/n*n≤m : m / n * n ≤ m
742
+ m/n<m : m ≥ 1 → n ≥ 2 → m / n < m
743
+ *-/-assoc : d ∣ n → (m * n) / d ≡ m * (n / d)
744
+ +-distrib-/ : m % d + n % d < d → (m + n) / d ≡ m / d + n / d
745
+ +-distrib-/-∣ˡ : d ∣ m → (m + n) / d ≡ m / d + n / d
746
+ +-distrib-/-∣ʳ : d ∣ n → (m + n) / d ≡ m / d + n / d
747
747
```
748
748
Additionally the ` {≢0 : False (divisor ℕ.≟ 0)} ` argument to all the
749
- division and modulus functions has been marked irrelevant. This means
750
- that the operations ` _%_ ` , ` _/_ ` etc. can now be used with ` cong ` .
749
+ division and modulus functions has been marked irrelevant. One useful consequence
750
+ of this is that the operations ` _%_ ` , ` _/_ ` etc. can now be used with ` cong ` .
751
751
752
752
* Added new proofs to ` Data.Nat.GCD ` :
753
753
``` agda
@@ -995,8 +995,7 @@ Other minor additions
995
995
dec⟶recomputable : Decidable R → Recomputable R
996
996
```
997
997
998
- * Added new alias definitions for ` Algebra.IdempotentCommutativeMonoid `
999
- and ` Algebra.Structures.IsIdempotentCommutativeMonoid ` :
998
+ * Added new aliases for ` IdempotentCommutativeMonoid ` in ` Algebra ` :
1000
999
``` agda
1001
1000
BoundedLattice = IdempotentCommutativeMonoid
1002
1001
IsBoundedLattice = IsIdempotentCommutativeMonoid
0 commit comments