src/HOL/Library/DAList_Multiset.thy
changeset 63040 eb4ddd18d635
parent 61585 a9599d3d7610
child 63195 f3f08c0d4aaf
--- a/src/HOL/Library/DAList_Multiset.thy	Sun Apr 24 21:31:14 2016 +0200
+++ b/src/HOL/Library/DAList_Multiset.thy	Mon Apr 25 16:09:26 2016 +0200
@@ -313,7 +313,7 @@
     have inv: "ys \<in> ?inv"
       using Cons(2) by auto
     note IH = Cons(1)[OF inv]
-    def Ys \<equiv> "Abs_multiset (count_of ys)"
+    define Ys where "Ys = Abs_multiset (count_of ys)"
     have id: "Abs_multiset (count_of ((a, n) # ys)) = ((op + {# a #}) ^^ n) Ys"
       unfolding Ys_def
     proof (rule multiset_eqI, unfold count)