aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-06 17:39:19 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-06 17:39:19 +0000
commit136a5746aa6d3b841db6327deb61802aef518e66 (patch)
tree9b6f9f17921fbecd9d7d1905e2e37aed634f87f3 /toplevel
parent371cc90e75226a2c4b8022860bc4bd09b3e6657a (diff)
Fixing bug #3030.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16567 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/vernacentries.ml4
1 files changed, 3 insertions, 1 deletions
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index d7d6bc8f1..841919a29 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -1625,7 +1625,9 @@ let vernac_focus gln =
if Int.equal n 0 then
Errors.error "Invalid goal number: 0. Goal numbering starts with 1."
else
- Proof.focus focus_command_cond () n p; print_subgoals ()
+ try Proof.focus focus_command_cond () n p; print_subgoals ()
+ with Proofview.IndexOutOfRange ->
+ Errors.error "No such unproven subgoal."
(* Unfocuses one step in the focus stack. *)
let vernac_unfocus () =