src/HOL/Library/Multiset.thy
changeset 63539 70d4d9e5707b
parent 63524 4ec755485732
child 63540 f8652d0534fa
--- a/src/HOL/Library/Multiset.thy	Thu Jul 21 10:52:27 2016 +0200
+++ b/src/HOL/Library/Multiset.thy	Fri Jul 22 08:02:37 2016 +0200
@@ -2493,9 +2493,9 @@
   obtains a M0 K where "M = M0 + {#a#}" "N = M0 + K"
     "a \<notin># K" "\<And>b. b \<in># K \<Longrightarrow> b < a"
 proof -
-  from assms obtain a M0 K where "M = M0 + {#a#}" "N = M0 + K"
-    "b \<in># K \<Longrightarrow> b < a" for b by (blast elim: mult1E)
-  moreover from this(3) [of a] have "a \<notin># K" by auto
+  from assms obtain a M0 K where "M = M0 + {#a#}" "N = M0 + K" and
+    *: "b \<in># K \<Longrightarrow> b < a" for b by (blast elim: mult1E)
+  moreover from * [of a] have "a \<notin># K" by auto
   ultimately show thesis by (auto intro: that)
 qed