this warning is hardly useful but produces noisy markers in the jedit interface
authornipkow
Tue, 12 May 2015 08:48:11 +0200
changeset 60184 7541f29492c3
parent 60183 4cd4c204578c
child 60185 cc71f01f9fde
this warning is hardly useful but produces noisy markers in the jedit interface
src/Pure/raw_simplifier.ML
--- a/src/Pure/raw_simplifier.ML	Sat May 09 12:19:24 2015 +0200
+++ b/src/Pure/raw_simplifier.ML	Tue May 12 08:48:11 2015 +0200
@@ -630,10 +630,6 @@
       val a = the (cong_name (head_of lhs)) handle Option.Option =>
         raise SIMPLIFIER ("Congruence must start with a constant or free variable", [thm]);
       val (xs, weak) = congs;
-      val _ =
-        if AList.defined (op =) xs a then
-          cond_warning ctxt (fn () => "Overwriting congruence rule for " ^ quote (#2 a))
-        else ();
       val xs' = AList.update (op =) (a, thm) xs;
       val weak' = if is_full_cong thm then weak else a :: weak;
     in ((xs', weak'), procs, mk_rews, termless, subgoal_tac, loop_tacs, solvers) end);