aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/2406.v
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-02-23 11:26:51 +0100
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-02-23 13:37:52 +0100
commitdf2f50db3703b4f7f88f00ac382c7f3f1efaceb3 (patch)
treec11084a17eec2bc25bdcbba715aa1ba50b108272 /test-suite/bugs/closed/2406.v
parent705bf896bfc552e95403d097fe9b8031c598d88b (diff)
Fix some typos in comments.
Diffstat (limited to 'test-suite/bugs/closed/2406.v')
-rw-r--r--test-suite/bugs/closed/2406.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/2406.v b/test-suite/bugs/closed/2406.v
index 1bd66ffcc..3766e795a 100644
--- a/test-suite/bugs/closed/2406.v
+++ b/test-suite/bugs/closed/2406.v
@@ -1,6 +1,6 @@
(* Check correct handling of unsupported notations *)
Notation "'’'" := (fun x => x) (at level 20).
-(* This fails with a syntax error but it is not catched by Fail
+(* This fails with a syntax error but it is not caught by Fail
Fail Definition crash_the_rooster f := ’.
*)