aboutsummaryrefslogtreecommitdiffhomepage
path: root/stm/lemmas.ml
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2013-10-11 18:30:54 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-06 09:58:53 +0200
commit57bee17f928fc67a599d2116edb42a59eeb21477 (patch)
treef8e1446f5869de08be1dc20c104d61d0e47ce57d /stm/lemmas.ml
parenta4043608f704f026de7eb5167a109ca48e00c221 (diff)
Rework handling of universes on top of the STM, allowing for delayed
computation in case of non-polymorphic proofs. Also fix plugins after forgotten merge conflicts. Still does not compile everything.
Diffstat (limited to 'stm/lemmas.ml')
-rw-r--r--stm/lemmas.ml13
1 files changed, 2 insertions, 11 deletions
diff --git a/stm/lemmas.ml b/stm/lemmas.ml
index 2aeb8141e..13194eb89 100644
--- a/stm/lemmas.ml
+++ b/stm/lemmas.ml
@@ -229,17 +229,8 @@ let save_remaining_recthms (locality,p,kind) body opaq i (id,((t_i,ctx_i),(_,imp
| _ -> anomaly (Pp.str "Not a proof by induction") in
match locality with
| Discharge ->
- let const = { const_entry_body =
- Future.from_val (body_i,Declareops.no_seff);
- const_entry_secctx = None;
- const_entry_type = Some t_i;
- const_entry_proj = None;
- const_entry_opaque = opaq;
- const_entry_feedback = None;
- const_entry_inline_code = false;
- const_entry_polymorphic = p;
- const_entry_universes = Univ.ContextSet.to_context ctx_i
- } in
+ let const = definition_entry ~types:t_i ~opaque:opaq ~poly:p
+ ~univs:(Univ.ContextSet.to_context ctx_i) body_i in
let c = SectionLocalDef const in
let _ = declare_variable id (Lib.cwd(), c, k) in
(Discharge,VarRef id,imps)