src/HOL/Fields.thy
changeset 61076 bdc1e2f0a86a
parent 60758 d8d85a8172b5
child 61238 e3d8a313a649
--- a/src/HOL/Fields.thy	Tue Sep 01 17:25:36 2015 +0200
+++ b/src/HOL/Fields.thy	Tue Sep 01 22:32:58 2015 +0200
@@ -1161,7 +1161,7 @@
     unfolding le_divide_eq if_P[OF \<open>0 < x\<close>] by simp
 next
   assume "\<not>0 < x" hence "x \<le> 0" by simp
-  obtain s::'a where s: "0 < s" "s < 1" using dense[of 0 "1\<Colon>'a"] by auto
+  obtain s::'a where s: "0 < s" "s < 1" using dense[of 0 "1::'a"] by auto
   hence "x \<le> s * x" using mult_le_cancel_right[of 1 x s] \<open>x \<le> 0\<close> by auto
   also note *[OF s]
   finally show ?thesis .