aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/pfedit.ml
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-21 13:08:08 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-09-12 10:47:32 +0200
commit8326639ef45b22cb066f65d17f27a77a678eb694 (patch)
tree911e1ea019b7dc3412071743573590053e181f2d /proofs/pfedit.ml
parentd542746c848d4795d4af97874a30fa5e98c8a6b2 (diff)
Add syntax [id]: to apply tactic to goal named id.
Diffstat (limited to 'proofs/pfedit.ml')
-rw-r--r--proofs/pfedit.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml
index 49195aecc..1b0b2f401 100644
--- a/proofs/pfedit.ml
+++ b/proofs/pfedit.ml
@@ -94,6 +94,7 @@ let solve ?with_end_tac gi tac pr =
| Some etac -> Proofview.tclTHEN tac etac in
let tac = match gi with
| Vernacexpr.SelectNth i -> Proofview.tclFOCUS i i tac
+ | Vernacexpr.SelectId id -> Proofview.tclFOCUSID id tac
| Vernacexpr.SelectAll -> tac
| Vernacexpr.SelectAllParallel ->
Errors.anomaly(str"SelectAllParallel not handled by Stm")
@@ -101,7 +102,7 @@ let solve ?with_end_tac gi tac pr =
Proof.run_tactic (Global.env ()) tac pr
with
| Proof_global.NoCurrentProof -> Errors.error "No focused proof"
- | Proofview.IndexOutOfRange ->
+ | Proofview.IndexOutOfRange ->
match gi with
| Vernacexpr.SelectNth i -> let msg = str "No such goal: " ++ int i ++ str "." in
Errors.errorlabstrm "" msg