diff -r d7b5e2a222c2 -r 00521f181510 src/HOL/Library/Multiset.thy --- a/src/HOL/Library/Multiset.thy Sat Jul 23 13:25:44 2016 +0200 +++ b/src/HOL/Library/Multiset.thy Mon Jul 25 11:30:31 2016 +0200 @@ -2429,11 +2429,11 @@ moreover have "(a, b) \ (r \ D \ D)\" using \(b, a) \ r\ using \b \# B\ and \a \# B\ by (auto simp: D_def) - ultimately obtain x where "x \# X" and "(a, x) \ r" + ultimately obtain x where x: "x \# X" "(a, x) \ r" using "1.IH" by blast - moreover then have "(b, x) \ r" + then have "(b, x) \ r" using \trans r\ and \(b, a) \ r\ by (auto dest: transD) - ultimately show ?thesis by blast + with x show ?thesis by blast qed blast qed } note B_less = this @@ -2512,9 +2512,9 @@ obtains a M0 K where "M = M0 + {#a#}" "N = M0 + K" "a \# K" "\b. b \# K \ b < a" proof - - from assms obtain a M0 K where "M = M0 + {#a#}" "N = M0 + K" - "b \# K \ b < a" for b by (blast elim: mult1E) - moreover from this(3) [of a] have "a \# K" by auto + from assms obtain a M0 K where "M = M0 + {#a#}" "N = M0 + K" and + *: "b \# K \ b < a" for b by (blast elim: mult1E) + moreover from * [of a] have "a \# K" by auto ultimately show thesis by (auto intro: that) qed