aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-14 15:24:56 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-14 15:24:56 +0000
commite4dd5d40cf0da9b0b692274508da244ba4288f5a (patch)
treee5300f3a48e33cf0434cb8150ceeca2a82065f93
parentf7521f22b4b3542ada80c7b5f8c29bc5ff4d69c8 (diff)
Amélioration message d'erreur
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1106 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--toplevel/vernacentries.ml4
1 files changed, 3 insertions, 1 deletions
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index fd58ae3ed..c19491772 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -1583,10 +1583,12 @@ let _ =
| _ -> invalid_arg "SOLVE"
in
(fun () ->
+ if not (refining ()) then
+ error "Unknown command of the non proof-editing mode";
solve_nth n (Tacinterp.interp tcom);
print_subgoals();
(* in case a strict subtree was completed,
- go back to the top of the prooftree *)
+ go back to the top of the prooftree *)
if subtree_solved () then
(reset_top_of_tree (); print_subgoals())
))