diff -r 70d4d9e5707b -r f8652d0534fa src/HOL/Library/Multiset.thy --- a/src/HOL/Library/Multiset.thy Fri Jul 22 08:02:37 2016 +0200 +++ b/src/HOL/Library/Multiset.thy Fri Jul 22 11:00:43 2016 +0200 @@ -2410,11 +2410,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