summaryrefslogtreecommitdiff
path: root/test-suite/success/unicode_utf8.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/unicode_utf8.v')
-rw-r--r--test-suite/success/unicode_utf8.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/success/unicode_utf8.v b/test-suite/success/unicode_utf8.v
index 8b7764e5..42e32ccc 100644
--- a/test-suite/success/unicode_utf8.v
+++ b/test-suite/success/unicode_utf8.v
@@ -75,7 +75,7 @@ Notation "x ≤ y" := (x<=y) (at level 70, no associativity).
Require Import ZArith.
Open Scope Z_scope.
-Locate "≤". (* still le, not Zle *)
+Locate "≤". (* still le, not Z.le *)
Notation "x ≤ y" := (x<=y) (at level 70, no associativity).
Locate "≤".
Close Scope Z_scope.