File tree 3 files changed +6
-9
lines changed
3 files changed +6
-9
lines changed Original file line number Diff line number Diff line change @@ -53,6 +53,10 @@ Non-backwards compatible changes
53
53
So ` [a-zA-Z]+.agdai? ` run on "the path _ build/Main.agdai corresponds to"
54
54
will return "Main.agdai" when it used to be happy to just return "n.agda".
55
55
56
+ * The constructors ` +0 ` and ` +[1+_] ` from ` Data.Integer.Base ` are no longer
57
+ exported by ` Data.Rational.Base ` . You will have to open ` Data.Integer(.Base) `
58
+ directly to use them.
59
+
56
60
Deprecated modules
57
61
------------------
58
62
Original file line number Diff line number Diff line change @@ -10,7 +10,7 @@ module Data.Rational.Base where
10
10
11
11
open import Data.Bool.Base using (Bool; true; false; if_then_else_)
12
12
open import Function.Base using (id)
13
- open import Data.Integer.Base as ℤ using (ℤ; +_; +0; -[1+_])
13
+ open import Data.Integer.Base as ℤ using (ℤ; +_; +0; +[1+_]; -[1+_])
14
14
import Data.Integer.GCD as ℤ
15
15
import Data.Integer.DivMod as ℤ
16
16
open import Data.Nat.GCD
@@ -35,13 +35,6 @@ open import Relation.Binary.PropositionalEquality
35
35
36
36
open ≡-Reasoning
37
37
38
- -- Note, these are re-exported publicly to maintain backwards
39
- -- compatability. Although we are unable (?) to put a warning on them,
40
- -- using these from `Data.Rational` should be viewed as a deprecated
41
- -- feature.
42
-
43
- open import Data.Integer public using (+0; +[1+_])
44
-
45
38
------------------------------------------------------------------------
46
39
-- Rational numbers in reduced form. Note that there is exactly one
47
40
-- way to represent every rational number.
Original file line number Diff line number Diff line change @@ -20,7 +20,7 @@ import Algebra.Morphism.RingMonomorphism as RingMonomorphisms
20
20
import Algebra.Morphism.LatticeMonomorphism as LatticeMonomorphisms
21
21
import Algebra.Properties.CommutativeSemigroup as CommSemigroupProperties
22
22
open import Data.Bool.Base using (T; true; false)
23
- open import Data.Integer.Base as ℤ using (ℤ; +_; -[1+_]; 0ℤ; 1ℤ; _◃_)
23
+ open import Data.Integer.Base as ℤ using (ℤ; +_; -[1+_]; +[1+_]; +0; 0ℤ; 1ℤ; _◃_)
24
24
open import Data.Integer.Coprimality using (coprime-divisor)
25
25
import Data.Integer.Properties as ℤ
26
26
open import Data.Integer.GCD using (gcd; gcd[i,j]≡0⇒i≡0; gcd[i,j]≡0⇒j≡0)
You can’t perform that action at this time.
0 commit comments