aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-04-18 14:47:34 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-04-18 14:47:34 +0000
commit060c10020b7fce5d47de7a882cff335779c6888e (patch)
tree3b6a598226c3b9cc60b89f047da65438496a78d0 /proofs
parentfc698ea73b9bbf20a12a14f9d6a07eb802a61d27 (diff)
Two dead functions in Tacmach.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15202 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
-rw-r--r--proofs/tacmach.ml8
-rw-r--r--proofs/tacmach.mli3
2 files changed, 0 insertions, 11 deletions
diff --git a/proofs/tacmach.ml b/proofs/tacmach.ml
index 75e9cdf62..58d72d4b2 100644
--- a/proofs/tacmach.ml
+++ b/proofs/tacmach.ml
@@ -73,14 +73,6 @@ let pf_get_new_ids ids gls =
(fun id acc -> (next_ident_away id (acc@avoid))::acc)
ids []
-let pf_interp_constr gls c =
- let evc = project gls in
- Constrintern.interp_constr evc (pf_env gls) c
-
-let pf_interp_type gls c =
- let evc = project gls in
- Constrintern.interp_type evc (pf_env gls) c
-
let pf_global gls id = Constrintern.construct_reference (pf_hyps gls) id
let pf_parse_const gls = compose (pf_global gls) id_of_string
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index 884a03070..402002de1 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -48,9 +48,6 @@ val pf_type_of : goal sigma -> constr -> types
val pf_check_type : goal sigma -> constr -> types -> unit
val pf_hnf_type_of : goal sigma -> constr -> types
-val pf_interp_constr : goal sigma -> Topconstr.constr_expr -> constr
-val pf_interp_type : goal sigma -> Topconstr.constr_expr -> types
-
val pf_get_hyp : goal sigma -> identifier -> named_declaration
val pf_get_hyp_typ : goal sigma -> identifier -> types