removed problematic simp rule
authoreberlm <eberlm@in.tum.de>
Mon, 03 Apr 2017 22:18:56 +0200
changeset 65354 4ff2ba82d668
parent 65353 ac9391e04ef2
child 65364 db7c97cdcfe7
child 65395 7504569a73c7
removed problematic simp rule
src/HOL/Library/Multiset.thy
--- a/src/HOL/Library/Multiset.thy	Mon Apr 03 19:41:17 2017 +0200
+++ b/src/HOL/Library/Multiset.thy	Mon Apr 03 22:18:56 2017 +0200
@@ -1894,7 +1894,7 @@
   ultimately show ?case by simp
 qed
 
-lemma mset_shuffle [simp]: "zs \<in> shuffle xs ys \<Longrightarrow> mset zs = mset xs + mset ys"
+lemma mset_shuffle: "zs \<in> shuffle xs ys \<Longrightarrow> mset zs = mset xs + mset ys"
   by (induction xs ys arbitrary: zs rule: shuffle.induct) auto
 
 lemma mset_insort [simp]: "mset (insort x xs) = add_mset x (mset xs)"