aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing/g_tacticnew.ml4
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-07-16 20:14:12 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-07-16 20:14:12 +0000
commitcbb8368f2345d2f2d779ca35bc634e49e3d50e3b (patch)
treef77608eac40fd2afcd0ad0d53414ccc488f8a7cd /parsing/g_tacticnew.ml4
parent763cf4f37e10d9a0e8a2a0e9286c02708a60bf08 (diff)
Suppression quotify
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5922 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'parsing/g_tacticnew.ml4')
-rw-r--r--parsing/g_tacticnew.ml437
1 files changed, 0 insertions, 37 deletions
diff --git a/parsing/g_tacticnew.ml4 b/parsing/g_tacticnew.ml4
index 33cfab4d9..b0ea9d835 100644
--- a/parsing/g_tacticnew.ml4
+++ b/parsing/g_tacticnew.ml4
@@ -71,9 +71,6 @@ let lpar_id_colon =
| _ -> raise Stream.Failure)
| _ -> raise Stream.Failure)
-(* open grammar entries, possibly in quotified form *)
-ifdef Quotify then open Qast
-
open Constr
open Prim
open Tactic
@@ -105,24 +102,6 @@ let local_compute = [FBeta;FIota;FDeltaBut [];FZeta]
let error_oldelim _ = error "OldElim no longer supported"
-ifdef Quotify then
- let induction_arg_of_constr = function
- | Qast.Node ("Nvar", [_;id]) -> Qast.Node ("ElimOnIdent", [id])
- | c -> Qast.Node ("ElimOnConstr", [c])
-
-ifdef Quotify then
-let make_red_flag s = Qast.Apply ("make_red_flag", [s])
-
-ifdef Quotify then
-let local_compute =
- Qast.List [
- Qast.Node ("FBeta", []);
- Qast.Node ("FDeltaBut", [Qast.List []]);
- Qast.Node ("FIota", []);
- Qast.Node ("FZeta", [])]
-
-ifdef Quotify then open Q
-
let join_to_constr loc c2 = (fst loc), snd (Topconstr.constr_loc c2)
(* Auxiliary grammar rules *)
@@ -136,22 +115,6 @@ GEXTEND Gram
[ [ n = integer -> Genarg.ArgArg n
| id = identref -> Genarg.ArgVar id ] ]
;
-(* autoarg_depth:
- [ [ n = OPT natural -> n ] ]
- ;
- autoarg_adding:
- [ [ IDENT "adding" ; "["; l = LIST1 global; "]" -> l | -> [] ] ]
- ;
- autoarg_destructing:
- [ [ IDENT "destructing" -> true | -> false ] ]
- ;
- autoarg_usingTDB:
- [ [ "using"; IDENT "tdb" -> true | -> false ] ]
- ;
- autoargs:
- [ [ a0 = autoarg_depth; l = autoarg_adding;
- a2 = autoarg_destructing; a3 = autoarg_usingTDB -> (a0,l,a2,a3) ] ]
- ;*)
(* An identifier or a quotation meta-variable *)
id_or_meta:
[ [ id = identref -> AI id