aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/coq-syntax.el
diff options
context:
space:
mode:
authorGravatar Jason Gross <jasongross9@gmail.com>2016-08-13 15:00:38 -0700
committerGravatar Erik Martin-Dorel <erik@martin-dorel.org>2016-08-14 00:00:38 +0200
commit01245b99b1d4b397ccfde65eeb59428f1d271539 (patch)
treeb04fdbd0934d5a6cb3b95e7c15b9bff75ca2d53e /coq/coq-syntax.el
parent462e3efa33e9ceeb19ede020d6471c3bb0215ea6 (diff)
Add Reserved Infix like Reserved Notation (#95)
Diffstat (limited to 'coq/coq-syntax.el')
-rw-r--r--coq/coq-syntax.el3
1 files changed, 2 insertions, 1 deletions
diff --git a/coq/coq-syntax.el b/coq/coq-syntax.el
index 8b09818b..195636a5 100644
--- a/coq/coq-syntax.el
+++ b/coq/coq-syntax.el
@@ -642,6 +642,7 @@ so for the following reasons:
("Require Export" nil "Require Export #." t "Require\\s-+Export")
("Require Import" nil "Require Import #." t "Require\\s-+Import")
("Require" nil "Require #." t "Require")
+ ("Reserved Infix" nil "Reserved Infix" nil "Reserved\\s-+Infix")
("Reserved Notation" nil "Reserved Notation" nil "Reserved\\s-+Notation")
("Reset Extraction Inline" nil "Reset Extraction Inline." t "Reset\\s-+Extraction\\s-+Inline")
("Save" nil "Save." t "Save")
@@ -1230,7 +1231,7 @@ It is used:
(defconst coq-exists-regexp "\\(?:\\_<exists\\_>\\|∃\\)")
(defvar coq-font-lock-terms
- (append
+ (append
(list ;; flattened by append above
(cons coq-symbol-binders 'coq-symbol-binder-face))
(when coq-symbol-highlight-enable