aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/term_typing.ml
diff options
context:
space:
mode:
Diffstat (limited to 'kernel/term_typing.ml')
-rw-r--r--kernel/term_typing.ml13
1 files changed, 0 insertions, 13 deletions
diff --git a/kernel/term_typing.ml b/kernel/term_typing.ml
index 147fe8a9d..437f7b832 100644
--- a/kernel/term_typing.ml
+++ b/kernel/term_typing.ml
@@ -24,10 +24,6 @@ open Entries
open Typeops
open Fast_typeops
-let debug = true
-let prerr_endline =
- if debug then prerr_endline else fun _ -> ()
-
let constrain_type env j poly = function
| `None ->
if not poly then (* Old-style polymorphism *)
@@ -46,15 +42,6 @@ let constrain_type env j poly = function
let map_option_typ = function None -> `None | Some x -> `Some x
-let local_constrain_type env j = function
- | None ->
- j.uj_type
- | Some t ->
- let tj = infer_type env t in
- let _ = judge_of_cast env j DEFAULTcast tj in
- assert (eq_constr t tj.utj_val);
- t
-
(* Insertion of constants and parameters in environment. *)
let mk_pure_proof c = (c, Univ.ContextSet.empty), Declareops.no_seff