aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing/pcoq.ml4
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-05-31 13:33:01 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-05-31 13:33:01 +0200
commit27dffdea5b46f6282c1584db0555213e744352fa (patch)
tree3f89cd9e8828f1ca1c8a1c10d74f020dcb7543f1 /parsing/pcoq.ml4
parentcb31cd671a0ef4da0cf834dad5b67776098bb0d1 (diff)
Revert "Rename Lexer -> CLexer."
Diffstat (limited to 'parsing/pcoq.ml4')
-rw-r--r--parsing/pcoq.ml44
1 files changed, 2 insertions, 2 deletions
diff --git a/parsing/pcoq.ml4 b/parsing/pcoq.ml4
index f01e25c61..28dc74e81 100644
--- a/parsing/pcoq.ml4
+++ b/parsing/pcoq.ml4
@@ -18,7 +18,7 @@ open Tok (* necessary for camlp4 *)
(** The parser of Coq *)
-module G = GrammarMake (CLexer)
+module G = GrammarMake (Lexer)
(* TODO: this is a workaround, since there isn't such
[warning_verbose] in new camlp4. In camlp5, this ref
@@ -51,7 +51,7 @@ ELSE
| tok -> Stoken ((=) tok, to_string tok)
END
-let gram_token_of_string s = gram_token_of_token (CLexer.terminal s)
+let gram_token_of_string s = gram_token_of_token (Lexer.terminal s)
let camlp4_verbosity silent f x =
let a = !warning_verbose in