src/HOL/Analysis/Homotopy.thy
changeset 71633 07bec530f02e
parent 71233 da28fd2852ed
child 71745 ad84f8a712b4
--- a/src/HOL/Analysis/Homotopy.thy	Mon Mar 30 10:35:10 2020 +0200
+++ b/src/HOL/Analysis/Homotopy.thy	Tue Mar 31 15:51:15 2020 +0200
@@ -901,7 +901,7 @@
     apply (rule pip [unfolded path_image_def, THEN subsetD])
     apply (rule image_eqI, blast)
     apply (simp add: algebra_simps)
-    by (metis add_mono_thms_linordered_semiring(1) affine_ineq linear mult.commute mult.left_neutral mult_right_mono not_le
+    by (metis add_mono_thms_linordered_semiring(1) affine_ineq linear mult.commute mult.left_neutral mult_right_mono
               add.commute zero_le_numeral)
   have qs: "\<And>a b. \<lbrakk>4 * b \<le> 3; \<not> b * 2 \<le> 1\<rbrakk> \<Longrightarrow> q (4 * b - 2) \<in> s"
     using path_image_def piq by fastforce