aboutsummaryrefslogtreecommitdiff
path: root/kernel/term_typing.ml
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2019-06-19 21:24:36 +0200
committerPierre-Marie Pédrot2019-06-24 11:02:11 +0200
commitbe3bba54e39a316ded975b7c5ac5723fed41aa88 (patch)
tree7f801ebcb9544af86394b1727c8c5733b898506b /kernel/term_typing.ml
parent4ceadecf179e9210eed42ef4847aa5ab8fa28bd6 (diff)
Enforce that transparent entries are forced beforehand.
Diffstat (limited to 'kernel/term_typing.ml')
-rw-r--r--kernel/term_typing.ml12
1 files changed, 4 insertions, 8 deletions
diff --git a/kernel/term_typing.ml b/kernel/term_typing.ml
index e28849c953..3b689953c8 100644
--- a/kernel/term_typing.ml
+++ b/kernel/term_typing.ml
@@ -196,13 +196,9 @@ let infer_declaration (type a) ~(trust : a trust) env (dcl : a constant_entry) =
(** Other definitions have to be processed immediately. *)
| DefinitionEntry c ->
let { const_entry_type = typ; _ } = c in
- let { const_entry_body = body; const_entry_feedback = feedback_id; _ } = c in
- (* Opaque constants must be provided with a non-empty const_entry_type,
- and thus should have been treated above. *)
- let body, ctx = match trust with
- | Pure ->
- let (body, ctx), () = Future.join body in
- body, ctx
+ let { const_entry_body = (body, ctx); const_entry_feedback = feedback_id; _ } = c in
+ let () = match trust with
+ | Pure -> ()
| SideEffects _ -> assert false
in
let env, usubst, univs = match c.const_entry_universes with
@@ -366,7 +362,7 @@ let translate_recipe env _kn r =
let translate_local_def env _id centry =
let open Cooking in
- let body = Future.from_val ((centry.secdef_body, Univ.ContextSet.empty), ()) in
+ let body = (centry.secdef_body, Univ.ContextSet.empty) in
let centry = {
const_entry_body = body;
const_entry_secctx = centry.secdef_secctx;