Skip to content

Commit 1798dfc

Browse files
Removed all deprecated elements up to v1.2 (#1715)
1 parent 02f15d8 commit 1798dfc

File tree

123 files changed

+148
-3644
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

123 files changed

+148
-3644
lines changed

CHANGELOG.md

+22-11
Original file line numberDiff line numberDiff line change
@@ -48,7 +48,7 @@ Non-backwards compatible changes
4848

4949
#### Removed deprecated names
5050

51-
* All modules and names that were deprecated prior to v1.0 have been removed.
51+
* All modules and names that were deprecated in v1.2 and before have been removed.
5252

5353
#### Moved `Codata` modules to `Codata.Sized`
5454

@@ -596,6 +596,9 @@ Deprecated names
596596
*-monoˡ-≤-neg ↦ *-monoˡ-≤-nonPos
597597
*-cancelˡ-<-neg ↦ *-cancelˡ-<-nonPos
598598
*-cancelʳ-<-neg ↦ *-cancelʳ-<-nonPos
599+
600+
^-semigroup-morphism ↦ ^-isMagmaHomomorphism
601+
^-monoid-morphism ↦ ^-isMonoidHomomorphism
599602
```
600603

601604
* In `Data.List.Properties`:
@@ -679,13 +682,6 @@ Deprecated names
679682
id-↔ ↦ ↔-id
680683
```
681684

682-
* Factorial, combinations and permutations for ℕ.
683-
```
684-
Data.Nat.Combinatorics
685-
Data.Nat.Combinatorics.Base
686-
Data.Nat.Combinatorics.Spec
687-
```
688-
689685
* In `Function.Construct.Symmetry`:
690686
```
691687
sym-⤖ ↦ ⤖-sym
@@ -701,6 +697,11 @@ Deprecated names
701697
fromForeign ↦ Foreign.Haskell.Coerce.coerce
702698
```
703699

700+
* In `Relation.Binary.Properties.Preorder`:
701+
```
702+
invIsPreorder ↦ converse-isPreorder
703+
invPreorder ↦ converse-preorder
704+
```
704705

705706
New modules
706707
-----------
@@ -748,6 +749,13 @@ New modules
748749
Data.List.Fresh.NonEmpty
749750
```
750751

752+
* Combinations and permutations for ℕ.
753+
```
754+
Data.Nat.Combinatorics
755+
Data.Nat.Combinatorics.Base
756+
Data.Nat.Combinatorics.Spec
757+
```
758+
751759
* Reflection utilities for some specific types:
752760
```
753761
Data.List.Reflection
@@ -1015,8 +1023,11 @@ Other minor changes
10151023
^-*-assoc : (i ^ m) ^ n ≡ i ^ (m ℕ.* n)
10161024
^-distribˡ-+-* : i ^ (m ℕ.+ n) ≡ i ^ m * i ^ n
10171025
1018-
^-semigroup-morphism : IsSemigroupMorphism ℕ.+-semigroup *-semigroup (i ^_)
1019-
^-monoid-morphism : IsMonoidMorphism ℕ.+-0-monoid *-1-monoid (i ^_)
1026+
*-rawMagma : RawMagma 0ℓ 0ℓ
1027+
*-1-rawMonoid : RawMonoid 0ℓ 0ℓ
1028+
1029+
^-isMagmaHomomorphism : IsMagmaHomomorphism ℕ.+-rawMagma *-rawMagma (i ^_)
1030+
^-isMonoidHomomorphism : IsMonoidHomomorphism ℕ.+-0-rawMonoid *-1-rawMonoid (i ^_)
10201031
```
10211032

10221033
* Added new functions in `Data.List`:
@@ -1690,4 +1701,4 @@ This is a full list of proofs that have changed form to use irrelevant instance
16901701
```agda
16911702
iterate : (A → A) → A → ℕ → A
16921703
iterate-is-fold : ∀ (z : A) s m → fold z s m ≡ iterate s z m
1693-
```
1704+
```

GNUmakefile

+3-2
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,7 @@
11
AGDA_EXEC ?= agda
2-
RTS_OPTIONS=+RTS -M4.0G -H3.5G -A128M -RTS
3-
AGDA=$(AGDA_EXEC) $(RTS_OPTIONS)
2+
AGDA_OPTIONS=-Werror
3+
AGDA_RTS_OPTIONS=+RTS -M4.0G -H3.5G -A128M -RTS
4+
AGDA=$(AGDA_EXEC) $(AGDA_OPTIONS) $(AGDA_RTS_OPTIONS)
45

56
# Before running `make test` the `fix-whitespace` program should
67
# be installed:

src/Algebra/Bundles.agda

-14
Original file line numberDiff line numberDiff line change
@@ -1039,17 +1039,3 @@ record Loop c ℓ : Set (suc (c ⊔ ℓ)) where
10391039

10401040
open Quasigroup quasigroup public
10411041
using (_≉_; ∙-rawMagma; \\-rawMagma; //-rawMagma)
1042-
1043-
------------------------------------------------------------------------
1044-
-- DEPRECATED NAMES
1045-
------------------------------------------------------------------------
1046-
-- Please use the new names as continuing support for the old names is
1047-
-- not guaranteed.
1048-
1049-
-- Version 1.0
1050-
1051-
RawSemigroup = RawMagma
1052-
{-# WARNING_ON_USAGE RawSemigroup
1053-
"Warning: RawSemigroup was deprecated in v1.0.
1054-
Please use RawMagma instead."
1055-
#-}

src/Algebra/FunctionProperties.agda

-20
This file was deleted.

src/Algebra/FunctionProperties/Core.agda

-17
This file was deleted.

src/Algebra/Lattice/Properties/BooleanAlgebra.agda

+12-37
Original file line numberDiff line numberDiff line change
@@ -6,9 +6,6 @@
66

77
{-# OPTIONS --without-K --safe #-}
88

9-
-- Disabled to prevent warnings from deprecated names
10-
{-# OPTIONS --warn=noUserWarning #-}
11-
129
open import Algebra.Lattice.Bundles
1310

1411
module Algebra.Lattice.Properties.BooleanAlgebra
@@ -17,7 +14,7 @@ module Algebra.Lattice.Properties.BooleanAlgebra
1714

1815
open BooleanAlgebra B
1916

20-
import Algebra.Properties.DistributiveLattice as DistribLatticeProperties
17+
import Algebra.Lattice.Properties.DistributiveLattice as DistribLatticeProperties
2118
open import Algebra.Core
2219
open import Algebra.Structures _≈_
2320
open import Algebra.Definitions _≈_
@@ -35,7 +32,6 @@ open import Data.Product using (_,_)
3532
-- Export properties from distributive lattices
3633

3734
open DistribLatticeProperties distributiveLattice public
38-
hiding (replace-equality)
3935

4036
------------------------------------------------------------------------
4137
-- The dual construction is also a boolean algebra
@@ -139,7 +135,7 @@ open DistribLatticeProperties distributiveLattice public
139135
; *-cong = ∧-cong
140136
; *-assoc = ∧-assoc
141137
; *-identity = ∧-identity
142-
; distrib = ∧-∨-distrib
138+
; distrib = ∧-distrib-∨
143139
}
144140
; zero = ∧-zero
145141
}
@@ -151,7 +147,7 @@ open DistribLatticeProperties distributiveLattice public
151147
; *-cong = ∨-cong
152148
; *-assoc = ∨-assoc
153149
; *-identity = ∨-identity
154-
; distrib = ∨-∧-distrib
150+
; distrib = ∨-distrib-∧
155151
}
156152
; zero = ∨-zero
157153
}
@@ -190,10 +186,10 @@ private
190186
lemma x y x∧y=⊥ x∨y=⊤ = begin
191187
¬ x ≈˘⟨ ∧-identityʳ _ ⟩
192188
¬ x ∧ ⊤ ≈˘⟨ ∧-congˡ x∨y=⊤ ⟩
193-
¬ x ∧ (x ∨ y) ≈⟨ ∧-∨-distribˡ _ _ _ ⟩
189+
¬ x ∧ (x ∨ y) ≈⟨ ∧-distribˡ-∨ _ _ _ ⟩
194190
¬ x ∧ x ∨ ¬ x ∧ y ≈⟨ ∨-congʳ $ ∧-complementˡ _ ⟩
195191
⊥ ∨ ¬ x ∧ y ≈˘⟨ ∨-congʳ x∧y=⊥ ⟩
196-
x ∧ y ∨ ¬ x ∧ y ≈˘⟨ ∧-∨-distribʳ _ _ _ ⟩
192+
x ∧ y ∨ ¬ x ∧ y ≈˘⟨ ∧-distribʳ-∨ _ _ _ ⟩
197193
(x ∨ ¬ x) ∧ y ≈⟨ ∧-congʳ $ ∨-complementʳ _ ⟩
198194
⊤ ∧ y ≈⟨ ∧-identityˡ _ ⟩
199195
y ∎
@@ -211,7 +207,7 @@ deMorgan₁ : ∀ x y → ¬ (x ∧ y) ≈ ¬ x ∨ ¬ y
211207
deMorgan₁ x y = lemma (x ∧ y) (¬ x ∨ ¬ y) lem₁ lem₂
212208
where
213209
lem₁ = begin
214-
(x ∧ y) ∧ (¬ x ∨ ¬ y) ≈⟨ ∧-∨-distribˡ _ _ _ ⟩
210+
(x ∧ y) ∧ (¬ x ∨ ¬ y) ≈⟨ ∧-distribˡ-∨ _ _ _ ⟩
215211
(x ∧ y) ∧ ¬ x ∨ (x ∧ y) ∧ ¬ y ≈⟨ ∨-congʳ $ ∧-congʳ $ ∧-comm _ _ ⟩
216212
(y ∧ x) ∧ ¬ x ∨ (x ∧ y) ∧ ¬ y ≈⟨ ∧-assoc _ _ _ ⟨ ∨-cong ⟩ ∧-assoc _ _ _ ⟩
217213
y ∧ (x ∧ ¬ x) ∨ x ∧ (y ∧ ¬ y) ≈⟨ (∧-congˡ $ ∧-complementʳ _) ⟨ ∨-cong ⟩
@@ -279,7 +275,7 @@ module XorRing
279275
¬-distribˡ-⊕ : x y ¬ (x ⊕ y) ≈ ¬ x ⊕ y
280276
¬-distribˡ-⊕ x y = begin
281277
¬ (x ⊕ y) ≈⟨ ¬-cong $ ⊕-def _ _ ⟩
282-
¬ ((x ∨ y) ∧ (¬ (x ∧ y))) ≈⟨ ¬-cong (∧-∨-distribʳ _ _ _) ⟩
278+
¬ ((x ∨ y) ∧ (¬ (x ∧ y))) ≈⟨ ¬-cong (∧-distribʳ-∨ _ _ _) ⟩
283279
¬ ((x ∧ ¬ (x ∧ y)) ∨ (y ∧ ¬ (x ∧ y))) ≈⟨ ¬-cong $ ∨-congˡ $ ∧-congˡ $ ¬-cong (∧-comm _ _) ⟩
284280
¬ ((x ∧ ¬ (x ∧ y)) ∨ (y ∧ ¬ (y ∧ x))) ≈⟨ ¬-cong $ lem _ _ ⟨ ∨-cong ⟩ lem _ _ ⟩
285281
¬ ((x ∧ ¬ y) ∨ (y ∧ ¬ x)) ≈⟨ deMorgan₂ _ _ ⟩
@@ -291,7 +287,7 @@ module XorRing
291287
lem : x y x ∧ ¬ (x ∧ y) ≈ x ∧ ¬ y
292288
lem x y = begin
293289
x ∧ ¬ (x ∧ y) ≈⟨ ∧-congˡ $ deMorgan₁ _ _ ⟩
294-
x ∧ (¬ x ∨ ¬ y) ≈⟨ ∧-∨-distribˡ _ _ _ ⟩
290+
x ∧ (¬ x ∨ ¬ y) ≈⟨ ∧-distribˡ-∨ _ _ _ ⟩
295291
(x ∧ ¬ x) ∨ (x ∧ ¬ y) ≈⟨ ∨-congʳ $ ∧-complementʳ _ ⟩
296292
⊥ ∨ (x ∧ ¬ y) ≈⟨ ∨-identityˡ _ ⟩
297293
x ∧ ¬ y ∎
@@ -349,15 +345,15 @@ module XorRing
349345
(¬ y ∨ ¬ z)) ≈⟨ ∨-congʳ lem₃ ⟩
350346
((x ∧ (y ∨ z)) ∧ ¬ x) ∨
351347
((x ∧ (y ∨ z)) ∧
352-
(¬ y ∨ ¬ z)) ≈˘⟨ ∧-∨-distribˡ _ _ _ ⟩
348+
(¬ y ∨ ¬ z)) ≈˘⟨ ∧-distribˡ-∨ _ _ _ ⟩
353349
(x ∧ (y ∨ z)) ∧
354350
(¬ x ∨ (¬ y ∨ ¬ z)) ≈˘⟨ ∧-congˡ $ ∨-congˡ (deMorgan₁ _ _) ⟩
355351
(x ∧ (y ∨ z)) ∧
356352
(¬ x ∨ ¬ (y ∧ z)) ≈˘⟨ ∧-congˡ (deMorgan₁ _ _) ⟩
357353
(x ∧ (y ∨ z)) ∧
358354
¬ (x ∧ (y ∧ z)) ≈⟨ helper refl lem₁ ⟩
359355
(x ∧ (y ∨ z)) ∧
360-
¬ ((x ∧ y) ∧ (x ∧ z)) ≈⟨ ∧-congʳ $ ∧-∨-distribˡ _ _ _ ⟩
356+
¬ ((x ∧ y) ∧ (x ∧ z)) ≈⟨ ∧-congʳ $ ∧-distribˡ-∨ _ _ _ ⟩
361357
((x ∧ y) ∨ (x ∧ z)) ∧
362358
¬ ((x ∧ y) ∧ (x ∧ z)) ≈˘⟨ ⊕-def _ _ ⟩
363359
(x ∧ y) ⊕ (x ∧ z) ∎
@@ -447,7 +443,7 @@ module XorRing
447443

