aboutsummaryrefslogtreecommitdiff
path: root/theories/Structures
diff options
context:
space:
mode:
authorVincent Laporte2019-10-28 15:15:11 +0000
committerVincent Laporte2019-10-31 14:10:58 +0000
commitc0fd4618ac7d35de8658fdcf626cdf26c0cca415 (patch)
tree1f358788147421aa4e13b7cbe99687bbd0e5386d /theories/Structures
parentfcebe5a64bb253862e52503b7d4dd6c4c1aebcdf (diff)
lia: depend only on ZArith_base
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/OrderedTypeEx.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Structures/OrderedTypeEx.v b/theories/Structures/OrderedTypeEx.v
index cc216b21f8..e889150d92 100644
--- a/theories/Structures/OrderedTypeEx.v
+++ b/theories/Structures/OrderedTypeEx.v
@@ -9,7 +9,7 @@
(************************************************************************)
Require Import OrderedType.
-Require Import ZArith.
+Require Import ZArith_base.
Require Import PeanoNat.
Require Import Ascii String.
Require Import NArith Ndec.