diff options
author | Gaëtan Gilbert <gaetan.gilbert@ens-lyon.fr> | 2017-08-31 17:28:46 +0200 |
---|---|---|
committer | Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net> | 2018-07-03 13:39:18 +0200 |
commit | c11bd7b181d6e53910dc8d39c5360f35c7b24674 (patch) | |
tree | 168f7c1ca05dc939e9d8af20efc1f678c5b189ba | |
parent | 1254a28735a242cda2221d2018075808c5b899c7 (diff) |
Cooking.cook_constant: remove unused env argument.
Unused since d95306323 (remove template polymorphic definitions).
-rw-r--r-- | kernel/cooking.ml | 2 | ||||
-rw-r--r-- | kernel/cooking.mli | 3 | ||||
-rw-r--r-- | kernel/term_typing.ml | 2 |
3 files changed, 3 insertions, 4 deletions
diff --git a/kernel/cooking.ml b/kernel/cooking.ml index 521a7d890..094609b96 100644 --- a/kernel/cooking.ml +++ b/kernel/cooking.ml @@ -204,7 +204,7 @@ let lift_univs cb subst auctx0 = let auctx' = Univ.subst_univs_level_abstract_universe_context (Univ.make_instance_subst subst) auctx in subst, (Polymorphic_const (AUContext.union auctx0 auctx')) -let cook_constant ~hcons env { from = cb; info } = +let cook_constant ~hcons { from = cb; info } = let { Opaqueproof.modlist; abstract } = info in let cache = RefTable.create 13 in let abstract, usubst, abs_ctx = abstract in diff --git a/kernel/cooking.mli b/kernel/cooking.mli index 4c254d2ea..6ebe691b8 100644 --- a/kernel/cooking.mli +++ b/kernel/cooking.mli @@ -10,7 +10,6 @@ open Constr open Declarations -open Environ (** {6 Cooking the constants. } *) @@ -26,7 +25,7 @@ type result = { cook_context : Constr.named_context option; } -val cook_constant : hcons:bool -> env -> recipe -> result +val cook_constant : hcons:bool -> recipe -> result val cook_constr : Opaqueproof.cooking_info -> constr -> constr (** {6 Utility functions used in module [Discharge]. } *) diff --git a/kernel/term_typing.ml b/kernel/term_typing.ml index bad449731..30127d166 100644 --- a/kernel/term_typing.ml +++ b/kernel/term_typing.ml @@ -554,7 +554,7 @@ let translate_recipe env kn r = be useless. It is detected by the dirpath of the constant being empty. *) let (_, dir, _) = Constant.repr3 kn in let hcons = DirPath.is_empty dir in - build_constant_declaration kn env (Cooking.cook_constant ~hcons env r) + build_constant_declaration kn env (Cooking.cook_constant ~hcons r) let translate_local_def env id centry = let open Cooking in |