448444
lem₃ = begin
449445
x ∨ ((y ∨ z) ∧ ¬ (y ∧ z)) ≈⟨ ∨-congˡ $ ∧-congˡ $ deMorgan₁ _ _ ⟩
450-
x ∨ ((y ∨ z) ∧ (¬ y ∨ ¬ z)) ≈⟨ ∨-∧-distribˡ _ _ _ ⟩
446+
x ∨ ((y ∨ z) ∧ (¬ y ∨ ¬ z)) ≈⟨ ∨-distribˡ-∧ _ _ _ ⟩
451447
(x ∨ (y ∨ z)) ∧ (x ∨ (¬ y ∨ ¬ z)) ≈˘⟨ ∨-assoc _ _ _ ⟨ ∧-cong ⟩ ∨-assoc _ _ _ ⟩
452448
((x ∨ y) ∨ z) ∧ ((x ∨ ¬ y) ∨ ¬ z) ∎
453449

@@ -466,7 +462,7 @@ module XorRing
466462
lem₄ = begin
467463
¬ (x ∧ ((y ∨ z) ∧ ¬ (y ∧ z))) ≈⟨ deMorgan₁ _ _ ⟩
468464
¬ x ∨ ¬ ((y ∨ z) ∧ ¬ (y ∧ z)) ≈⟨ ∨-congˡ lem₄′ ⟩
469-
¬ x ∨ ((y ∨ ¬ z) ∧ (¬ y ∨ z)) ≈⟨ ∨-∧-distribˡ _ _ _ ⟩
465+
¬ x ∨ ((y ∨ ¬ z) ∧ (¬ y ∨ z)) ≈⟨ ∨-distribˡ-∧ _ _ _ ⟩
470466
(¬ x ∨ (y ∨ ¬ z)) ∧
471467
(¬ x ∨ (¬ y ∨ z)) ≈˘⟨ ∨-assoc _ _ _ ⟨ ∧-cong ⟩ ∨-assoc _ _ _ ⟩
472468
((¬ x ∨ y) ∨ ¬ z) ∧
@@ -536,27 +532,6 @@ module XorRing
536532
{ isCommutativeRing = ⊕-∧-isCommutativeRing
537533
}
538534

