aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Relations_2.v
diff options
context:
space:
mode:
authorGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2016-10-24 17:28:51 +0200
committerGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2016-10-24 17:28:51 +0200
commit7e38b6627caaab7d19c4fc0ee542a67d9f8970c2 (patch)
tree375ed6a0a45131e479dea6d3d8c9cf64a786fcf7 /theories/Sets/Relations_2.v
parent46462c3cc69e97bf3260f1aad5faaa6eaf6c2722 (diff)
Remove v62 from stdlib.
This old compatibility hint database can be safely removed now that coq-contribs do not depend on it anymore.
Diffstat (limited to 'theories/Sets/Relations_2.v')
-rw-r--r--theories/Sets/Relations_2.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Sets/Relations_2.v b/theories/Sets/Relations_2.v
index f1026e31a..1e0b83fe5 100644
--- a/theories/Sets/Relations_2.v
+++ b/theories/Sets/Relations_2.v
@@ -48,7 +48,7 @@ Definition Strongly_confluent : Prop :=
End Relations_2.
-Hint Resolve Rstar_0: sets v62.
-Hint Resolve Rstar1_0: sets v62.
-Hint Resolve Rstar1_1: sets v62.
-Hint Resolve Rplus_0: sets v62.
+Hint Resolve Rstar_0: sets.
+Hint Resolve Rstar1_0: sets.
+Hint Resolve Rstar1_1: sets.
+Hint Resolve Rplus_0: sets.