aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/interface
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-10-14 14:14:31 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-10-14 14:14:31 +0000
commit8540611088775052e997bd6c0810faabc23e46c6 (patch)
tree3699abdcf3085f6096a8c7fa039bfd220bcf9369 /contrib/interface
parentaa27ea16ab398eda93bdccc9c82b163ba1e23100 (diff)
TacCall attend une référence
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3142 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/interface')
-rw-r--r--contrib/interface/xlate.ml3
1 files changed, 1 insertions, 2 deletions
diff --git a/contrib/interface/xlate.ml b/contrib/interface/xlate.ml
index 5060b17a8..ef7539bff 100644
--- a/contrib/interface/xlate.ml
+++ b/contrib/interface/xlate.ml
@@ -981,11 +981,10 @@ let rec (xlate_tacarg:raw_tactic_arg -> ct_TACTIC_ARG) =
and (xlate_call_or_tacarg:raw_tactic_arg -> ct_TACTIC_COM) =
function
(* Moved from xlate_tactic *)
- | TacCall (_,Reference r, a::l) ->
+ | TacCall (_, r, a::l) ->
CT_simple_user_tac
(reference_to_ct_ID r,
CT_tactic_arg_list(xlate_tacarg a,List.map xlate_tacarg l))
- | TacCall (_,_,_) -> xlate_error ""
| Reference (Coqast.RIdent (_,s)) -> ident_tac s
| t -> xlate_error "TODO: result other than tactic or constr"