539-
⊕-¬-distribˡ = ¬-distribˡ-⊕
540-
{-# WARNING_ON_USAGE ⊕-¬-distribˡ
541-
"Warning: ⊕-¬-distribˡ was deprecated in v1.1.
542-
Please use ¬-distribˡ-⊕ instead."
543-
#-}
544-
⊕-¬-distribʳ = ¬-distribʳ-⊕
545-
{-# WARNING_ON_USAGE ⊕-¬-distribʳ
546-
"Warning: ⊕-¬-distribʳ was deprecated in v1.1.
547-
Please use ¬-distribʳ-⊕ instead."
548-
#-}
549-
isCommutativeRing = ⊕-∧-isCommutativeRing
550-
{-# WARNING_ON_USAGE isCommutativeRing
551-
"Warning: isCommutativeRing was deprecated in v1.1.
552-
Please use ⊕-∧-isCommutativeRing instead."
553-
#-}
554-
commutativeRing = ⊕-∧-commutativeRing
555-
{-# WARNING_ON_USAGE commutativeRing
556-
"Warning: commutativeRing was deprecated in v1.1.
557-
Please use ⊕-∧-commutativeRing instead."
558-
#-}
559-
560535

561536
infixl 6 _⊕_
562537

src/Algebra/Morphism/Structures.agda

+1
Original file line numberDiff line numberDiff line change
@@ -467,6 +467,7 @@ module RingMorphisms (R₁ : RawRing a ℓ₁) (R₂ : RawRing b ℓ₂) where
467467
------------------------------------------------------------------------
468468
-- Morphisms over quasigroup-like structures
469469
------------------------------------------------------------------------
470+
470471
module QuasigroupMorphisms (Q₁ : RawQuasigroup a ℓ₁) (Q₂ : RawQuasigroup b ℓ₂) where
471472

472473
open RawQuasigroup Q₁ renaming (Carrier to A; ∙-rawMagma to ∙-rawMagma₁;

src/Algebra/Operations/CommutativeMonoid.agda

-21
Original file line numberDiff line numberDiff line change
@@ -6,13 +6,9 @@
66

77
{-# OPTIONS --without-K --safe #-}
88

9-
-- Disabled to prevent warnings from deprecated Table
10-
{-# OPTIONS --warn=noUserWarning #-}
11-
129
open import Algebra
1310
open import Data.List.Base as List using (List; []; _∷_; _++_)
1411
open import Data.Fin.Base using (Fin; zero)
15-
open import Data.Table.Base as Table using (Table)
1612
open import Data.Nat.Base as ℕ using (ℕ; zero; suc)
1713
open import Function.Base using (_∘_)
1814
open import Relation.Binary.Core using (_Preserves_⟶_; _Preserves₂_⟶_⟶_)
@@ -40,23 +36,6 @@ open CommutativeMonoid CM
4036

4137
open import Relation.Binary.Reasoning.Setoid setoid
4238

43-
-- Summation over lists/tables
44-
45-
sumₗ : List Carrier Carrier
46-
sumₗ = List.foldr _+_ 0#
47-
48-
sumₜ : {n} Table Carrier n Carrier
49-
sumₜ = Table.foldr _+_ 0#
50-
51-
-- An alternative mathematical-style syntax for sumₜ
52-
53-
infixl 10 sumₜ-syntax
54-
55-
sumₜ-syntax : n (Fin n Carrier) Carrier
56-
sumₜ-syntax _ = sumₜ ∘ Table.tabulate
57-
58-
syntax sumₜ-syntax n (λ i x) = ∑[ i < n ] x
59-
6039
------------------------------------------------------------------------
6140
-- Multiplication
6241

src/Algebra/Properties/BooleanAlgebra.agda

-13
Original file line numberDiff line numberDiff line change
@@ -38,19 +38,6 @@ open import Data.Product using (_,_)
3838
-- Please use the new names as continuing support for the old names is
3939
-- not guaranteed.
4040

41-
-- Version 1.1
42-
43-
¬⊥=⊤ = ⊥≉⊤
44-
{-# WARNING_ON_USAGE ¬⊥=⊤
45-
"Warning: ¬⊥=⊤ was deprecated in v1.1.
46-
Please use ⊥≉⊤ instead."
47-
#-}
48-
¬⊤=⊥ = ⊤≉⊥
49-
{-# WARNING_ON_USAGE ¬⊤=⊥
50-
"Warning: ¬⊤=⊥ was deprecated in v1.1.
51-
Please use ⊤≉⊥ instead."
52-
#-}
53-
5441
-- Version 1.4
5542

5643
replace-equality : {_≈′_ : Rel Carrier b₂}

0 commit comments

Comments
 (0)