aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorThéo Zimmermann2018-08-17 18:11:47 +0200
committerThéo Zimmermann2018-08-27 20:00:58 +0200
commit7a7e39f8a0279a149c6b7c20f026cb629aa489f7 (patch)
tree3cb4ed6d8957628b5d3d0c02d7d8fecc7ceb72d1
parenta71ac77f94936319e7e47bedecb44c2b75f73d5e (diff)
Update test-suite for focusing on named goals.
-rw-r--r--test-suite/success/BracketsWithGoalSelector.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/success/BracketsWithGoalSelector.v b/test-suite/success/BracketsWithGoalSelector.v
index ed035f5213..2f7425bce6 100644
--- a/test-suite/success/BracketsWithGoalSelector.v
+++ b/test-suite/success/BracketsWithGoalSelector.v
@@ -14,3 +14,12 @@ Proof.
Fail Qed.
}
Qed.
+
+Lemma foo (n: nat) (P : nat -> Prop):
+ P n.
+Proof.
+ intros.
+ refine (nat_ind _ ?[Base] ?[Step] _).
+ [Base]: { admit. }
+ [Step]: { admit. }
+Abort.