aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/decl_mode/g_decl_mode.ml4
diff options
context:
space:
mode:
Diffstat (limited to 'plugins/decl_mode/g_decl_mode.ml4')
-rw-r--r--plugins/decl_mode/g_decl_mode.ml46
1 files changed, 3 insertions, 3 deletions
diff --git a/plugins/decl_mode/g_decl_mode.ml4 b/plugins/decl_mode/g_decl_mode.ml4
index 28aa93975..11862747a 100644
--- a/plugins/decl_mode/g_decl_mode.ml4
+++ b/plugins/decl_mode/g_decl_mode.ml4
@@ -11,7 +11,7 @@
(* arnaud: veiller à l'aspect tutorial des commentaires *)
open Pp
-
+open Tok
open Decl_expr
open Names
open Term
@@ -85,9 +85,9 @@ let vernac_proof_instr instr =
(* We create a new parser entry [proof_mode]. The Declarative proof mode
will replace the normal parser entry for tactics with this one. *)
-let proof_mode = Gram.Entry.create "vernac:proof_command"
+let proof_mode = Gram.entry_create "vernac:proof_command"
(* Auxiliary grammar entry. *)
-let proof_instr = Gram.Entry.create "proofmode:instr"
+let proof_instr = Gram.entry_create "proofmode:instr"
(* Before we can write an new toplevel command (see below)
which takes a [proof_instr] as argument, we need to declare