aboutsummaryrefslogtreecommitdiffhomepage
path: root/stm/lemmas.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/lemmas.ml
parente58beb05c80140fbc5f1d0646ece48675370fdc7 (diff)
Vi2vo: fix handling of univ constraints coming from the body
Diffstat (limited to 'stm/lemmas.ml')
-rw-r--r--stm/lemmas.ml3
1 files changed, 2 insertions, 1 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 *)