aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/term_typing.ml
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-05-16 00:06:51 +0200
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-05-28 15:28:24 +0200
commit4552729b88058946055dddde1533057e25bfc5a9 (patch)
tree38c4c1440c9aa03430b63da175663f96bcf668dd /kernel/term_typing.ml
parentb053d98fb17d2f46878f49d7adf4839ae632c10b (diff)
Unify pre_env and env
We now have only two notions of environments in the kernel: env and safe_env.
Diffstat (limited to 'kernel/term_typing.ml')
-rw-r--r--kernel/term_typing.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/kernel/term_typing.ml b/kernel/term_typing.ml
index e621a61c7..7352c1882 100644
--- a/kernel/term_typing.ml
+++ b/kernel/term_typing.ml
@@ -460,7 +460,7 @@ let build_constant_declaration kn env result =
let tps =
let res =
match result.cook_proj with
- | None -> compile_constant_body env univs def
+ | None -> Cbytegen.compile_constant_body ~fail_on_error:false env univs def
| Some pb ->
(* The compilation of primitive projections is a bit tricky, because
they refer to themselves (the body of p looks like fun c =>
@@ -480,7 +480,7 @@ let build_constant_declaration kn env result =
}
in
let env = add_constant kn cb env in
- compile_constant_body env univs def
+ Cbytegen.compile_constant_body ~fail_on_error:false env univs def
in Option.map Cemitcodes.from_val res
in
{ const_hyps = hyps;