src/HOL/Analysis/Urysohn.thy
changeset 78320 eb9a9690b8f5
parent 78283 6fa0812135e0
child 78336 6bae28577994
--- a/src/HOL/Analysis/Urysohn.thy	Mon Jul 10 18:48:22 2023 +0100
+++ b/src/HOL/Analysis/Urysohn.thy	Tue Jul 11 20:21:58 2023 +0100
@@ -380,7 +380,7 @@
       and ga: "g ` SA \<subseteq> {- d}" and gb: "g ` SB \<subseteq> {d}"
       using Urysohn_lemma \<open>normal_space X\<close> by metis
     then have g_le_d: "\<And>x. x \<in> topspace X \<Longrightarrow> \<bar>g x\<bar> \<le> d"
-      by (simp add: abs_le_iff continuous_map_def minus_le_iff)
+      by (fastforce simp: abs_le_iff continuous_map_def minus_le_iff)
     have g_eq_d: "\<And>x. \<lbrakk>x \<in> S; f x - h x \<le> -d\<rbrakk> \<Longrightarrow> g x = -d"
       using ga by (auto simp: SA_def)
     have g_eq_negd: "\<And>x. \<lbrakk>x \<in> S; f x - h x \<ge> d\<rbrakk> \<Longrightarrow> g x = d"