aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/goal_selector.v
diff options
context:
space:
mode:
authorGravatar Cyprien Mangin <cyprien.mangin@m4x.org>2016-06-30 19:41:53 +0200
committerGravatar Cyprien Mangin <cyprien.mangin@m4x.org>2016-06-30 19:52:12 +0200
commitfd47b2d2638518fe62ce9c63557d2dab219d9558 (patch)
tree5e2d89f69ec5a3a27ee1bb346ce0cfed69a95807 /test-suite/success/goal_selector.v
parent9501ddd635adea7db07b4df60b8bda1d557dff18 (diff)
Goal selectors now use the keyword [only].
This fixes some parsing problems when doing things like [let n := 2 in idtac n]. See bug #4877.
Diffstat (limited to 'test-suite/success/goal_selector.v')
-rw-r--r--test-suite/success/goal_selector.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/test-suite/success/goal_selector.v b/test-suite/success/goal_selector.v
index 91fb54d9a..868140517 100644
--- a/test-suite/success/goal_selector.v
+++ b/test-suite/success/goal_selector.v
@@ -34,7 +34,7 @@ Qed.
Goal True -> True.
Proof.
- intros y; 1-2 : repeat idtac.
+ intros y; only 1-2 : repeat idtac.
1-1:match goal with y : _ |- _ => let x := y in idtac x end.
Fail 1-1:let x := y in idtac x.
1:let x := y in idtac x.
@@ -44,12 +44,12 @@ Qed.
Goal True /\ (True /\ True).
Proof.
dup.
- - split; 2: (split; exact I).
+ - split; only 2: (split; exact I).
exact I.
- - split; 2: split; exact I.
+ - split; only 2: split; exact I.
Qed.
Goal True -> exists (x : Prop), x.
Proof.
- intro H; eexists ?[x]. [x]: exact True. 1: assumption.
+ intro H; eexists ?[x]; only [x]: exact True. 1: assumption.
Qed.