Skip to content

Commit d02343d

Browse files
Merge branch 'master' into experimental
2 parents 7374cb6 + 622cfae commit d02343d

File tree

44 files changed

+2016
-723
lines changed

Some content is hidden

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

44 files changed

+2016
-723
lines changed

CHANGELOG.md

Lines changed: 9 additions & 562 deletions
Large diffs are not rendered by default.

CHANGELOG/v1.4.md

Lines changed: 661 additions & 124 deletions
Large diffs are not rendered by default.

README.agda

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11
module README where
22

33
------------------------------------------------------------------------
4-
-- The Agda standard library, version 1.4-dev
4+
-- The Agda standard library, version 1.5-dev
55
--
66
-- Authors: Nils Anders Danielsson, Matthew Daggitt, Guillaume Allais
77
-- with contributions from Andreas Abel, Stevan Andjelkovic,
@@ -16,7 +16,8 @@ module README where
1616
-- Noam Zeilberger and other anonymous contributors.
1717
------------------------------------------------------------------------
1818

19-
-- This version of the library has been tested using Agda 2.6.1.
19+
-- This version of the library has been tested using Agda 2.6.1 and
20+
-- 2.6.1.1.
2021

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

README/Design/Fixity.agda

Lines changed: 34 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,34 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- Documentation describing some of the fixity choices
5+
------------------------------------------------------------------------
6+
7+
{-# OPTIONS --without-K --safe #-}
8+
9+
-- There is no actual code in here, just design note.
10+
11+
module README.Design.Fixity where
12+
13+
14+
-- binary relations of all kinds are infix 4
15+
-- multiplication-like: infixl 7 _*_
16+
-- addition-like infixl 6 _+_
17+
-- negation-like infix 8 ¬_
18+
-- and-like infixr 7 _∧_
19+
-- or-like infixr 6 _∨_
20+
-- post-fix inverse infix 8 _⁻¹
21+
-- bind infixl 1 _>>=_
22+
-- list concat-like infixr 5 _∷_
23+
-- ternary reasoning infix 1 _⊢_≈_
24+
-- composition infixr 9 _∘_
25+
-- application infixr -1 _$_ _$!_
26+
27+
-- Reasoning:
28+
-- QED infix 3 _∎
29+
-- stepping infixr 2 _≡⟨⟩_ step-≡ step-≡˘
30+
-- begin infix 1 begin_
31+
32+
-- type formers:
33+
-- product-like infixr 2 _×_ _-×-_ _-,-_
34+
-- sum-like infixr 1 _⊎_

lib.cabal

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
11
name: lib
2-
version: 1.4-dev
2+
version: 1.5-dev
33
cabal-version: >= 1.10
44
build-type: Simple
55
description: Helper programs.

notes/installation-guide.md

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -1,19 +1,19 @@
11
Installation instructions
22
=========================
33

4-
Use version v1.3 of the standard library with Agda 2.6.1.
4+
Use version v1.4 of the standard library with Agda 2.6.1 and 2.6.1.1.
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.3 of the standard library. This can either be
9+
2. Download the tarball of v1.4 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.3.tar.gz
13+
wget -O agda-stdlib.tar https://github.com/agda/agda-stdlib/archive/v1.4.tar.gz
1414
```
1515
Note that you can replace `wget` with other popular tools such as `curl` and that
16-
you can replace `1.3` with any other version of the library you desire.
16+
you can replace `1.4` 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.3 of the standard library with Agda 2.6.1.
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.3
27+
cd agda-stdlib-1.4
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.3/standard-library.agda-lib
34+
$HERE/agda-stdlib-1.4/standard-library.agda-lib
3535
```
3636

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

notes/release-guide.txt

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -26,6 +26,10 @@ procedure should be followed:
2626
cd agda
2727
make fast-forward-std-lib
2828

29+
* Build the latest version of Agda
30+
31+
make quicker-install-bin
32+
2933
* Run the tests involving the library:
3034

3135
make test

src/Data/Fin/Properties.agda

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -151,13 +151,13 @@ fromℕ-def : ∀ n → fromℕ n ≡ fromℕ< ℕₚ.≤-refl
151151
fromℕ-def zero = refl
152152
fromℕ-def (suc n) = cong suc (fromℕ-def n)
153153

154-
fromℕ<-irrelevant : m n {o} m ≡ n
155-
(m<o : m ℕ.< o)
156-
(n<o : n ℕ.< o)
157-
fromℕ< m<o ≡ fromℕ< n<o
158-
fromℕ<-irrelevant 0 0 r (s≤s z≤n) (s≤s z≤n) = refl
159-
fromℕ<-irrelevant (suc _) (suc _) r (s≤s (s≤s p)) (s≤s (s≤s q))
160-
= cong suc (fromℕ<-irrelevant _ _ (ℕₚ.suc-injective r) (s≤s p) (s≤s q))
154+
fromℕ<-cong : m n {o} m ≡ n
155+
(m<o : m ℕ.< o)
156+
(n<o : n ℕ.< o)
157+
fromℕ< m<o ≡ fromℕ< n<o
158+
fromℕ<-cong 0 0 r (s≤s z≤n) (s≤s z≤n) = refl
159+
fromℕ<-cong (suc _) (suc _) r (s≤s (s≤s p)) (s≤s (s≤s q))
160+
= cong suc (fromℕ<-cong _ _ (ℕₚ.suc-injective r) (s≤s p) (s≤s q))
161161

162162
fromℕ<-injective : m n {o}
163163
(m<o : m ℕ.< o)

src/Data/Graph/Acyclic.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -170,6 +170,8 @@ module _ {ℓ e} {N : Set ℓ} {E : Set e} where
170170
-- Finds the context and remaining graph corresponding to a given node
171171
-- index.
172172

173+
infix 4 _[_]
174+
173175
_[_] : {n} Graph N E n (i : Fin n) Graph N E (suc (n - suc i))
174176
(c & g) [ zero ] = c & g
175177
(c & g) [ suc i ] = g [ i ]

src/Data/Integer/Divisibility/Signed.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -127,6 +127,8 @@ module ∣-Reasoning where
127127
------------------------------------------------------------------------
128128
-- Other properties of _∣_
129129

130+
infix 4 _∣?_
131+
130132
_∣?_ : Decidable _∣_
131133
k ∣? m = DEC.map′ ∣ᵤ⇒∣ ∣⇒∣ᵤ (∣ k ∣ ℕ.∣? ∣ m ∣)
132134

0 commit comments

Comments
 (0)