aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-03-30 11:13:41 +0200
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-03-30 11:21:52 +0200
commitb4f2e48b9e128a62d63668621844b571d3449cbf (patch)
treec11c1b314742bb7eab40c25d25ed6db6f8de2e9f /parsing
parentd58900ce20a6a7144db386a02093d3fc1c54c894 (diff)
grammar: export hypident
This is necessary to make ssr compile with both camlp4/5
Diffstat (limited to 'parsing')
-rw-r--r--parsing/g_tactic.ml42
-rw-r--r--parsing/pcoq.ml41
-rw-r--r--parsing/pcoq.mli1
3 files changed, 3 insertions, 1 deletions
diff --git a/parsing/g_tactic.ml4 b/parsing/g_tactic.ml4
index b42b2c6dd..69593f993 100644
--- a/parsing/g_tactic.ml4
+++ b/parsing/g_tactic.ml4
@@ -202,7 +202,7 @@ let merge_occurrences loc cl = function
GEXTEND Gram
GLOBAL: simple_tactic constr_with_bindings quantified_hypothesis
bindings red_expr int_or_var open_constr uconstr
- simple_intropattern clause_dft_concl;
+ simple_intropattern clause_dft_concl hypident;
int_or_var:
[ [ n = integer -> ArgArg n
diff --git a/parsing/pcoq.ml4 b/parsing/pcoq.ml4
index cf6435fec..6a9848c1c 100644
--- a/parsing/pcoq.ml4
+++ b/parsing/pcoq.ml4
@@ -375,6 +375,7 @@ module Tactic =
make_gen_entry utactic (rawwit wit_constr_with_bindings) "constr_with_bindings"
let bindings =
make_gen_entry utactic (rawwit wit_bindings) "bindings"
+ let hypident = Gram.entry_create "hypident"
let constr_may_eval = make_gen_entry utactic (rawwit wit_constr_may_eval) "constr_may_eval"
let uconstr =
make_gen_entry utactic (rawwit wit_uconstr) "uconstr"
diff --git a/parsing/pcoq.mli b/parsing/pcoq.mli
index dbd2aadf9..e23b65e12 100644
--- a/parsing/pcoq.mli
+++ b/parsing/pcoq.mli
@@ -215,6 +215,7 @@ module Tactic :
val open_constr : open_constr_expr Gram.entry
val constr_with_bindings : constr_expr with_bindings Gram.entry
val bindings : constr_expr bindings Gram.entry
+ val hypident : (Id.t located * Locus.hyp_location_flag) Gram.entry
val constr_may_eval : (constr_expr,reference or_by_notation,constr_expr) may_eval Gram.entry
val uconstr : constr_expr Gram.entry
val quantified_hypothesis : quantified_hypothesis Gram.entry