aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Cyprien Mangin <cyprien.mangin@m4x.org>2016-06-03 10:43:24 +0200
committerGravatar Cyprien Mangin <cyprien.mangin@m4x.org>2016-06-14 06:21:31 +0200
commit95a7ddee80fef2d499dce36a7e37fc5c6e374018 (patch)
tree990b4931fe0ff1c715c93a7dfddd13f1718956cd /test-suite
parent98ed04803e022e66e17f91526ef708484fd17217 (diff)
Ident selectors cannot be used inside an Ltac expression.
They can still be used at the toplevel.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/success/destruct.v2
-rw-r--r--test-suite/success/goal_selector.v2
2 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/success/destruct.v b/test-suite/success/destruct.v
index fd71f3c42..90a60daa6 100644
--- a/test-suite/success/destruct.v
+++ b/test-suite/success/destruct.v
@@ -106,7 +106,7 @@ Goal exists x, S 0 = S x.
eexists ?[x].
destruct (S _). (* Incompatible occurrences but takes the first one since Oct 2014 *)
change (0 = S ?x).
-?[x]: exact 0. (* Incidentally test applying a tactic to a goal on the shelve *)
+[x]: exact 0. (* Incidentally test applying a tactic to a goal on the shelve *)
Abort.
Goal exists n p:nat, (S n,S n) = (S p,S p) /\ p = n.
diff --git a/test-suite/success/goal_selector.v b/test-suite/success/goal_selector.v
index dd7ad1013..91fb54d9a 100644
--- a/test-suite/success/goal_selector.v
+++ b/test-suite/success/goal_selector.v
@@ -51,5 +51,5 @@ Qed.
Goal True -> exists (x : Prop), x.
Proof.
- intro H; eexists ?[x]; ?[x]: exact True; assumption.
+ intro H; eexists ?[x]. [x]: exact True. 1: assumption.
Qed.