aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tacinterp.ml
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 /tactics/tacinterp.ml
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 'tactics/tacinterp.ml')
-rw-r--r--tactics/tacinterp.ml8
1 files changed, 4 insertions, 4 deletions
diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml
index 5f2baf8f8..18b7604fb 100644
--- a/tactics/tacinterp.ml
+++ b/tactics/tacinterp.ml
@@ -854,7 +854,7 @@ and intern_genarg ist x =
| ConstrMayEvalArgType ->
in_gen globwit_constr_may_eval
(intern_constr_may_eval ist (out_gen rawwit_constr_may_eval x))
- | QuantVarArgType ->
+ | QuantHypArgType ->
in_gen globwit_quant_hyp
(intern_quantified_hypothesis ist (out_gen rawwit_quant_hyp x))
| RedExprArgType ->
@@ -1609,7 +1609,7 @@ and interp_genarg ist goal x =
in_gen wit_constr (pf_interp_constr ist goal (out_gen globwit_constr x))
| ConstrMayEvalArgType ->
in_gen wit_constr_may_eval (interp_constr_may_eval ist goal (out_gen globwit_constr_may_eval x))
- | QuantVarArgType ->
+ | QuantHypArgType ->
in_gen wit_quant_hyp
(interp_declared_or_quantified_hypothesis ist goal
(out_gen globwit_quant_hyp x))
@@ -1828,7 +1828,7 @@ and interp_atomic ist gl = function
| TacticArgType n ->
val_interp ist gl (out_gen (globwit_tactic n) x)
| StringArgType | BoolArgType
- | QuantVarArgType | RedExprArgType
+ | QuantHypArgType | RedExprArgType
| OpenConstrArgType _ | ConstrWithBindingsArgType | BindingsArgType
| ExtraArgType _ | List0ArgType _ | List1ArgType _ | OptArgType _ | PairArgType _
-> error "This generic type is not supported in alias"
@@ -2121,7 +2121,7 @@ and subst_genarg subst (x:glob_generic_argument) =
in_gen globwit_constr (subst_rawconstr subst (out_gen globwit_constr x))
| ConstrMayEvalArgType ->
in_gen globwit_constr_may_eval (subst_raw_may_eval subst (out_gen globwit_constr_may_eval x))
- | QuantVarArgType ->
+ | QuantHypArgType ->
in_gen globwit_quant_hyp
(subst_declared_or_quantified_hypothesis subst
(out_gen globwit_quant_hyp x))