src/HOL/Tools/Sledgehammer/sledgehammer_mepo.ML
changeset 56245 84fc7dfa3cd4
parent 55286 7bbbd9393ce0
child 57149 7524b440686c
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_mepo.ML	Fri Mar 21 15:12:03 2014 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_mepo.ML	Fri Mar 21 20:33:56 2014 +0100
@@ -187,9 +187,9 @@
       if T = HOLogic.boolT then do_formula else do_term ext_arg
     and do_formula t =
       (case t of
-        Const (@{const_name all}, _) $ Abs (_, _, t') => do_formula t'
-      | @{const "==>"} $ t1 $ t2 => do_formula t1 #> do_formula t2
-      | Const (@{const_name "=="}, Type (_, [T, _])) $ t1 $ t2 =>
+        Const (@{const_name Pure.all}, _) $ Abs (_, _, t') => do_formula t'
+      | @{const Pure.imp} $ t1 $ t2 => do_formula t1 #> do_formula t2
+      | Const (@{const_name Pure.eq}, Type (_, [T, _])) $ t1 $ t2 =>
         do_term_or_formula false T t1 #> do_term_or_formula true T t2
       | @{const Trueprop} $ t1 => do_formula t1
       | @{const False} => I