aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/leminv.mli
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-12-14 15:56:25 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-12-14 15:56:25 +0000
commit67f5c70a480c95cfb819fc68439781b5e5e95794 (patch)
tree67b88843ba54b4aefc7f604e18e3a71ec7202fd3 /tactics/leminv.mli
parentcc03a5f82efa451b6827af9a9b42cee356ed4f8a (diff)
Modulification of identifier
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16071 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/leminv.mli')
-rw-r--r--tactics/leminv.mli10
1 files changed, 5 insertions, 5 deletions
diff --git a/tactics/leminv.mli b/tactics/leminv.mli
index 45538690c..5019ceda5 100644
--- a/tactics/leminv.mli
+++ b/tactics/leminv.mli
@@ -16,14 +16,14 @@ open Constrexpr
open Misctypes
val lemInv_gen : quantified_hypothesis -> constr -> tactic
-val lemInvIn_gen : quantified_hypothesis -> constr -> identifier list -> tactic
+val lemInvIn_gen : quantified_hypothesis -> constr -> Id.t list -> tactic
val lemInv_clause :
- quantified_hypothesis -> constr -> identifier list -> tactic
+ quantified_hypothesis -> constr -> Id.t list -> tactic
val inversion_lemma_from_goal :
- int -> identifier -> identifier located -> sorts -> bool ->
- (identifier -> tactic) -> unit
+ int -> Id.t -> Id.t located -> sorts -> bool ->
+ (Id.t -> tactic) -> unit
val add_inversion_lemma_exn :
- identifier -> constr_expr -> glob_sort -> bool -> (identifier -> tactic) ->
+ Id.t -> constr_expr -> glob_sort -> bool -> (Id.t -> tactic) ->
unit