aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide/coqOps.ml
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-11 16:37:29 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-12 13:37:13 +0200
commit666dbb093b09c37941cfb856cdf96fda09c3bac9 (patch)
tree1b1620a19279d02a1aefe5231a39b35d3cfb2b56 /ide/coqOps.ml
parenteec197a86c37b0298fd551c0e5de23ac0c276f66 (diff)
Quick fix for avoiding infinitely many respawning and Warning "Coq
died" when coqtop or coqtopide.cmxs are in inconsistent state.
Diffstat (limited to 'ide/coqOps.ml')
-rw-r--r--ide/coqOps.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/ide/coqOps.ml b/ide/coqOps.ml
index b242bd092..e528666a4 100644
--- a/ide/coqOps.ml
+++ b/ide/coqOps.ml
@@ -732,7 +732,8 @@ object(self)
method handle_reset_initial why =
let action () =
- if why = Coq.Unexpected then warning "Coqtop died badly. Resetting.";
+ if why = Coq.Unexpected then warning "Coqtop died badly. Resetting."
+ else
(* clear the stack *)
if Doc.focused document then Doc.unfocus document;
while not (Doc.is_empty document) do