aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/tacexpr.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-20 14:02:58 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-20 14:02:58 +0000
commit98f6a9d847f4fac14696f51096c8334c9bffda6f (patch)
tree3ab3dabe0f93f38b17434976f0b0c9833b8e3ff5 /proofs/tacexpr.ml
parentfbcd19a076f255614012fd076863ca296c1b2626 (diff)
Only one "in" clause in "destruct" even for a multiple "destruct".
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12348 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/tacexpr.ml')
-rw-r--r--proofs/tacexpr.ml12
1 files changed, 7 insertions, 5 deletions
diff --git a/proofs/tacexpr.ml b/proofs/tacexpr.ml
index ba3c27e63..c3e12c0de 100644
--- a/proofs/tacexpr.ml
+++ b/proofs/tacexpr.ml
@@ -115,10 +115,12 @@ let goal_location_of = function
| _ ->
error "Not a simple \"in\" clause (one hypothesis or the conclusion)"
-type ('constr,'id) induction_clause =
- ('constr with_bindings induction_arg list * 'constr with_bindings option *
- (intro_pattern_expr located option * intro_pattern_expr located option) *
- 'id gclause option)
+type 'constr induction_clause =
+ ('constr with_bindings induction_arg list * 'constr with_bindings option *
+ (intro_pattern_expr located option * intro_pattern_expr located option))
+
+type ('constr,'id) induction_clause_list =
+ 'constr induction_clause list * 'id gclause option
type multi =
| Precisely of int
@@ -170,7 +172,7 @@ type ('constr,'pat,'cst,'ind,'ref,'id,'tac) gen_atomic_tactic_expr =
(* Derived basic tactics *)
| TacSimpleInductionDestruct of rec_flag * quantified_hypothesis
- | TacInductionDestruct of rec_flag * evars_flag * ('constr,'id) induction_clause list
+ | TacInductionDestruct of rec_flag * evars_flag * ('constr,'id) induction_clause_list
| TacDoubleInduction of quantified_hypothesis * quantified_hypothesis
| TacDecomposeAnd of 'constr
| TacDecomposeOr of 'constr