src/HOL/Multivariate_Analysis/Brouwer_Fixpoint.thy
changeset 54775 2d3df8633dad
parent 53846 2e4b435e17bc
child 55493 47cac23e3d22
--- a/src/HOL/Multivariate_Analysis/Brouwer_Fixpoint.thy	Mon Dec 16 14:49:18 2013 +0100
+++ b/src/HOL/Multivariate_Analysis/Brouwer_Fixpoint.thy	Mon Dec 16 17:08:22 2013 +0100
@@ -4241,7 +4241,7 @@
   have "{a..b} \<noteq> {}"
     using assms by auto
   with i have *: "a\<bullet>i \<le> b\<bullet>i" "u\<bullet>i \<le> v\<bullet>i"
-    using assms(2) by (auto simp add: interval_eq_empty not_less)
+    using assms(2) by (auto simp add: interval_eq_empty interval)
   have x: "a\<bullet>i\<le>x\<bullet>i" "x\<bullet>i\<le>b\<bullet>i"
     using assms(1)[unfolded mem_interval] using i by auto
   have "0 \<le> (x \<bullet> i - a \<bullet> i) / (b \<bullet> i - a \<bullet> i) * (v \<bullet> i - u \<bullet> i)"