src/HOL/HOL.thy
changeset 67405 e9ab4ad7bd15
parent 67399 eab6ce8368fa
child 67443 3abf6a722518
--- a/src/HOL/HOL.thy	Thu Jan 11 12:32:07 2018 +0100
+++ b/src/HOL/HOL.thy	Thu Jan 11 13:48:17 2018 +0100
@@ -1607,7 +1607,7 @@
     type T = ((term -> bool) * stamp) list;
     val empty = [];
     val extend = I;
-    fun merge data : T = Library.merge (eq_snd (=)) data;
+    fun merge data : T = Library.merge (eq_snd (op =)) data;
   );
   fun add m = Data.map (cons (m, stamp ()));
   fun matches thy t = exists (fn (m, _) => m t) (Data.get thy);