aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Arnaud Spiwack <arnaud@spiwack.net>2015-03-12 17:46:35 +0100
committerGravatar Arnaud Spiwack <arnaud@spiwack.net>2015-03-13 16:41:03 +0100
commitedb3302188af4b5b75111339e3f466a6ec09aef2 (patch)
tree5eeff106590577a84c7c42d1cba35649c2d90776
parent71fcb53fd93edcac1925f97d619871e8597e24e2 (diff)
Declarative mode: make it so that unfocussing can only be done for closed subproofs.
The front-end is supposed to take care of that, but it may help to catch bugs.
-rw-r--r--plugins/decl_mode/decl_mode.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/decl_mode/decl_mode.ml b/plugins/decl_mode/decl_mode.ml
index da41cd86d..07df7c7f0 100644
--- a/plugins/decl_mode/decl_mode.ml
+++ b/plugins/decl_mode/decl_mode.ml
@@ -96,7 +96,7 @@ let get_goal_stack pts =
let proof_focus = Proof.new_focus_kind ()
-let proof_cond = Proof.no_cond proof_focus
+let proof_cond = Proof.done_cond proof_focus
let focus p =
let inf = get_goal_stack p in