aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-10-06 08:46:53 +0200
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-10-06 08:47:01 +0200
commit6adbf7d9678257aa42ef0d3b30db2e484cd148ad (patch)
treed4b30bbc451049a90cc6dd201f49c3ead984c317 /plugins
parent866d2b75a2d213443e8498b4585326a955ed1558 (diff)
decl_mode: stay in declarative mode
This solution is a bit dumb, but I guess does what one expects. Each decl mode proof commands stays in proof mode.
Diffstat (limited to 'plugins')
-rw-r--r--plugins/decl_mode/decl_proof_instr.ml1
1 files changed, 1 insertions, 0 deletions
diff --git a/plugins/decl_mode/decl_proof_instr.ml b/plugins/decl_mode/decl_proof_instr.ml
index 41d93fc4f..a21447fbb 100644
--- a/plugins/decl_mode/decl_proof_instr.ml
+++ b/plugins/decl_mode/decl_proof_instr.ml
@@ -1463,6 +1463,7 @@ let do_instr raw_instr pts =
postprocess pts raw_instr.instr;
(* spiwack: this should restore a compatible semantics with
v8.3 where we never stayed focused on 0 goal. *)
+ Proof_global.set_proof_mode "Declarative" ;
Decl_mode.maximal_unfocus ()
let proof_instr raw_instr =