src/HOL/Hilbert_Choice.thy
changeset 61076 bdc1e2f0a86a
parent 61032 b57df8eecad6
child 61424 c3658c18b7bc
--- a/src/HOL/Hilbert_Choice.thy	Tue Sep 01 17:25:36 2015 +0200
+++ b/src/HOL/Hilbert_Choice.thy	Tue Sep 01 22:32:58 2015 +0200
@@ -287,7 +287,7 @@
   proof (rule UNIV_eq_I)
     fix x :: 'a
     from b1b2 have "x = inv (\<lambda>y. if y = x then b1 else b2) b1" by (simp add: inv_into_def)
-    thus "x \<in> range (\<lambda>f\<Colon>'a \<Rightarrow> 'b. inv f b1)" by blast
+    thus "x \<in> range (\<lambda>f::'a \<Rightarrow> 'b. inv f b1)" by blast
   qed
   ultimately show "finite (UNIV :: 'a set)" by simp
 qed