src/HOL/Multivariate_Analysis/Integration.thy
changeset 59765 26d1c71784f1
parent 59647 c6f413b660cf
child 60180 09a7481c03b1
--- a/src/HOL/Multivariate_Analysis/Integration.thy	Fri Mar 20 14:06:15 2015 +0000
+++ b/src/HOL/Multivariate_Analysis/Integration.thy	Fri Mar 20 16:11:28 2015 +0000
@@ -1466,7 +1466,7 @@
       using division_ofD[OF p] by auto
     show "\<exists>p. p division_of \<Union>insert x F"
       using elementary_union_interval[OF p[unfolded *], of a b]
-      unfolding Union_insert x * by auto
+      unfolding Union_insert x * by metis
   qed (insert assms, auto)
   then show ?thesis
     apply -
@@ -4662,7 +4662,7 @@
           apply auto
           done
         ultimately show "u\<bullet>j = a\<bullet>j \<and> v\<bullet>j = a\<bullet>j \<or> u\<bullet>j = b\<bullet>j \<and> v\<bullet>j = b\<bullet>j \<or> u\<bullet>j = a\<bullet>j \<and> v\<bullet>j = b\<bullet>j"
-          unfolding not_less de_Morgan_disj using ab[rule_format,of j] uv(2) j by auto
+          unfolding not_less de_Morgan_disj using ab[rule_format,of j] uv(2) j by force
       qed
       have "(1/2) *\<^sub>R (a+b) \<in> cbox a b"
         unfolding mem_box using ab by(auto intro!: less_imp_le simp: inner_simps)