aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/bteauto.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2016-06-09 23:24:57 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2016-06-16 18:21:08 +0200
commit2194292dbe88674fd9a606bb22f28d332f670f77 (patch)
tree21c2e91b13a5de21856554b17f5dfaa61101e253 /test-suite/success/bteauto.v
parentaf7a9a4e44739968b68aeb1cb0a1f70a1aa34e88 (diff)
Revise syntax of Hint Cut
As noticed by C. Cohen it was confusingly different from standard notation.
Diffstat (limited to 'test-suite/success/bteauto.v')
-rw-r--r--test-suite/success/bteauto.v9
1 files changed, 5 insertions, 4 deletions
diff --git a/test-suite/success/bteauto.v b/test-suite/success/bteauto.v
index 34238fe13..4b28da19d 100644
--- a/test-suite/success/bteauto.v
+++ b/test-suite/success/bteauto.v
@@ -50,9 +50,10 @@ End Backtracking.
Hint Resolve 100 eq_sym eq_trans : core.
-Hint Cut [!*; eq_sym; eq_sym] : core.
-Hint Cut [!*; eq_trans; eq_trans] : core.
-Hint Cut [!*; eq_trans; eq_sym; eq_trans] : core.
+Hint Cut [(_)* eq_sym eq_sym] : core.
+Hint Cut [_* eq_trans eq_trans] : core.
+Hint Cut [_* eq_trans eq_sym eq_trans] : core.
+
Goal forall x y z : nat, x = y -> z = y -> x = z.
Proof.
@@ -73,7 +74,7 @@ Module Hierarchies.
Fail Timeout 1 Definition makeA' : A := _.
- Hint Cut [!*; mkB; aofb] : typeclass_instances.
+ Hint Cut [_* mkB aofb] : typeclass_instances.
Fail Definition makeA' : A := _.
Fail Definition makeB' : B := _.
End Hierarchies.