aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/elim.mli
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-11-24 08:19:55 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-11-24 08:19:55 +0000
commitf9676380178d7af90d8cdf64662866c82139f116 (patch)
tree78a9e7e9d79a858d62f89b6efb53be0d05f66457 /tactics/elim.mli
parent6c28c8f38c6f47cc772d42e5cc54398785d63bc0 (diff)
Auto,Dhyp,Elim / Reduction de Evar / declarations eliminations
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@132 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/elim.mli')
-rw-r--r--tactics/elim.mli33
1 files changed, 33 insertions, 0 deletions
diff --git a/tactics/elim.mli b/tactics/elim.mli
new file mode 100644
index 000000000..ee1b10a37
--- /dev/null
+++ b/tactics/elim.mli
@@ -0,0 +1,33 @@
+
+(* $Id$ *)
+
+(*i*)
+open Names
+open Term
+open Proof_trees
+open Tacmach
+open Tacticals
+(*i*)
+
+(* Eliminations tactics. *)
+
+val introElimAssumsThen :
+ (branch_assumptions -> tactic) -> branch_args -> tactic
+
+val introCaseAssumsThen :
+ (branch_assumptions -> tactic) -> branch_args -> tactic
+
+val general_decompose_clause : (clause * constr -> bool) -> clause -> tactic
+val general_decompose : (clause * constr -> bool) -> constr -> tactic
+val decompose_nonrec : constr -> tactic
+val decompose_and : constr -> tactic
+val decompose_or : constr -> tactic
+val h_decompose : identifier list -> constr -> tactic
+
+val double_ind : int -> int -> tactic
+
+val intro_pattern : intro_pattern -> tactic
+val intros_pattern : intro_pattern list -> tactic
+val dyn_intro_pattern : tactic_arg list -> tactic
+val v_intro_pattern : tactic_arg list -> tactic
+val h_intro_pattern : intro_pattern -> tactic