aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
-rw-r--r--doc/changelog/07-commands-and-options/13556-master.rst4
-rw-r--r--doc/sphinx/user-extensions/syntax-extensions.rst2
-rw-r--r--test-suite/output/bug_12908.v2
-rw-r--r--vernac/metasyntax.ml4
4 files changed, 8 insertions, 4 deletions
diff --git a/doc/changelog/07-commands-and-options/13556-master.rst b/doc/changelog/07-commands-and-options/13556-master.rst
new file mode 100644
index 0000000000..05a60026a3
--- /dev/null
+++ b/doc/changelog/07-commands-and-options/13556-master.rst
@@ -0,0 +1,4 @@
+- **Changed:**
+ The warning `custom-entry-overriden` has been renamed to `custom-entry-overridden` (with two d's).
+ (`#13556 <https://github.com/coq/coq/pull/13556>`_,
+ by Simon Friis Vindum).
diff --git a/doc/sphinx/user-extensions/syntax-extensions.rst b/doc/sphinx/user-extensions/syntax-extensions.rst
index 4dbf3b150b..73f90b0056 100644
--- a/doc/sphinx/user-extensions/syntax-extensions.rst
+++ b/doc/sphinx/user-extensions/syntax-extensions.rst
@@ -309,7 +309,7 @@ at the time of use of the notation.
a notation should only be used for printing.
If a notation to be used both for parsing and printing is
- overriden, both the parsing and printing are invalided, even if the
+ overridden, both the parsing and printing are invalided, even if the
overriding rule is only parsing.
If a given notation string occurs only in ``only printing`` rules,
diff --git a/test-suite/output/bug_12908.v b/test-suite/output/bug_12908.v
index 6f7be22fa0..7ab218a27a 100644
--- a/test-suite/output/bug_12908.v
+++ b/test-suite/output/bug_12908.v
@@ -7,7 +7,7 @@ Check forall m n, mult' m n = Nat.mul (Nat.mul 2 m) n.
End A.
Module B.
-(* Test that an overriden scoped notation is deactivated *)
+(* Test that an overridden scoped notation is deactivated *)
Infix "*" := mult' : nat_scope.
Check forall m n, mult' m n = Nat.mul (Nat.mul 2 m) n.
End B.
diff --git a/vernac/metasyntax.ml b/vernac/metasyntax.ml
index 06eb330958..e6244ee3b5 100644
--- a/vernac/metasyntax.ml
+++ b/vernac/metasyntax.ml
@@ -1822,9 +1822,9 @@ let add_syntactic_definition ~local deprecation env ident (vars,c) { onlyparsing
(* Declaration of custom entry *)
let warn_custom_entry =
- CWarnings.create ~name:"custom-entry-overriden" ~category:"parsing"
+ CWarnings.create ~name:"custom-entry-overridden" ~category:"parsing"
(fun s ->
- strbrk "Custom entry " ++ str s ++ strbrk " has been overriden.")
+ strbrk "Custom entry " ++ str s ++ strbrk " has been overridden.")
let load_custom_entry _ _ = ()