Skip to content

Commit

Permalink
[ fix #547 ] Add --safe flags to all safe modules (#549)
Browse files Browse the repository at this point in the history
  • Loading branch information
gallais authored and MatthewDaggitt committed Dec 7, 2018
1 parent d7d3831 commit 64c9035
Show file tree
Hide file tree
Showing 392 changed files with 393 additions and 391 deletions.
2 changes: 1 addition & 1 deletion src/Algebra.agda
Expand Up @@ -5,7 +5,7 @@
-- (packed in records together with sets, operations, etc.)
------------------------------------------------------------------------

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

module Algebra where

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/FunctionProperties.agda
Expand Up @@ -4,7 +4,7 @@
-- Properties of functions, such as associativity and commutativity
------------------------------------------------------------------------

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

open import Level
open import Relation.Binary
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/FunctionProperties/Consequences.agda
Expand Up @@ -5,7 +5,7 @@
-- commutativity
------------------------------------------------------------------------

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

open import Relation.Binary using (Rel; Setoid; Substitutive; Symmetric; Total)

Expand Down
Expand Up @@ -5,7 +5,7 @@
-- commutativity (specialised to propositional equality)
------------------------------------------------------------------------

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

module Algebra.FunctionProperties.Consequences.Propositional
{a} {A : Set a} where
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/FunctionProperties/Core.agda
Expand Up @@ -9,7 +9,7 @@
-- Algebra.FunctionProperties is a parameterised module, and some of
-- the parameters are irrelevant for these definitions.

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

module Algebra.FunctionProperties.Core where

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Morphism.agda
Expand Up @@ -4,7 +4,7 @@
-- Morphisms between algebraic structures
------------------------------------------------------------------------

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

module Algebra.Morphism where

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Operations/CommutativeMonoid.agda
Expand Up @@ -5,7 +5,7 @@
-- exponentiation)
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Operations/Semiring.agda
Expand Up @@ -5,7 +5,7 @@
-- exponentiation)
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/AbelianGroup.agda
Expand Up @@ -4,7 +4,7 @@
-- Some derivable properties
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/BooleanAlgebra.agda
Expand Up @@ -4,7 +4,7 @@
-- Some derivable properties
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/BooleanAlgebra/Expression.agda
Expand Up @@ -4,7 +4,7 @@
-- Boolean algebra expressions
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/CommutativeMonoid.agda
Expand Up @@ -4,7 +4,7 @@
-- Some derivable properties
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/DistributiveLattice.agda
Expand Up @@ -4,7 +4,7 @@
-- Some derivable properties
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/Group.agda
Expand Up @@ -4,7 +4,7 @@
-- Some derivable properties
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/Lattice.agda
Expand Up @@ -4,7 +4,7 @@
-- Some derivable properties
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Properties/Ring.agda
Expand Up @@ -4,7 +4,7 @@
-- Some derivable properties
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/CommutativeMonoid.agda
Expand Up @@ -6,7 +6,7 @@
-- Adapted from Algebra.Monoid-solver
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/CommutativeMonoid/Example.agda
Expand Up @@ -4,7 +4,7 @@
-- An example of how Algebra.CommutativeMonoidSolver can be used
------------------------------------------------------------------------

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

module Algebra.Solver.CommutativeMonoid.Example where

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/IdempotentCommutativeMonoid.agda
Expand Up @@ -6,7 +6,7 @@
-- Adapted from Algebra.Monoid-solver
------------------------------------------------------------------------

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

open import Algebra

Expand Down
Expand Up @@ -5,7 +5,7 @@
-- used
------------------------------------------------------------------------

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

module Algebra.Solver.IdempotentCommutativeMonoid.Example where

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/Monoid.agda
Expand Up @@ -4,7 +4,7 @@
-- Solver for monoid equalities
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/Ring.agda
Expand Up @@ -15,7 +15,7 @@
-- more equalities it returns, the more expressions the ring solver can
-- solve.

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

open import Algebra
open import Algebra.Solver.Ring.AlmostCommutativeRing
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/Ring/AlmostCommutativeRing.agda
Expand Up @@ -5,7 +5,7 @@
-- commutative rings), used by the ring solver
------------------------------------------------------------------------

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

module Algebra.Solver.Ring.AlmostCommutativeRing where

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/Ring/Lemmas.agda
Expand Up @@ -6,7 +6,7 @@

