src/HOL/Analysis/Convex_Euclidean_Space.thy
changeset 64240 eabf80376aab
parent 64122 74fde524799e
child 64267 b9a1486e79be
--- a/src/HOL/Analysis/Convex_Euclidean_Space.thy	Sun Oct 16 09:31:03 2016 +0200
+++ b/src/HOL/Analysis/Convex_Euclidean_Space.thy	Sun Oct 16 09:31:04 2016 +0200
@@ -11985,7 +11985,7 @@
   have "UNIV \<subseteq> {x. a \<bullet> x = b} \<Longrightarrow> a = 0 \<and> b = 0"
     apply (drule_tac c = "((b+1) / (a \<bullet> a)) *\<^sub>R a" in subsetD)
     apply simp_all
-    by (metis add_cancel_right_right divide_1 zero_neq_one)
+    by (metis add_cancel_right_right div_by_1 zero_neq_one)
   then show ?thesis by force
 qed