aboutsummaryrefslogtreecommitdiff
path: root/theories/Structures
diff options
context:
space:
mode:
authorGaëtan Gilbert2021-01-07 13:55:23 +0100
committerGaëtan Gilbert2021-01-18 13:08:17 +0100
commit4419a101a4f5a108be90cf4e420f0b6961e6caac (patch)
treec3a3dcede7a5901685d28da3d540451e39c4b6f1 /theories/Structures
parent58a4f645ee6d306cb824c2ac2dfa21e460b9692a (diff)
Support locality attributes for Hint Rewrite (including export)
We deprecate unspecified locality as was done for Hint. Close #13724
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/OrdersFacts.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Structures/OrdersFacts.v b/theories/Structures/OrdersFacts.v
index 4ac54d280a..c3e67b9d5a 100644
--- a/theories/Structures/OrdersFacts.v
+++ b/theories/Structures/OrdersFacts.v
@@ -53,7 +53,7 @@ Module Type CompareFacts (Import O:DecStrOrder').
rewrite compare_gt_iff; intuition.
Qed.
- Hint Rewrite compare_eq_iff compare_lt_iff compare_gt_iff : order.
+ Global Hint Rewrite compare_eq_iff compare_lt_iff compare_gt_iff : order.
Instance compare_compat : Proper (eq==>eq==>Logic.eq) compare.
Proof.