aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing/egrammar.mli
diff options
context:
space:
mode:
Diffstat (limited to 'parsing/egrammar.mli')
-rw-r--r--parsing/egrammar.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/parsing/egrammar.mli b/parsing/egrammar.mli
index e632e5bb8..14e4cfd37 100644
--- a/parsing/egrammar.mli
+++ b/parsing/egrammar.mli
@@ -22,7 +22,7 @@ open Mod_subst
(*i*)
(** Mapping of grammar productions to camlp4 actions
- Used for Coq-level Notation and Tactic Notation,
+ Used for Coq-level Notation and Tactic Notation,
and for ML-level tactic and vernac extensions
*)
@@ -32,14 +32,14 @@ type grammar_constr_prod_item =
| GramConstrTerminal of Token.pattern
| GramConstrNonTerminal of constr_prod_entry_key * identifier option
-type notation_grammar =
+type notation_grammar =
int * Gramext.g_assoc option * notation * grammar_constr_prod_item list
(* For tactic and vernac notations *)
type grammar_prod_item =
| GramTerminal of string
- | GramNonTerminal of loc * argument_type *
+ | GramNonTerminal of loc * argument_type *
Gram.te prod_entry_key * identifier option
(* Adding notations *)