aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/interface
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 /plugins/interface
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 'plugins/interface')
-rw-r--r--plugins/interface/depends.ml2
-rw-r--r--plugins/interface/xlate.ml4
2 files changed, 3 insertions, 3 deletions
diff --git a/plugins/interface/depends.ml b/plugins/interface/depends.ml
index 1a5bfaf33..a8bad4c66 100644
--- a/plugins/interface/depends.ml
+++ b/plugins/interface/depends.ml
@@ -305,7 +305,7 @@ let rec depends_of_gen_tactic_expr depends_of_'constr depends_of_'ind depends_of
(* Derived basic tactics *)
| TacSimpleInductionDestruct _
| TacDoubleInduction _ -> acc
- | TacInductionDestruct (_, _, [cwbial, cwbo, _, _]) ->
+ | TacInductionDestruct (_, _, ([cwbial, cwbo, _], _)) ->
list_union_map (depends_of_'a_induction_arg depends_of_'constr_with_bindings)
cwbial
(Option.fold_right depends_of_'constr_with_bindings cwbo acc)
diff --git a/plugins/interface/xlate.ml b/plugins/interface/xlate.ml
index a322c7a72..613c31db7 100644
--- a/plugins/interface/xlate.ml
+++ b/plugins/interface/xlate.ml
@@ -1229,11 +1229,11 @@ and xlate_tac =
CT_dauto(xlate_int_or_var_opt_to_int_opt a, xlate_int_opt b)
| TacDAuto (a, b, _) ->
xlate_error "TODO: dauto using"
- | TacInductionDestruct(true,false,[a,b,(None,c),None]) ->
+ | TacInductionDestruct(true,false,([a,b,(None,c)],None)) ->
CT_new_destruct
(List.map xlate_int_or_constr a, xlate_using b,
xlate_with_names c)
- | TacInductionDestruct(false,false,[a,b,(None,c),None]) ->
+ | TacInductionDestruct(false,false,([a,b,(None,c)],None)) ->
CT_new_induction
(List.map xlate_int_or_constr a, xlate_using b,
xlate_with_names c)