aboutsummaryrefslogtreecommitdiffhomepage
path: root/stm/stm.ml
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-12-23 17:26:38 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-12-23 17:26:42 +0100
commitb5f0c9f7cd409ab42f034309eedb7eb0247e05cf (patch)
treece2a5e4db982f4522788cb6e3e36900ac5da0990 /stm/stm.ml
parente58beb05c80140fbc5f1d0646ece48675370fdc7 (diff)
Vi2vo: fix handling of univ constraints coming from the body
Diffstat (limited to 'stm/stm.ml')
-rw-r--r--stm/stm.ml4
1 files changed, 3 insertions, 1 deletions
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;