aboutsummaryrefslogtreecommitdiff
path: root/proofs/tacmach.mli
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2019-04-05 02:30:45 +0200
committerEmilio Jesus Gallego Arias2019-04-05 15:05:53 +0200
commit54fdae0929f2a05a89cd5c463b9a739ab2e239b8 (patch)
tree80c38984687249bba8a66e24ad04a48de80c2bfa /proofs/tacmach.mli
parent3c06ce8dc3a95e5dfe3a4c0a9acdc7dd5dac75cb (diff)
[api] [proofs] Remove dependency of proofs on interp.
We perform some cleanup and remove dependency of `proofs/` on `interp/`, which seems logical. In fact, `interp` + `parsing` are quite self-contained, so if there is interest we could also make tactics to depend directly on proofs.
Diffstat (limited to 'proofs/tacmach.mli')
-rw-r--r--proofs/tacmach.mli2
1 files changed, 0 insertions, 2 deletions
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index 1454140dd7..218011c316 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -33,7 +33,6 @@ val pf_hyps_types : Goal.goal sigma -> (Id.t Context.binder_annot * type
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_global : Goal.goal sigma -> Id.t -> evar_map * constr
val pf_unsafe_type_of : Goal.goal sigma -> constr -> types
val pf_type_of : Goal.goal sigma -> constr -> evar_map * types
val pf_hnf_type_of : Goal.goal sigma -> constr -> types
@@ -76,7 +75,6 @@ val pr_glls : Goal.goal list sigma -> Pp.t
module New : sig
val pf_apply : (env -> evar_map -> 'a) -> Proofview.Goal.t -> 'a
- val pf_global : Id.t -> Proofview.Goal.t -> GlobRef.t
(** FIXME: encapsulate the level in an existential type. *)
val of_old : (Goal.goal Evd.sigma -> 'a) -> Proofview.Goal.t -> 'a