src/HOL/Set.thy
changeset 34974 18b41bba42b5
parent 34209 c7f621786035
child 34999 5312d2ffee3b
--- a/src/HOL/Set.thy	Thu Jan 28 11:48:43 2010 +0100
+++ b/src/HOL/Set.thy	Thu Jan 28 11:48:49 2010 +0100
@@ -928,7 +928,7 @@
   outer-level constant, which in this case is just "op :"; we instead need
   to use term-nets to associate patterns with rules.  Also, if a rule fails to
   apply, then the formula should be kept.
-  [("HOL.uminus", Compl_iff RS iffD1), ("HOL.minus", [Diff_iff RS iffD1]),
+  [("uminus", Compl_iff RS iffD1), ("minus", [Diff_iff RS iffD1]),
    ("Int", [IntD1,IntD2]),
    ("Collect", [CollectD]), ("Inter", [InterD]), ("INTER", [INT_D])]
  *)