aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/pfedit.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-04-08 14:23:53 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-04-08 14:23:53 +0000
commitae6c56036f05b10b8ec728f474f4fe04ba90c752 (patch)
tree84552c6363dc73449c359e0c9bca926ef3225c3d /proofs/pfedit.mli
parent12fe4b7af1170d00963277a29fd6acc1123aa6d9 (diff)
Applying Tom Prince's patch for build_constant_by_tactic not able to
use a lemma name chosen by the caller (here tclABSTRACT) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13972 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/pfedit.mli')
-rw-r--r--proofs/pfedit.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/proofs/pfedit.mli b/proofs/pfedit.mli
index dde52d0cc..c16445ba3 100644
--- a/proofs/pfedit.mli
+++ b/proofs/pfedit.mli
@@ -180,6 +180,6 @@ val instantiate_nth_evar_com : int -> Topconstr.constr_expr -> unit
(** [build_by_tactic typ tac] returns a term of type [typ] by calling [tac] *)
-val build_constant_by_tactic : named_context_val -> types -> tactic ->
+val build_constant_by_tactic : identifier -> named_context_val -> types -> tactic ->
Entries.definition_entry
val build_by_tactic : types -> tactic -> constr