aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2019-11-27 23:34:56 +0100
committerEmilio Jesus Gallego Arias2019-11-27 23:34:56 +0100
commitd2a995927ccb01dae73960780c7fa0fed0a37e6d (patch)
tree2895a7b5681c7507bfc07929189c7fa0ca29cf77
parentac99c6aba0091d5c1ee9511508e25d399425b61b (diff)
parent2f33fce7ac580d1966476d6d2c0f06a3ec920e6d (diff)
Merge PR #11187: Remove deprecated commands `AddPath`, `AddRecPath` and `DelPath`
Reviewed-by: ejgallego
-rw-r--r--doc/changelog/07-commands-and-options/11187-remove-addpath.rst5
-rw-r--r--tools/coqdoc/output.ml2
-rw-r--r--vernac/g_vernac.mlg10
3 files changed, 7 insertions, 10 deletions
diff --git a/doc/changelog/07-commands-and-options/11187-remove-addpath.rst b/doc/changelog/07-commands-and-options/11187-remove-addpath.rst
new file mode 100644
index 0000000000..283c44fda6
--- /dev/null
+++ b/doc/changelog/07-commands-and-options/11187-remove-addpath.rst
@@ -0,0 +1,5 @@
+- Removed legacy commands ``AddPath``, ``AddRecPath``, and ``DelPath``
+ which were undocumented, broken variants of :cmd:`Add LoadPath`,
+ :cmd:`Add Rec LoadPath`, and :cmd:`Remove LoadPath`
+ (`#11187 <https://github.com/coq/coq/pull/11187>`_,
+ by Maxime Dénès and Théo Zimmermann).
diff --git a/tools/coqdoc/output.ml b/tools/coqdoc/output.ml
index 717c06a868..ae1e1c6ed3 100644
--- a/tools/coqdoc/output.ml
+++ b/tools/coqdoc/output.ml
@@ -30,7 +30,7 @@ let build_table l =
let is_keyword =
build_table
- [ "About"; "AddPath"; "Axiom"; "Abort"; "Chapter"; "Check"; "Coercion"; "Compute"; "CoFixpoint";
+ [ "About"; "Axiom"; "Abort"; "Chapter"; "Check"; "Coercion"; "Compute"; "CoFixpoint";
"CoInductive"; "Corollary"; "Defined"; "Definition"; "End"; "Eval"; "Example";
"Export"; "Fact"; "Fix"; "Fixpoint"; "From"; "Function"; "Generalizable"; "Global"; "Grammar";
"Guarded"; "Goal"; "Hint"; "Debug"; "On";
diff --git a/vernac/g_vernac.mlg b/vernac/g_vernac.mlg
index 3095ab3fe1..8d6724c3b1 100644
--- a/vernac/g_vernac.mlg
+++ b/vernac/g_vernac.mlg
@@ -939,15 +939,7 @@ GRAMMAR EXTEND Gram
| IDENT "Remove"; IDENT "LoadPath"; dir = ne_string ->
{ VernacRemoveLoadPath dir }
- (* For compatibility *)
- | IDENT "AddPath"; dir = ne_string; "as"; alias = as_dirpath ->
- { VernacAddLoadPath (false, dir, alias) }
- | IDENT "AddRecPath"; dir = ne_string; "as"; alias = as_dirpath ->
- { VernacAddLoadPath (true, dir, alias) }
- | IDENT "DelPath"; dir = ne_string ->
- { VernacRemoveLoadPath dir }
-
- (* Type-Checking (pas dans le refman) *)
+ (* Type-Checking *)
| "Type"; c = lconstr -> { VernacGlobalCheck c }
(* Printing (careful factorization of entries) *)