aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-21 21:04:29 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-21 21:04:29 +0000
commita581a7ba67cf3fadb2f80db0f0174cd385162bd6 (patch)
tree5f4280b5a11981f6c36d8e12e76cbba95e15ef01
parent0e0769892a42d5790efa9e33023c3f4332417add (diff)
Harmonisation de l'interprétation des intropattern
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8967 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--tactics/tacinterp.ml18
1 files changed, 10 insertions, 8 deletions
diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml
index 0c7f65c2a..7ab8df773 100644
--- a/tactics/tacinterp.ml
+++ b/tactics/tacinterp.ml
@@ -1018,11 +1018,11 @@ let interp_ident ist id =
try match List.assoc id ist.lfun with
| VIntroPattern (IntroIdentifier id) -> id
| VConstr c when isVar c ->
- (* This happends e.g. in definitions like "Tac H = Clear H; Intro H" *)
+ (* This happens e.g. in definitions like "Tac H = Clear H; Intro H" *)
(* c is then expected not to belong to the proof context *)
(* would be checkable if env were known from interp_ident *)
destVar c
- | _ -> user_err_loc(loc,"interp_ident", str "An ltac name (" ++ pr_id id ++
+ | _ -> user_err_loc(loc,"", str "An ltac name (" ++ pr_id id ++
str ") should have been bound to an identifier")
with Not_found -> id
@@ -1037,11 +1037,11 @@ let interp_intro_pattern_var ist id =
try match List.assoc id ist.lfun with
| VIntroPattern ipat -> ipat
| VConstr c when isVar c ->
- (* This happends e.g. in definitions like "Tac H = Clear H; Intro H" *)
+ (* This happens e.g. in definitions like "Tac H = Clear H; Intro H" *)
(* c is then expected not to belong to the proof context *)
- (* would be checkable if env were known from interp_ident *)
+ (* would be checkable if env were known from interp_intro_pattern_var *)
IntroIdentifier (destVar c)
- | _ -> user_err_loc(loc,"interp_ident", str "An ltac name (" ++ pr_id id ++
+ | _ -> user_err_loc(loc,"", str "An ltac name (" ++ pr_id id ++
str ") should have been bound to an introduction pattern")
with Not_found -> IntroIdentifier id
@@ -1437,7 +1437,7 @@ and interp_tacarg ist gl = function
| TacVoid -> VVoid
| Reference r -> interp_ltac_reference false false ist gl r
| Integer n -> VInteger n
- | IntroPattern ipat -> VIntroPattern ipat
+ | IntroPattern ipat -> VIntroPattern (interp_intro_pattern ist ipat)
| ConstrMayEval c -> VConstr (interp_constr_may_eval ist gl c)
| MetaIdArg (loc,id) -> assert false
| TacCall (loc,r,[]) -> interp_ltac_reference false true ist gl r
@@ -1874,9 +1874,11 @@ and interp_atomic ist gl = function
| PreIdentArgType ->
failwith "pre-identifiers cannot be bound"
| IntroPatternArgType ->
- VIntroPattern (out_gen globwit_intro_pattern x)
+ VIntroPattern
+ (interp_intro_pattern ist (out_gen globwit_intro_pattern x))
| IdentArgType ->
- VIntroPattern (IntroIdentifier (out_gen globwit_ident x))
+ VIntroPattern
+ (IntroIdentifier (interp_ident ist (out_gen globwit_ident x)))
| VarArgType ->
VConstr (mkVar (interp_hyp ist gl (out_gen globwit_var x)))
| RefArgType ->