aboutsummaryrefslogtreecommitdiff
path: root/proofs/tacmach.mli
diff options
context:
space:
mode:
authorGaëtan Gilbert2020-02-18 14:15:24 +0100
committerGaëtan Gilbert2020-02-18 14:15:24 +0100
commit5d535c7c624cc4ebae23b173254ba6492b33bee2 (patch)
tree8c10b853a80a2e811c2a6f53f94766ad84242a16 /proofs/tacmach.mli
parentaf3fd09e2f0cc2eac2bc8802a6818baf0c184563 (diff)
Deprecate unsafe_type_of
Diffstat (limited to 'proofs/tacmach.mli')
-rw-r--r--proofs/tacmach.mli2
1 files changed, 2 insertions, 0 deletions
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index aed1c89bfe..b4247f39b9 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -34,6 +34,7 @@ val pf_nth_hyp_id : Goal.goal sigma -> int -> Id.t
val pf_last_hyp : Goal.goal sigma -> named_declaration
val pf_ids_of_hyps : Goal.goal sigma -> Id.t list
val pf_unsafe_type_of : Goal.goal sigma -> constr -> types
+[@@ocaml.deprecated "Use [type_of] or retyping according to your needs."]
val pf_type_of : Goal.goal sigma -> constr -> evar_map * types
val pf_hnf_type_of : Goal.goal sigma -> constr -> types
@@ -83,6 +84,7 @@ module New : sig
(** WRONG: To be avoided at all costs, it typechecks the term entirely but
forgets the universe constraints necessary to retypecheck it *)
val pf_unsafe_type_of : Proofview.Goal.t -> constr -> types
+ [@@ocaml.deprecated "Use [type_of] or retyping according to your needs."]
(** This function does no type inference and expects an already well-typed term.
It recomputes its type in the fastest way possible (no conversion is ever involved) *)