aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Unicode/Utf8.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Unicode/Utf8.v')
-rw-r--r--theories/Unicode/Utf8.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Unicode/Utf8.v b/theories/Unicode/Utf8.v
index 86ab47768..db7ff08c7 100644
--- a/theories/Unicode/Utf8.v
+++ b/theories/Unicode/Utf8.v
@@ -20,5 +20,5 @@ Check ∀ x z, True -> (∃ y v, x + v ≥ y + z) ∨ x ≤ 0.
(* Integer Arithmetic *)
(* TODO: this should come after ZArith
-Notation "x ≤ y" := (Zle x y) (at level 70, no associativity).
+Notation "x ≤ y" := (Z.le x y) (at level 70, no associativity).
*)