Skip to content
Merged
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension


Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
4 changes: 2 additions & 2 deletions .github/workflows/ci-ubuntu.yml
Original file line number Diff line number Diff line change
Expand Up @@ -76,11 +76,11 @@ jobs:
if [[ '${{ github.ref }}' == 'refs/heads/experimental' \
|| '${{ github.base_ref }}' == 'experimental' ]]; then
# Pick Agda version for experimental
echo "AGDA_COMMIT=18cc53941e924b144c0f1f3953280ef726009f7e" >> "${GITHUB_ENV}";
echo "AGDA_COMMIT=ef912c68fd329ad3046d156e3c1a70a7fec19ba1" >> "${GITHUB_ENV}";
echo "AGDA_HTML_DIR=html/experimental" >> "${GITHUB_ENV}"
else
# Pick Agda version for master
echo "AGDA_COMMIT=tags/v2.7.0.1" >> "${GITHUB_ENV}";
echo "AGDA_COMMIT=tags/v2.8.0-rc3" >> "${GITHUB_ENV}";
echo "AGDA_HTML_DIR=html/master" >> "${GITHUB_ENV}"
fi

Expand Down
2 changes: 1 addition & 1 deletion CHANGELOG/v1.3.md
Original file line number Diff line number Diff line change
Expand Up @@ -226,7 +226,7 @@ Deprecated modules

* A warning is now raised whenever you import a deprecated module. This should
aid the transition to the new modules. These warnings can be disabled locally
by adding the pragma `{-# OPTIONS --warn=noUserWarning #-}` to the top of a module.
by adding the pragma `{-# OPTIONS --warning=noUserWarning #-}` to the top of a module.

The following modules have been renamed as part of a drive to improve
consistency across the library. The deprecated modules still exist and
Expand Down
2 changes: 2 additions & 0 deletions README.md
Original file line number Diff line number Diff line change
Expand Up @@ -2,6 +2,8 @@

[![Ubuntu build](https://github.com/agda/agda-stdlib/actions/workflows/ci-ubuntu.yml/badge.svg?branch=experimental)](https://github.com/agda/agda-stdlib/actions/workflows/ci-ubuntu.yml)

**Note**: The library is currently tracking Agda 2.8.0 release candidate 3 in preparation for the release of Agda 2.8.0 and version 2.3 of the library. You will need to have the release candidate installed in order to type-check it.

The Agda standard library
=========================

Expand Down
4 changes: 2 additions & 2 deletions src/Algebra/Construct/Initial.agda
Original file line number Diff line number Diff line change
Expand Up @@ -75,10 +75,10 @@ rawMagma = record { ℤero }
-- Structures

isEquivalence : IsEquivalence _≈_
isEquivalence = record { ℤero }
isEquivalence = record { refl = refl; sym = sym; trans = λ {k = k} → trans {k = k} }

isMagma : IsMagma _≈_ _∙_
isMagma = record { isEquivalence = isEquivalence ; ∙-cong = ∙-cong }
isMagma = record { isEquivalence = isEquivalence ; ∙-cong = λ {y = y} {u = u} {v = v} → ∙-cong {y = y} {v = v} }

isSemigroup : IsSemigroup _≈_ _∙_
isSemigroup = record { isMagma = isMagma ; assoc = λ () }
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Operations/Semiring.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@

-- Disabled to prevent warnings from deprecated
-- Algebra.Operations.CommutativeMonoid
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

open import Algebra
import Algebra.Operations.CommutativeMonoid as MonoidOperations
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/BooleanAlgebra.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@
{-# OPTIONS --cubical-compatible --safe #-}

-- Disabled to prevent warnings from deprecated names
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

open import Algebra.Lattice.Bundles

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/DistributiveLattice.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@
{-# OPTIONS --cubical-compatible --safe #-}

-- Disabled to prevent warnings from deprecated names
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

open import Algebra.Lattice.Bundles
open import Algebra.Lattice.Structures.Biased
Expand Down
2 changes: 1 addition & 1 deletion src/Data/Fin/Induction.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-} -- for deprecated _≺_ (issue #1726)
{-# OPTIONS --warning=noUserWarning #-} -- for deprecated _≺_ (issue #1726)

module Data.Fin.Induction where

Expand Down
2 changes: 1 addition & 1 deletion src/Data/Fin/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-} -- for deprecated _≺_ and _≻toℕ_ (issue #1726)
{-# OPTIONS --warning=noUserWarning #-} -- for deprecated _≺_ and _≻toℕ_ (issue #1726)

module Data.Fin.Properties where

Expand Down
2 changes: 1 addition & 1 deletion src/Data/List.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@
-- lists.

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-} -- for deprecated scans
{-# OPTIONS --warning=noUserWarning #-} -- for deprecated scans

module Data.List where

Expand Down
2 changes: 1 addition & 1 deletion src/Data/List/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@
-- equalities than _≡_.

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-} -- for deprecated scans
{-# OPTIONS --warning=noUserWarning #-} -- for deprecated scans

module Data.List.Properties where

Expand Down
2 changes: 1 addition & 1 deletion src/Data/List/Solver.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@
{-# OPTIONS --cubical-compatible --safe #-}

-- Disabled to prevent warnings from deprecated monoid solver
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Data.List.Solver where

Expand Down
2 changes: 1 addition & 1 deletion src/Data/Rational/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-} -- for +-rawMonoid, *-rawMonoid (issue #1865, #1844, #1755)
{-# OPTIONS --warning=noUserWarning #-} -- for +-rawMonoid, *-rawMonoid (issue #1865, #1844, #1755)

module Data.Rational.Properties where

Expand Down
2 changes: 1 addition & 1 deletion src/Data/Rational/Unnormalised/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-} -- for +-rawMonoid, *-rawMonoid (issue #1865, #1844, #1755)
{-# OPTIONS --warning=noUserWarning #-} -- for +-rawMonoid, *-rawMonoid (issue #1865, #1844, #1755)

module Data.Rational.Unnormalised.Properties where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/Bijection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.Bijection where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/Equivalence.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.Equivalence where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/HalfAdjointEquivalence.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.HalfAdjointEquivalence where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/Injection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.Injection where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/Inverse.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.Inverse where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/LeftInverse.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.LeftInverse where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/Related.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.Related where

Expand Down
2 changes: 1 addition & 1 deletion src/Function/Surjection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}
{-# OPTIONS --warning=noUserWarning #-}

module Function.Surjection where

Expand Down