src/HOL/Library/Multiset.thy
changeset 63540 f8652d0534fa
parent 63539 70d4d9e5707b
child 63547 00521f181510
--- 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) \<in> (r \<inter> D \<times> D)\<inverse>"
           using \<open>(b, a) \<in> r\<close> using \<open>b \<in># B\<close> and \<open>a \<in># B\<close>
           by (auto simp: D_def)
-        ultimately obtain x where "x \<in># X" and "(a, x) \<in> r"
+        ultimately obtain x where x: "x \<in># X" "(a, x) \<in> r"
           using "1.IH" by blast
-        moreover then have "(b, x) \<in> r"
+        then have "(b, x) \<in> r"
           using \<open>trans r\<close> and \<open>(b, a) \<in> r\<close> by (auto dest: transD)
-        ultimately show ?thesis by blast
+        with x show ?thesis by blast
       qed blast
     qed }
   note B_less = this