-- Note that these proofs use all "almost commutative ring" properties.

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

open import Algebra
open import Algebra.Solver.Ring.AlmostCommutativeRing
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/Ring/NaturalCoefficients.agda
Expand Up @@ -5,7 +5,7 @@
-- coefficient "ring"
------------------------------------------------------------------------

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

open import Algebra
import Algebra.Operations.Semiring as SemiringOps
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/Ring/NaturalCoefficients/Default.agda
Expand Up @@ -9,7 +9,7 @@
-- characteristic 0.
------------------------------------------------------------------------

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

open import Algebra

Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Solver/Ring/Simple.agda
Expand Up @@ -5,7 +5,7 @@
-- decidable equality
------------------------------------------------------------------------

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

open import Algebra.Solver.Ring.AlmostCommutativeRing
open import Relation.Binary
Expand Down
2 changes: 1 addition & 1 deletion src/Algebra/Structures.agda
Expand Up @@ -5,7 +5,7 @@
-- etc.)
------------------------------------------------------------------------

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

open import Relation.Binary using (Rel; Setoid; IsEquivalence)

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Applicative.agda
Expand Up @@ -7,7 +7,7 @@
-- Note that currently the applicative functor laws are not included
-- here.

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

module Category.Applicative where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Applicative/Indexed.agda
Expand Up @@ -7,7 +7,7 @@
-- Note that currently the applicative functor laws are not included
-- here.

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

module Category.Applicative.Indexed where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Applicative/Predicate.agda
Expand Up @@ -7,7 +7,7 @@
-- Note that currently the applicative functor laws are not included
-- here.

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

module Category.Applicative.Predicate where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Comonad.agda
Expand Up @@ -6,7 +6,7 @@

-- Note that currently the monad laws are not included here.

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

module Category.Comonad where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Functor.agda
Expand Up @@ -6,7 +6,7 @@

-- Note that currently the functor laws are not included here.

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

module Category.Functor where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Functor/Predicate.agda
Expand Up @@ -6,7 +6,7 @@

-- Note that currently the functor laws are not included here.

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

module Category.Functor.Predicate where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Monad.agda
Expand Up @@ -6,7 +6,7 @@

-- Note that currently the monad laws are not included here.

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

module Category.Monad where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Monad/Continuation.agda
Expand Up @@ -4,7 +4,7 @@
-- A delimited continuation monad
------------------------------------------------------------------------

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

module Category.Monad.Continuation where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Monad/Indexed.agda
Expand Up @@ -6,7 +6,7 @@

-- Note that currently the monad laws are not included here.

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

module Category.Monad.Indexed where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Monad/Partiality.agda
Expand Up @@ -4,7 +4,7 @@
-- The partiality monad
------------------------------------------------------------------------

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

module Category.Monad.Partiality where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Monad/Partiality/All.agda
Expand Up @@ -4,7 +4,7 @@
-- An All predicate for the partiality monad
------------------------------------------------------------------------

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

module Category.Monad.Partiality.All where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Monad/Predicate.agda
Expand Up @@ -6,7 +6,7 @@

-- Note that currently the monad laws are not included here.

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

module Category.Monad.Predicate where

Expand Down
2 changes: 1 addition & 1 deletion src/Category/Monad/State.agda
Expand Up @@ -4,7 +4,7 @@
-- The state monad
------------------------------------------------------------------------

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

module Category.Monad.State where

Expand Down
2 changes: 1 addition & 1 deletion src/Codata/Cofin.agda
Expand Up @@ -4,7 +4,7 @@
-- "Finite" sets indexed on coinductive "natural" numbers
------------------------------------------------------------------------

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

module Codata.Cofin where

Expand Down
2 changes: 1 addition & 1 deletion src/Codata/Cofin/Literals.agda
Expand Up @@ -4,7 +4,7 @@
-- Conat Literals
------------------------------------------------------------------------

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

module Codata.Cofin.Literals where

Expand Down
2 changes: 1 addition & 1 deletion src/Codata/Colist.agda
Expand Up @@ -4,7 +4,7 @@
-- The Colist type and some operations
------------------------------------------------------------------------

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

module Codata.Colist where

Expand Down

0 comments on commit 64c9035

Please sign in to comment.