aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/TestCase.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-10-06 12:17:45 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-10-06 12:17:45 -0400
commit2c56adb6bc1eb93904366b7acf9a5cc739c919fc (patch)
treef69fa7c85fee2c6317016bdc1f7b95e85b010eb0 /src/Compilers/TestCase.v
parente9c62c5187350066ef80d993805d9b8c19d53a9c (diff)
Coq 8.5 can't handle symbol-free notations
Diffstat (limited to 'src/Compilers/TestCase.v')
-rw-r--r--src/Compilers/TestCase.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/Compilers/TestCase.v b/src/Compilers/TestCase.v
index 83f280d12..858c09a26 100644
--- a/src/Compilers/TestCase.v
+++ b/src/Compilers/TestCase.v
@@ -32,12 +32,12 @@ Inductive op : flat_type base_type -> flat_type base_type -> Type :=
| Add : op (Prod tnat tnat) tnat
| Mul : op (Prod tnat tnat) tnat
| Sub : op (Prod tnat tnat) tnat.
-Notation "x" := (Syntax.Op (Const x) _) (only printing, at level 10) : expr_scope.
-Notation "x" := (Syntax.Var x) (only printing, at level 10) : expr_scope.
+Notation "' x" := (Syntax.Op (Const x) _) (only printing, at level 10) : expr_scope.
+Notation "' x" := (Syntax.Var x) (only printing, at level 10) : expr_scope.
Notation "a + b" := (Syntax.Op Add (a, b)%expr) : expr_scope.
Notation "a * b" := (Syntax.Op Mul (a, b)%expr) : expr_scope.
Notation "a - b" := (Syntax.Op Sub (a, b)%expr) : expr_scope.
-Notation "x" := (Named.Op (Const x) _) (only printing, at level 10) : nexpr_scope.
+Notation "' x" := (Named.Op (Const x) _) (only printing, at level 10) : nexpr_scope.
Notation "a + b" := (Named.Op Add (a, b)%nexpr) : nexpr_scope.
Notation "a * b" := (Named.Op Mul (a, b)%nexpr) : nexpr_scope.
Notation "a - b" := (Named.Op Sub (a, b)%nexpr) : nexpr_scope.