aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/interface
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-13 15:22:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-13 15:22:04 +0000
commit0ea28e6a440e39f9f9645aa55afbfa38a0560b27 (patch)
tree0c211363f17f8b61de400d1cf65ffd88e33cbaea /contrib/interface
parent04d270a46e8c481e0b1f21904c6b25f0b7359fa0 (diff)
Reflet dans l'arbre de syntaxe de la difference syntaxique entre 'Variables a b:A' et 'Variables (a:A) (b:A)'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5198 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/interface')
-rw-r--r--contrib/interface/name_to_ast.ml2
-rw-r--r--contrib/interface/xlate.ml9
2 files changed, 8 insertions, 3 deletions
diff --git a/contrib/interface/name_to_ast.ml b/contrib/interface/name_to_ast.ml
index 29582c382..844352693 100644
--- a/contrib/interface/name_to_ast.ml
+++ b/contrib/interface/name_to_ast.ml
@@ -155,7 +155,7 @@ let make_variable_ast name typ implicits =
let make_variable_ast name typ implicits =
(VernacAssumption
((Local,Definitional),
- [false,((dummy_loc,name), constr_to_ast (body_of_type typ))]))
+ [false,([dummy_loc,name], constr_to_ast (body_of_type typ))]))
::(implicits_to_ast_list implicits);;
diff --git a/contrib/interface/xlate.ml b/contrib/interface/xlate.ml
index 7cf169ec7..d2aff445f 100644
--- a/contrib/interface/xlate.ml
+++ b/contrib/interface/xlate.ml
@@ -1281,8 +1281,13 @@ let cvt_optional_eval_for_definition c1 optional_eval =
xlate_formula c1))
let cvt_vernac_binder = function
- | ((_,id),c) ->
- CT_binder(CT_id_opt_ne_list (xlate_ident_opt (Some id),[]),xlate_formula c)
+ | (id::idl,c) ->
+ CT_binder(
+ CT_id_opt_ne_list
+ (xlate_ident_opt (Some (snd id)),
+ List.map (fun id -> xlate_ident_opt (Some (snd id))) idl),
+ xlate_formula c)
+ | ([],_) -> xlate_error "Empty list of vernac binder"
let cvt_vernac_binders args =
CT_binder_list(List.map cvt_vernac_binder args)