aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/term_typing.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-04-07 01:21:41 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-04-07 01:21:41 +0200
commitd939a024cd077c8abce709dd69eb805cab9068db (patch)
treed962846a251f5ee3a8ce1d92f10793bd9e395f95 /kernel/term_typing.ml
parent78aca729a95d5e622c251d247abf29159dfe66a4 (diff)
Inline the only use of hcons_j in Term_typing.
Diffstat (limited to 'kernel/term_typing.ml')
-rw-r--r--kernel/term_typing.ml8
1 files changed, 2 insertions, 6 deletions
diff --git a/kernel/term_typing.ml b/kernel/term_typing.ml
index e203fce9a..6dfa64357 100644
--- a/kernel/term_typing.ml
+++ b/kernel/term_typing.ml
@@ -191,10 +191,6 @@ let rec unzip ctx j =
| `Cut (n,ty,arg) :: ctx ->
unzip ctx { j with uj_val = mkApp (mkLambda (n,ty,j.uj_val),arg) }
-let hcons_j j =
- (** Do not hashcons type: it is not used by the callers of this function. *)
- { uj_val = hcons_constr j.uj_val; uj_type = j.uj_type}
-
let feedback_completion_typecheck =
let open Feedback in
Option.iter (fun state_id ->
@@ -231,13 +227,13 @@ let infer_declaration ~trust env kn dcl =
let body,env,ectx = skip_trusted_seff valid_signatures body env in
let j = infer env body in
unzip ectx j in
- let j = hcons_j j in
let subst = Univ.LMap.empty in
let _ = judge_of_cast env j DEFAULTcast tyj in
assert (eq_constr typ tyj.utj_val);
+ let c = hcons_constr j.uj_val in
let _typ = RegularArity (Vars.subst_univs_level_constr subst typ) in
feedback_completion_typecheck feedback_id;
- j.uj_val, uctx) in
+ c, uctx) in
let def = OpaqueDef (Opaqueproof.create proofterm) in
def, RegularArity typ, None, c.const_entry_polymorphic,
c.const_entry_universes,