aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing/g_ltacnew.ml4
diff options
context:
space:
mode:
Diffstat (limited to 'parsing/g_ltacnew.ml4')
-rw-r--r--parsing/g_ltacnew.ml46
1 files changed, 3 insertions, 3 deletions
diff --git a/parsing/g_ltacnew.ml4 b/parsing/g_ltacnew.ml4
index 2caad4680..945009ae9 100644
--- a/parsing/g_ltacnew.ml4
+++ b/parsing/g_ltacnew.ml4
@@ -31,7 +31,7 @@ open Q
type let_clause_kind =
| LETTOPCLAUSE of Names.identifier * constr_expr
| LETCLAUSE of
- (Names.identifier Util.located * constr_expr may_eval option * raw_tactic_arg)
+ (Names.identifier Util.located * (constr_expr, Libnames.reference Genarg.or_metanum) may_eval option * raw_tactic_arg)
ifdef Quotify then
module Prelude = struct
@@ -60,7 +60,7 @@ end
let arg_of_expr = function
TacArg a -> a
- | e -> Tacexp e
+ | e -> Tacexp (e:raw_tactic_expr)
open Prelude
@@ -136,7 +136,7 @@ GEXTEND Gram
tactic_atom:
[ [ id = METAIDENT -> MetaIdArg (loc,id)
| r = reference -> Reference r
- | "?"; n = natural -> MetaNumArg (loc,n)
+ | "?"; n = natural -> ConstrMayEval (ConstrTerm (CMeta (loc,n)))
| "()" -> TacVoid ] ]
;
input_fun: