src/HOL/HOL.thy
changeset 43597 b4a093e755db
parent 43560 d1650e3720fd
child 43654 3f1a44c2d645
--- a/src/HOL/HOL.thy	Wed Jun 29 20:39:41 2011 +0200
+++ b/src/HOL/HOL.thy	Wed Jun 29 21:34:16 2011 +0200
@@ -1232,7 +1232,7 @@
   fun proc ss ct =
     (case Thm.term_of ct of
       eq $ lhs $ rhs =>
-        (case find_first (is_neq eq lhs rhs) (Simplifier.prems_of_ss ss) of
+        (case find_first (is_neq eq lhs rhs) (Simplifier.prems_of ss) of
           SOME thm => SOME (thm RS neq_to_EQ_False)
         | NONE => NONE)
      | _ => NONE);