summaryrefslogtreecommitdiff
path: root/test-suite/modules/plik.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/modules/plik.v')
-rw-r--r--test-suite/modules/plik.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/test-suite/modules/plik.v b/test-suite/modules/plik.v
index f1f59df0..50bfd960 100644
--- a/test-suite/modules/plik.v
+++ b/test-suite/modules/plik.v
@@ -1,4 +1,3 @@
-Definition toto:=[x:Set]x.
+Definition toto (x : Set) := x.
-Grammar constr constr8 :=
- toto [ "#" constr7($b) ] -> [ (toto $b) ].
+(* <Warning> : Grammar is replaced by Notation *) \ No newline at end of file