aboutsummaryrefslogtreecommitdiff
path: root/theories/MSets/MSetGenTree.v
diff options
context:
space:
mode:
authorAndrej Dudenhefner2021-03-23 19:20:18 +0100
committerAndrej Dudenhefner2021-03-26 09:15:49 +0100
commitd7ccf45bbb1b73006c5804bcfc18bb3f6f7c90fd (patch)
treec3070d2ba11ba761eaad10ca44a47e167c1c2637 /theories/MSets/MSetGenTree.v
parent71453f1643b55679d44caee30ce5541b5aa47263 (diff)
remove in List.v deprecated/unnecessary dependencies: Le, Gt, Minus, Lt, Setoid
fix unexpectedly broken MSetGenTree.v add changelog entry
Diffstat (limited to 'theories/MSets/MSetGenTree.v')
-rw-r--r--theories/MSets/MSetGenTree.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/MSets/MSetGenTree.v b/theories/MSets/MSetGenTree.v
index 37d20bffad..c1928fef8d 100644
--- a/theories/MSets/MSetGenTree.v
+++ b/theories/MSets/MSetGenTree.v
@@ -30,6 +30,7 @@
*)
Require Import FunInd Orders OrdersFacts MSetInterface PeanoNat.
+Require Arith. (* contains deprecated dependencies *)
Local Open Scope list_scope.
Local Open Scope lazy_bool_scope.