aboutsummaryrefslogtreecommitdiffhomepage
path: root/stm
diff options
context:
space:
mode:
Diffstat (limited to 'stm')
-rw-r--r--stm/lemmas.ml3
-rw-r--r--stm/stm.ml4
2 files changed, 5 insertions, 2 deletions
diff --git a/stm/lemmas.ml b/stm/lemmas.ml
index 4bc6f4ee6..48ec66ce6 100644
--- a/stm/lemmas.ml
+++ b/stm/lemmas.ml
@@ -462,7 +462,8 @@ let save_proof ?proof = function
| Vernacexpr.Proved (is_opaque,idopt) ->
let (proof_obj,terminator) =
match proof with
- | None -> Proof_global.close_proof (fun x -> x)
+ | None ->
+ Proof_global.close_proof ~keep_body_ucst_sepatate:false (fun x -> x)
| Some proof -> proof
in
(* if the proof is given explicitly, nothing has to be deleted *)
diff --git a/stm/stm.ml b/stm/stm.ml
index 72f7dcbe7..c966d9bb8 100644
--- a/stm/stm.ml
+++ b/stm/stm.ml
@@ -1126,7 +1126,8 @@ end = struct (* {{{ *)
Proof_global.set_terminator
(Lemmas.standard_proof_terminator []
(Lemmas.mk_hook (fun _ _ -> ())));
- let proof = Proof_global.close_proof (fun x -> x) in
+ let proof =
+ Proof_global.close_proof ~keep_body_ucst_sepatate:true (fun x -> x) in
vernac_interp stop ~proof
{ verbose = false; loc;
expr = (VernacEndProof (Proved (true,None))) };
@@ -1705,6 +1706,7 @@ let known_state ?(redefine_qed=false) ~cache id =
let proof =
if keep != VtKeep then None
else Some(Proof_global.close_proof
+ ~keep_body_ucst_sepatate:false
(State.exn_on id ~valid:eop)) in
if proof = None then prerr_endline "NONE!!!!!";
reach view.next;