aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorcoqbot-app[bot]2020-11-05 09:29:41 +0000
committerGitHub2020-11-05 09:29:41 +0000
commit5af74f736d5d621e3934be17d25c69b4ed3c0edf (patch)
treeaecd1ef2031113682340bd3daf298721804030c1
parent81eecfc24f3bb7b7055b6bef5a3db37d1952d0ee (diff)
parente047599a7851d5c757635e966067ca9271577692 (diff)
Merge PR #13231: Remove warning on SSR Search having moved.
Reviewed-by: gares
-rw-r--r--plugins/ssr/ssrvernac.mlg16
-rw-r--r--plugins/ssr/ssrvernac.mli2
-rw-r--r--plugins/ssrsearch/g_search.mlg4
3 files changed, 0 insertions, 22 deletions
diff --git a/plugins/ssr/ssrvernac.mlg b/plugins/ssr/ssrvernac.mlg
index a49a5e8b28..99cf197b78 100644
--- a/plugins/ssr/ssrvernac.mlg
+++ b/plugins/ssr/ssrvernac.mlg
@@ -304,21 +304,6 @@ END
{
- let warn_search_moved_enabled = ref true
- let warn_search_moved = CWarnings.create ~name:"ssr-search-moved"
- ~category:"deprecated" ~default:CWarnings.Enabled
- (fun () ->
- (Pp.strbrk
- "In previous versions of Coq, loading SSReflect had the effect of \
- replacing the built-in 'Search' command with an SSReflect version \
- of that command. \
- Coq's own search feature was still available via 'SearchAbout' \
- (but that alias is deprecated). \
- This replacement no longer happens; now 'Search' calls Coq's own search \
- feature even when SSReflect is loaded. \
- If you want to use SSReflect's deprecated Search command \
- instead of the built-in one, please Require the ssrsearch module."))
-
open G_vernac
}
@@ -328,7 +313,6 @@ GRAMMAR EXTEND Gram
query_command:
[ [ IDENT "Search"; s = search_query; l = search_queries; "." ->
{ let (sl,m) = l in
- if !warn_search_moved_enabled then warn_search_moved ();
fun g ->
Vernacexpr.VernacSearch (Vernacexpr.Search (s::sl),g, m) }
] ]
diff --git a/plugins/ssr/ssrvernac.mli b/plugins/ssr/ssrvernac.mli
index 93339313f0..327a2d4660 100644
--- a/plugins/ssr/ssrvernac.mli
+++ b/plugins/ssr/ssrvernac.mli
@@ -9,5 +9,3 @@
(************************************************************************)
(* This file is (C) Copyright 2006-2015 Microsoft Corporation and Inria. *)
-
-val warn_search_moved_enabled : bool ref
diff --git a/plugins/ssrsearch/g_search.mlg b/plugins/ssrsearch/g_search.mlg
index 5e002e09cc..54fdea0860 100644
--- a/plugins/ssrsearch/g_search.mlg
+++ b/plugins/ssrsearch/g_search.mlg
@@ -301,10 +301,6 @@ let ssrdisplaysearch gr env t =
let pr_res = pr_global gr ++ str ":" ++ spc () ++ pr_lconstr_env env Evd.empty t in
Feedback.msg_notice (hov 2 pr_res ++ fnl ())
-(* Remove the warning entirely when this plugin is loaded. *)
-let _ =
- Ssreflect_plugin.Ssrvernac.warn_search_moved_enabled := false
-
let deprecated_search =
CWarnings.create
~name:"deprecated-ssr-search"