File tree Expand file tree Collapse file tree 3 files changed +47
-0
lines changed Expand file tree Collapse file tree 3 files changed +47
-0
lines changed Original file line number Diff line number Diff line change @@ -291,6 +291,12 @@ New modules
291
291
Algebra.Morphism.LatticeMonomorphism
292
292
```
293
293
294
+ * Solvers for rationals
295
+ ```
296
+ Data.Rational.Solver
297
+ Data.Rational.Unnormalised.Solver
298
+ ```
299
+
294
300
* New ternary relation on lists:
295
301
```
296
302
Data.List.Relation.Ternary.Appending
Original file line number Diff line number Diff line change
1
+ ------------------------------------------------------------------------
2
+ -- The Agda standard library
3
+ --
4
+ -- Automatic solvers for equations over rationals
5
+ ------------------------------------------------------------------------
6
+
7
+ {-# OPTIONS --without-K --safe #-}
8
+
9
+ module Data.Rational.Solver where
10
+
11
+ import Algebra.Solver.Ring.Simple as Solver
12
+ import Algebra.Solver.Ring.AlmostCommutativeRing as ACR
13
+ open import Data.Rational.Properties using (_≟_; +-*-commutativeRing)
14
+
15
+ ------------------------------------------------------------------------
16
+ -- A module for automatically solving propositional equivalences
17
+ -- containing _+_ and _*_
18
+
19
+ module +-*-Solver =
20
+ Solver (ACR.fromCommutativeRing +-*-commutativeRing) _≟_
Original file line number Diff line number Diff line change
1
+ ------------------------------------------------------------------------
2
+ -- The Agda standard library
3
+ --
4
+ -- Automatic solvers for equations over rationals
5
+ ------------------------------------------------------------------------
6
+
7
+ {-# OPTIONS --without-K --safe #-}
8
+
9
+ module Data.Rational.Unnormalised.Solver where
10
+
11
+ import Algebra.Solver.Ring.Simple as Solver
12
+ import Algebra.Solver.Ring.AlmostCommutativeRing as ACR
13
+ open import Data.Rational.Unnormalised.Properties using (_≃?_; +-*-commutativeRing)
14
+
15
+ ------------------------------------------------------------------------
16
+ -- A module for automatically solving propositional equivalences
17
+ -- containing _+_ and _*_
18
+
19
+ module +-*-Solver =
20
+ Solver (ACR.fromCommutativeRing +-*-commutativeRing) _≃?_
21
+
You can’t perform that action at this time.
0 commit comments