File tree Expand file tree Collapse file tree 1 file changed +2
-7
lines changed Expand file tree Collapse file tree 1 file changed +2
-7
lines changed Original file line number Diff line number Diff line change 1
1
------------------------------------------------------------------------
2
2
-- The Agda standard library
3
3
--
4
- -- This module is DEPRECATED. Please use Tactic.MonoidSolver instead
4
+ -- A solver for equations over monoids
5
5
------------------------------------------------------------------------
6
6
7
7
{-# OPTIONS --without-K --safe #-}
@@ -10,12 +10,7 @@ open import Algebra
10
10
11
11
module Algebra.Solver.Monoid {m₁ m₂} (M : Monoid m₁ m₂) where
12
12
13
- {-# WARNING_ON_IMPORT
14
- "Algebra.Solver.Monoid was deprecated in v1.3.
15
- Use Tactic.MonoidSolver instead."
16
- #-}
17
-
18
- open import Data.Fin.Base as Fin hiding (_≟_)
13
+ open import Data.Fin.Base as Fin
19
14
import Data.Fin.Properties as Fin
20
15
open import Data.List.Base hiding (lookup)
21
16
import Data.List.Relation.Binary.Equality.DecPropositional as ListEq
You can’t perform that action at this time.
0 commit comments