diff -r 91da58bb560d -r c2128ab11f61 src/HOL/Analysis/Continuous_Extension.thy --- a/src/HOL/Analysis/Continuous_Extension.thy Tue Oct 17 13:56:58 2017 +0200 +++ b/src/HOL/Analysis/Continuous_Extension.thy Thu Oct 19 17:16:01 2017 +0100 @@ -281,10 +281,7 @@ "\x. f x \ closed_segment a b" "\x. f x = a \ x \ S" "\x. f x = b \ x \ T" -apply (rule Urysohn_local_strong [of UNIV S T]) -using assms -apply (auto simp: closed_closedin) -done +using assms by (auto intro: Urysohn_local_strong [of UNIV S T]) proposition Urysohn: assumes US: "closed S" @@ -295,10 +292,7 @@ "\x. f x \ closed_segment a b" "\x. x \ S \ f x = a" "\x. x \ T \ f x = b" -apply (rule Urysohn_local [of UNIV S T a b]) -using assms -apply (auto simp: closed_closedin) -done +using assms by (auto intro: Urysohn_local [of UNIV S T a b]) subsection\ The Dugundji extension theorem, and Tietze variants as corollaries.\