aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernacentries.ml
diff options
context:
space:
mode:
Diffstat (limited to 'toplevel/vernacentries.ml')
-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 () =