@@ -6,6 +6,10 @@ The library has been tested using Agda 2.6.1 and 2.6.1.1.
6
6
Highlights
7
7
----------
8
8
9
+ * Drastically reorganised the module hierarchy in the dependency graph of
10
+ the ` IO ` module so that we may compile a program as simple as hello world
11
+ without pulling upwards of 130 modules.
12
+
9
13
* First verified implementation of a sorting algorithm (available from ` Data.List.Sort ` ).
10
14
11
15
Bug-fixes
@@ -14,6 +18,16 @@ Bug-fixes
14
18
Non-backwards compatible changes
15
19
--------------------------------
16
20
21
+ * ` Data.List.Relation.Binary.Lex.Core ` has been thinned to minimise its
22
+ dependencies. The more complex properties (` transitive ` , ` respects₂ ` ,
23
+ ` []<[]-⇔ ` , ` ∷<∷-⇔ ` , and ` decidable ` ) have been moved to
24
+ ` Data.List.Relation.Binary.Lex ` .
25
+
26
+ * ` Data.String.Base ` has been thinned to minimise its dependencies. The more
27
+ complex functions (` parensIfSpace ` , ` wordsBy ` , ` words ` , ` linesBy ` , ` lines ` ,
28
+ ` rectangle ` , ` rectangleˡ ` , ` rectangleʳ ` , ` rectangleᶜ ` ) have been moved to
29
+ ` Data.String ` .
30
+
17
31
Deprecated modules
18
32
------------------
19
33
@@ -116,6 +130,30 @@ New modules
116
130
Data.Nat.PseudoRandom.LCG
117
131
```
118
132
133
+ * Broke up ` Data.List.Relation.Binary.Pointwise ` and introduced:
134
+ ```
135
+ Data.List.Relation.Binary.Pointwise.Base
136
+ Data.List.Relation.Binary.Pointwise.Properties
137
+ ```
138
+
139
+ * Broke up ` Codata.Musical.Colist ` into a multitude of modules:
140
+ ```
141
+ Codata.Musical.Colist.Base
142
+ Codata.Musical.Colist.Properties
143
+ Codata.Musical.Colist.Bisimilarity
144
+ Codata.Musical.Colist.Relation.Unary.All
145
+ Codata.Musical.Colist.Relation.Unary.All.Properties
146
+ Codata.Musical.Colist.Relation.Unary.Any
147
+ Codata.Musical.Colist.Relation.Unary.Any.Properties
148
+ ```
149
+
150
+ * Broke up ` IO ` into a many smaller modules:
151
+ ```
152
+ IO.Base
153
+ IO.Finite
154
+ IO.Infinite
155
+ ```
156
+
119
157
* Instantiate a homogeneously indexed bundle at a particular index
120
158
```
121
159
Relation.Binary.Indexed.Homogeneous.Construct.At
@@ -130,6 +168,11 @@ New modules
130
168
Other minor additions
131
169
---------------------
132
170
171
+ * Added new function in ` Data.Char.Base ` :
172
+ ``` agda
173
+ _≈ᵇ_ : (c d : Char) → Bool
174
+ ```
175
+
133
176
* Added new proofs in ` Algebra.Morphism.GroupMonomorphism ` :
134
177
``` agda
135
178
⁻¹-distrib-∙ : ((x ◦ y) ⁻¹₂ ≈₂ (x ⁻¹₂) ◦ (y ⁻¹₂)) → ((x ∙ y) ⁻¹₁ ≈₁ (x ⁻¹₁) ∙ (y ⁻¹₁))
@@ -370,7 +413,7 @@ Other minor additions
370
413
371
414
* Added new proofs to ` Data.List.Relation.Binary.Pointwise ` :
372
415
``` agda
373
- foldr⁺ : (R w x → R y z → R (w • y) (x ◦ z)) →
416
+ foldr⁺ : (R w x → R y z → R (w • y) (x ◦ z)) →
374
417
R e f → Pointwise R xs ys → R (foldr _•_ e xs) (foldr _◦_ f ys)
375
418
lookup⁻ : length xs ≡ length ys →
376
419
(toℕ i ≡ toℕ j → R (lookup xs i) (lookup ys j)) →
0 commit comments