aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/extratactics.ml4
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-23 10:09:59 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-23 10:09:59 +0000
commit50f76559841b54cc5350c4d70ab192d0081d569e (patch)
treedbd87f3db407d9fddb39ce9ae85c679b5b609293 /tactics/extratactics.ml4
parent93642cdc3acb9f4e8d1b4ac1f1621d1104f04e54 (diff)
Correction ident -> hyp pour dinterpréter des identificateurs devant être interprétés comme termes
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8977 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/extratactics.ml4')
-rw-r--r--tactics/extratactics.ml427
1 files changed, 18 insertions, 9 deletions
diff --git a/tactics/extratactics.ml4 b/tactics/extratactics.ml4
index 521bf5409..41b79fefb 100644
--- a/tactics/extratactics.ml4
+++ b/tactics/extratactics.ml4
@@ -50,10 +50,15 @@ let pr_by_arg_tac _prc _prlc prtac opt_c =
n'ai pas reussi
*)
+let pr_in_hyp = function
+ | None -> mt ()
+ | Some id -> spc () ++ hov 2 (str "in" ++ spc () ++ Nameops.pr_id id)
+
let pr_in_arg_hyp _prc _prlc _prtac opt_c =
- match opt_c with
- | None -> mt ()
- | Some id -> spc () ++ hov 2 (str "by" ++ spc () ++ Nameops.pr_id id)
+ pr_in_hyp (Util.option_map snd opt_c)
+
+let pr_in_arg_hyp_typed _prc _prlc _prtac =
+ pr_in_hyp
ARGUMENT EXTEND by_arg_tac
TYPED AS tactic_opt
@@ -63,9 +68,13 @@ ARGUMENT EXTEND by_arg_tac
END
ARGUMENT EXTEND in_arg_hyp
- TYPED AS ident_opt
- PRINTED BY pr_in_arg_hyp
-| [ "in" ident(c) ] -> [ Some (c) ]
+ TYPED AS var_opt
+ PRINTED BY pr_in_arg_hyp_typed
+ RAW_TYPED AS var_opt
+ RAW_PRINTED BY pr_in_arg_hyp
+ GLOB_TYPED AS var_opt
+ GLOB_PRINTED BY pr_in_arg_hyp
+| [ "in" hyp(c) ] -> [ Some (c) ]
| [ ] -> [ None ]
END
@@ -183,9 +192,9 @@ TACTIC EXTEND autorewrite
[ autorewrite Refiner.tclIDTAC l ]
| [ "autorewrite" "with" ne_preident_list(l) "using" tactic(t) ] ->
[ autorewrite (snd t) l ]
-| [ "autorewrite" "with" ne_preident_list(l) "in" ident(id) ] ->
+| [ "autorewrite" "with" ne_preident_list(l) "in" hyp(id) ] ->
[ autorewrite_in id Refiner.tclIDTAC l ]
-| [ "autorewrite" "with" ne_preident_list(l) "in" ident(id) "using" tactic(t) ] ->
+| [ "autorewrite" "with" ne_preident_list(l) "in" hyp(id) "using" tactic(t) ] ->
[ autorewrite_in id (snd t) l ]
END
@@ -283,7 +292,7 @@ END
TACTIC EXTEND setoid_symmetry
[ "setoid_symmetry" ] -> [ setoid_symmetry ]
- | [ "setoid_symmetry" "in" ident(n) ] -> [ setoid_symmetry_in n ]
+ | [ "setoid_symmetry" "in" hyp(n) ] -> [ setoid_symmetry_in n ]
END
TACTIC EXTEND setoid_reflexivity