aboutsummaryrefslogtreecommitdiff
path: root/proofs
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2014-08-01 01:34:54 +0200
committerPierre-Marie Pédrot2014-08-01 01:34:54 +0200
commitd89eaa87029b05ab79002632e9c375fd877c2941 (patch)
treeae4ed61b588b6c485d999c773f1f3c717a27273d /proofs
parent636af8ab15807a93ce08778fac18cbe273fcf49d (diff)
Removing more tactic compatibility layer.
Diffstat (limited to 'proofs')
-rw-r--r--proofs/tacmach.ml1
-rw-r--r--proofs/tacmach.mli1
2 files changed, 2 insertions, 0 deletions
diff --git a/proofs/tacmach.ml b/proofs/tacmach.ml
index d58d1f5a01..f87d03183e 100644
--- a/proofs/tacmach.ml
+++ b/proofs/tacmach.ml
@@ -194,6 +194,7 @@ module New = struct
Constrintern.construct_reference hyps id
let pf_env = Proofview.Goal.env
+ let pf_concl = Proofview.Goal.concl
let pf_type_of gl t =
pf_apply type_of gl t
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index cd4e796d5b..c7729e4160 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -115,6 +115,7 @@ module New : sig
val of_old : (Proof_type.goal Evd.sigma -> 'a) -> [ `NF ] Proofview.Goal.t -> 'a
val pf_env : 'a Proofview.Goal.t -> Environ.env
+ val pf_concl : [ `NF ] Proofview.Goal.t -> types
val pf_type_of : 'a Proofview.Goal.t -> Term.constr -> Term.types
val pf_conv_x : 'a Proofview.Goal.t -> Term.constr -> Term.constr -> bool