src/HOL/Tools/Nitpick/nitpick_nut.ML
changeset 38864 4abe644fcea5
parent 38795 848be46708dc
child 39343 eac5f82eefb6
--- a/src/HOL/Tools/Nitpick/nitpick_nut.ML	Sat Aug 28 20:24:40 2010 +0800
+++ b/src/HOL/Tools/Nitpick/nitpick_nut.ML	Sat Aug 28 16:14:32 2010 +0200
@@ -447,7 +447,7 @@
                 val t1 = incr_boundvars n t1
                 val t2 = incr_boundvars n t2
                 val xs = map Bound (n - 1 downto 0)
-                val equation = Const (@{const_name "op ="},
+                val equation = Const (@{const_name HOL.eq},
                                       body_T --> body_T --> bool_T)
                                    $ betapplys (t1, xs) $ betapplys (t2, xs)
                 val t =
@@ -515,9 +515,9 @@
           do_description_operator The @{const_name undefined_fast_The} x t1
         | (Const (x as (@{const_name Eps}, _)), [t1]) =>
           do_description_operator Eps @{const_name undefined_fast_Eps} x t1
-        | (Const (@{const_name "op ="}, T), [t1]) =>
+        | (Const (@{const_name HOL.eq}, T), [t1]) =>
           Op1 (SingletonSet, range_type T, Any, sub t1)
-        | (Const (@{const_name "op ="}, T), [t1, t2]) => sub_equals T t1 t2
+        | (Const (@{const_name HOL.eq}, T), [t1, t2]) => sub_equals T t1 t2
         | (Const (@{const_name HOL.conj}, _), [t1, t2]) =>
           Op2 (And, bool_T, Any, sub' t1, sub' t2)
         | (Const (@{const_name HOL.disj}, _), [t1, t2]) =>