Skip to content

Commit 7568753

Browse files
authored
Changes for release of v1.7.3 (#2141)
1 parent b2e6385 commit 7568753

27 files changed

+250
-27
lines changed

CHANGELOG.md

+15-6
Original file line numberDiff line numberDiff line change
@@ -1,9 +1,18 @@
1-
Version 1.7.2
1+
Version 1.7.3
22
=============
33

4-
The library has been tested using Agda 2.6.3.
4+
The library has been tested using Agda 2.6.4.
55

6-
* In accordance with changes to the flags in Agda 2.6.3, all modules that previously used
7-
the `--without-K` flag now use the `--cubical-compatible` flag instead.
8-
9-
* Updated the code using `primFloatToWord64` - the library API has remained unchanged.
6+
* To avoid _large indices_ that are by default no longer allowed in Agda 2.6.4,
7+
universe levels have been increased in the following definitions:
8+
- `Data.Star.Decoration.DecoratedWith`
9+
- `Data.Star.Pointer.Pointer`
10+
- `Reflection.AnnotatedAST.Typeₐ`
11+
- `Reflection.AnnotatedAST.AnnotationFun`
12+
13+
* The following aliases have been added:
14+
- `IO.Primitive.pure` as alias for `IO.Primitive.return`
15+
- modules `Effect.*` as aliases for modules `Category.*`
16+
17+
These allow to address said objects with the new name they will have in v2.0 of the library,
18+
to ease the transition from v1.7.3 to v2.0.

CHANGELOG/v1.7.2.md

+9
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,9 @@
1+
Version 1.7.2
2+
=============
3+
4+
The library has been tested using Agda 2.6.3.
5+
6+
* In accordance with changes to the flags in Agda 2.6.3, all modules that previously used
7+
the `--without-K` flag now use the `--cubical-compatible` flag instead.
8+
9+
* Updated the code using `primFloatToWord64` - the library API has remained unchanged.

CITATION.cff

+8
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,8 @@
1+
cff-version: 1.2.0
2+
message: "If you use this software, please cite it as below."
3+
authors:
4+
- name: "The Agda Community"
5+
title: "Agda Standard Library"
6+
version: 1.7.3
7+
date-released: 2023-10-15
8+
url: "https://github.com/agda/agda-stdlib"

README.agda

+2-2
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@
33
module README where
44

55
------------------------------------------------------------------------
6-
-- The Agda standard library, version 1.7.2
6+
-- The Agda standard library, version 1.7.3
77
--
88
-- Authors: Nils Anders Danielsson, Matthew Daggitt, Guillaume Allais
99
-- with contributions from Andreas Abel, Stevan Andjelkovic,
@@ -18,7 +18,7 @@ module README where
1818
-- Noam Zeilberger and other anonymous contributors.
1919
------------------------------------------------------------------------
2020

21-
-- This version of the library has been tested using Agda 2.6.2.
21+
-- This version of the library has been tested using Agda 2.6.4.
2222

2323
-- The library comes with a .agda-lib file, for use with the library
2424
-- management system.

agda-stdlib-utils.cabal

+9-7
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
11
name: agda-stdlib-utils
2-
version: 1.7.2
2+
version: 1.7.3
33
cabal-version: >= 1.10
44
build-type: Simple
55
description: Helper programs.
@@ -11,24 +11,26 @@ tested-with: GHC == 8.0.2
1111
GHC == 8.8.4
1212
GHC == 8.10.7
1313
GHC == 9.0.2
14-
GHC == 9.2.1
15-
GHC == 9.4.4
14+
GHC == 9.2.8
15+
GHC == 9.4.7
16+
GHC == 9.6.3
17+
GHC == 9.8.1
1618

1719
executable GenerateEverything
1820
hs-source-dirs: .
1921
main-is: GenerateEverything.hs
2022
default-language: Haskell2010
2123
default-extensions: PatternGuards, PatternSynonyms
22-
build-depends: base >= 4.9.0.0 && < 4.18
24+
build-depends: base >= 4.9.0.0 && < 4.20
2325
, directory >= 1.0.0.0 && < 1.4
2426
, filemanip >= 0.3.6.2 && < 0.4
2527
, filepath >= 1.4.1.0 && < 1.5
26-
, mtl >= 2.2.2 && < 2.3
28+
, mtl >= 2.2.2 && < 2.4
2729

2830
executable AllNonAsciiChars
2931
hs-source-dirs: .
3032
main-is: AllNonAsciiChars.hs
3133
default-language: Haskell2010
32-
build-depends: base >= 4.9.0.0 && < 4.18
34+
build-depends: base >= 4.9.0.0 && < 4.20
3335
, filemanip >= 0.3.6.2 && < 0.4
34-
, text >= 1.2.3.0 && < 2.1
36+
, text >= 1.2.3.0 && < 2.2

notes/installation-guide.md

+6-6
Original file line numberDiff line numberDiff line change
@@ -1,19 +1,19 @@
11
Installation instructions
22
=========================
33

4-
Use version v1.7.2 of the standard library with Agda 2.6.2.
4+
Use version v1.7.3 of the standard library with Agda 2.6.4.
55

66
1. Navigate to a suitable directory `$HERE` (replace appropriately) where
77
you would like to install the library.
88

9-
2. Download the tarball of v1.7.2 of the standard library. This can either be
9+
2. Download the tarball of v1.7.3 of the standard library. This can either be
1010
done manually by visiting the Github repository for the library, or via the
1111
command line as follows:
1212
```
13-
wget -O agda-stdlib.tar https://github.com/agda/agda-stdlib/archive/v1.7.2.tar.gz
13+
wget -O agda-stdlib.tar https://github.com/agda/agda-stdlib/archive/v1.7.3.tar.gz
1414
```
1515
Note that you can replace `wget` with other popular tools such as `curl` and that
16-
you can replace `1.7.2` with any other version of the library you desire.
16+
you can replace `1.7.3` with any other version of the library you desire.
1717

1818
3. Extract the standard library from the tarball. Again this can either be
1919
done manually or via the command line as follows:
@@ -24,14 +24,14 @@ Use version v1.7.2 of the standard library with Agda 2.6.2.
2424
4. [ OPTIONAL ] If using [cabal](https://www.haskell.org/cabal/) then run
2525
the commands to install via cabal:
2626
```
27-
cd agda-stdlib-1.7.2
27+
cd agda-stdlib-1.7.3
2828
cabal install
2929
```
3030

3131
5. Register the standard library with Agda's package system by adding
3232
the following line to `$HOME/.agda/libraries`:
3333
```
34-
$HERE/agda-stdlib-1.7.2/standard-library.agda-lib
34+
$HERE/agda-stdlib-1.7.3/standard-library.agda-lib
3535
```
3636

3737
Now, the standard library is ready to be used either:

src/Data/Star/Decoration.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -28,7 +28,7 @@ data NonEmptyEdgePred {ℓ r p : Level} {I : Set ℓ} (T : Rel I r)
2828
-- Decorating an edge with more information.
2929

3030
data DecoratedWith {ℓ r p : Level} {I : Set ℓ} {T : Rel I r} (P : EdgePred p T)
31-
: Rel (NonEmpty (Star T)) p where
31+
: Rel (NonEmpty (Star T)) (ℓ ⊔ r ⊔ p) where
3232
: {i j k} {x : T i j} {xs : Star T j k}
3333
(p : P x) DecoratedWith P (nonEmpty (x ◅ xs)) (nonEmpty xs)
3434

src/Data/Star/Pointer.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ open import Relation.Binary.Construct.Closure.ReflexiveTransitive
2121

2222
data Pointer {r p q} {T : Rel I r}
2323
(P : EdgePred p T) (Q : EdgePred q T)
24-
: Rel (Maybe (NonEmpty (Star T))) (p ⊔ q) where
24+
: Rel (Maybe (NonEmpty (Star T))) (ℓ ⊔ r ⊔ p ⊔ q) where
2525
step : {i j k} {x : T i j} {xs : Star T j k}
2626
(p : P x) Pointer P Q (just (nonEmpty (x ◅ xs)))
2727
(just (nonEmpty xs))

src/Effect/Applicative.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Applicative`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Applicative where
11+
12+
open import Category.Applicative public

src/Effect/Applicative/Indexed.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Applicative.Indexed`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Applicative.Indexed where
11+
12+
open import Category.Applicative.Indexed public

src/Effect/Applicative/Predicate.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Applicative.Predicate`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Applicative.Predicate where
11+
12+
open import Category.Applicative.Predicate public

src/Effect/Comonad.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Comonad`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Comonad where
11+
12+
open import Category.Comonad public

src/Effect/Functor.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Functor`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Functor where
11+
12+
open import Category.Functor public

src/Effect/Functor/Indexed.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Functor.Indexed`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Functor.Indexed where
11+
12+
open import Category.Functor.Indexed public

src/Effect/Functor/Predicate.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Functor.Predicate`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Functor.Predicate where
11+
12+
open import Category.Functor.Predicate public

src/Effect/Monad.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad where
11+
12+
open import Category.Monad public

src/Effect/Monad/Continuation.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.Continuation`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.Continuation where
11+
12+
open import Category.Monad.Continuation public

src/Effect/Monad/Indexed.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.Indexed`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.Indexed where
11+
12+
open import Category.Monad.Indexed public

src/Effect/Monad/Partiality.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.Partiality`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.Partiality where
11+
12+
open import Category.Monad.Partiality public

src/Effect/Monad/Partiality/All.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.Partiality.All`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.Partiality.All where
11+
12+
open import Category.Monad.Partiality.All public
+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.Partiality.Instances`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.Partiality.Instances where
11+
12+
open import Category.Monad.Partiality.Instances public

src/Effect/Monad/Predicate.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.Predicate`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.Predicate where
11+
12+
open import Category.Monad.Predicate public

src/Effect/Monad/Reader.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.Reader`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.Reader where
11+
12+
open import Category.Monad.Reader public

src/Effect/Monad/State.agda

+12
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- This module duplicates `Category.Monad.State`
5+
-- for forward compatibility with v2.0.
6+
------------------------------------------------------------------------
7+
8+
{-# OPTIONS --cubical-compatible --safe #-}
9+
10+
module Effect.Monad.State where
11+
12+
open import Category.Monad.State public

src/IO/Primitive.agda

+3
Original file line numberDiff line numberDiff line change
@@ -27,3 +27,6 @@ postulate
2727
{-# COMPILE GHC _>>=_ = \_ _ _ _ -> (>>=) #-}
2828
{-# COMPILE UHC return = \_ _ x -> UHC.Agda.Builtins.primReturn x #-}
2929
{-# COMPILE UHC _>>=_ = \_ _ _ _ x y -> UHC.Agda.Builtins.primBind x y #-}
30+
31+
-- Forward compatibility with v2.0.
32+
pure = return

src/Reflection/Annotated.agda

+3-3
Original file line numberDiff line numberDiff line change
@@ -35,8 +35,8 @@ Annotation : ∀ ℓ → Set (suc ℓ)
3535
Annotation ℓ = {u} ⟦ u ⟧ Set
3636

3737
-- An annotated type is a family over an Annotation and a reflected term.
38-
Typeₐ : Univ Set (suc )
39-
Typeₐ ℓ u = Annotation ℓ ⟦ u ⟧ Set
38+
Typeₐ : Univ Set (suc (suc ℓ))
39+
Typeₐ ℓ u = Annotation ℓ ⟦ u ⟧ Set (suc ℓ)
4040

4141
private
4242
variable
@@ -168,7 +168,7 @@ mutual
168168

169169
-- An annotation function computes the top-level annotation given a
170170
-- term annotated at all sub-terms.
171-
AnnotationFun : Annotation ℓ Set
171+
AnnotationFun : Annotation ℓ Set (suc ℓ)
172172
AnnotationFun Ann = u {t : ⟦ u ⟧} Annotated′ Ann t Ann t
173173

174174

0 commit comments

Comments
 (0)