src/HOL/Decision_Procs/Approximation.thy
changeset 38549 d0385f2764d8
parent 37887 2ae085b07f2f
child 38558 32ad17fe2b9c
--- a/src/HOL/Decision_Procs/Approximation.thy	Thu Aug 19 10:27:12 2010 +0200
+++ b/src/HOL/Decision_Procs/Approximation.thy	Thu Aug 19 11:02:14 2010 +0200
@@ -3301,11 +3301,11 @@
 ML {*
   fun reorder_bounds_tac prems i =
     let
-      fun variable_of_bound (Const ("Trueprop", _) $
+      fun variable_of_bound (Const (@{const_name "Trueprop"}, _) $
                              (Const (@{const_name Set.member}, _) $
                               Free (name, _) $ _)) = name
-        | variable_of_bound (Const ("Trueprop", _) $
-                             (Const ("op =", _) $
+        | variable_of_bound (Const (@{const_name "Trueprop"}, _) $
+                             (Const (@{const_name "op ="}, _) $
                               Free (name, _) $ _)) = name
         | variable_of_bound t = raise TERM ("variable_of_bound", [t])