aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-26 17:08:16 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-26 17:08:16 +0000
commit099fb1b4c5084bb899e4910e42c971cdfa81e1aa (patch)
tree33aa85efc447dd483613243a65ce5a31763d8d5e /parsing
parent989718e36ca338a64c248723d2590bb3eb4854a5 (diff)
Petite correction nom QuantHypArgType suite suppression traducteur
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7739 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'parsing')
-rw-r--r--parsing/argextend.ml46
-rw-r--r--parsing/pptactic.ml6
-rw-r--r--parsing/q_coqast.ml42
3 files changed, 7 insertions, 7 deletions
diff --git a/parsing/argextend.ml4 b/parsing/argextend.ml4
index 331df4c70..d1f82c1d9 100644
--- a/parsing/argextend.ml4
+++ b/parsing/argextend.ml4
@@ -29,7 +29,7 @@ let rec make_rawwit loc = function
| SortArgType -> <:expr< Genarg.rawwit_sort >>
| ConstrArgType -> <:expr< Genarg.rawwit_constr >>
| ConstrMayEvalArgType -> <:expr< Genarg.rawwit_constr_may_eval >>
- | QuantVarArgType -> <:expr< Genarg.rawwit_quant_hyp >>
+ | QuantHypArgType -> <:expr< Genarg.rawwit_quant_hyp >>
| TacticArgType n -> <:expr< Genarg.rawwit_tactic $mlexpr_of_int n$ >>
| RedExprArgType -> <:expr< Genarg.rawwit_red_expr >>
| OpenConstrArgType b -> <:expr< Genarg.rawwit_open_constr_gen $mlexpr_of_bool b$ >>
@@ -52,7 +52,7 @@ let rec make_globwit loc = function
| IdentArgType -> <:expr< Genarg.globwit_ident >>
| VarArgType -> <:expr< Genarg.globwit_var >>
| RefArgType -> <:expr< Genarg.globwit_ref >>
- | QuantVarArgType -> <:expr< Genarg.globwit_quant_hyp >>
+ | QuantHypArgType -> <:expr< Genarg.globwit_quant_hyp >>
| SortArgType -> <:expr< Genarg.globwit_sort >>
| ConstrArgType -> <:expr< Genarg.globwit_constr >>
| ConstrMayEvalArgType -> <:expr< Genarg.globwit_constr_may_eval >>
@@ -78,7 +78,7 @@ let rec make_wit loc = function
| IdentArgType -> <:expr< Genarg.wit_ident >>
| VarArgType -> <:expr< Genarg.wit_var >>
| RefArgType -> <:expr< Genarg.wit_ref >>
- | QuantVarArgType -> <:expr< Genarg.wit_quant_hyp >>
+ | QuantHypArgType -> <:expr< Genarg.wit_quant_hyp >>
| SortArgType -> <:expr< Genarg.wit_sort >>
| ConstrArgType -> <:expr< Genarg.wit_constr >>
| ConstrMayEvalArgType -> <:expr< Genarg.wit_constr_may_eval >>
diff --git a/parsing/pptactic.ml b/parsing/pptactic.ml
index 9803c0031..8360e280a 100644
--- a/parsing/pptactic.ml
+++ b/parsing/pptactic.ml
@@ -141,7 +141,7 @@ let rec pr_raw_generic prc prlc prtac prref x =
| ConstrMayEvalArgType ->
pr_arg (pr_may_eval prc prlc prref)
(out_gen rawwit_constr_may_eval x)
- | QuantVarArgType ->
+ | QuantHypArgType ->
pr_arg pr_quantified_hypothesis (out_gen rawwit_quant_hyp x)
| RedExprArgType ->
pr_arg (pr_red_expr (prc,prlc,prref)) (out_gen rawwit_red_expr x)
@@ -184,7 +184,7 @@ let rec pr_glob_generic prc prlc prtac x =
| ConstrMayEvalArgType ->
pr_arg (pr_may_eval prc prlc
(pr_or_var (pr_and_short_name pr_evaluable_reference))) (out_gen globwit_constr_may_eval x)
- | QuantVarArgType ->
+ | QuantHypArgType ->
pr_arg pr_quantified_hypothesis (out_gen globwit_quant_hyp x)
| RedExprArgType ->
pr_arg (pr_red_expr
@@ -229,7 +229,7 @@ let rec pr_generic prc prlc prtac x =
| ConstrArgType -> pr_arg prc (out_gen wit_constr x)
| ConstrMayEvalArgType ->
pr_arg prc (out_gen wit_constr_may_eval x)
- | QuantVarArgType ->
+ | QuantHypArgType ->
pr_arg pr_quantified_hypothesis (out_gen wit_quant_hyp x)
| RedExprArgType ->
pr_arg (pr_red_expr (prc,prlc,pr_evaluable_reference))
diff --git a/parsing/q_coqast.ml4 b/parsing/q_coqast.ml4
index d28b36924..f8172ac6e 100644
--- a/parsing/q_coqast.ml4
+++ b/parsing/q_coqast.ml4
@@ -173,7 +173,7 @@ let rec mlexpr_of_argtype loc = function
| Genarg.IdentArgType -> <:expr< Genarg.IdentArgType >>
| Genarg.VarArgType -> <:expr< Genarg.VarArgType >>
| Genarg.StringArgType -> <:expr< Genarg.StringArgType >>
- | Genarg.QuantVarArgType -> <:expr< Genarg.QuantVarArgType >>
+ | Genarg.QuantHypArgType -> <:expr< Genarg.QuantHypArgType >>
| Genarg.OpenConstrArgType b -> <:expr< Genarg.OpenConstrArgType $mlexpr_of_bool b$ >>
| Genarg.ConstrWithBindingsArgType -> <:expr< Genarg.ConstrWithBindingsArgType >>
| Genarg.BindingsArgType -> <:expr< Genarg.BindingsArgType >>