src/HOL/Analysis/Weierstrass_Theorems.thy
changeset 69508 2a4c8a2a3f8e
parent 69260 0a9688695a1b
child 69517 dc20f278e8f3
--- a/src/HOL/Analysis/Weierstrass_Theorems.thy	Wed Dec 26 20:57:23 2018 +0100
+++ b/src/HOL/Analysis/Weierstrass_Theorems.thy	Thu Dec 27 19:48:28 2018 +0100
@@ -767,7 +767,7 @@
   assumes "compact S"  "\<And>c. P(\<lambda>x. c::real)"
           "\<And>f. P f \<Longrightarrow> continuous_on S f"
           "\<And>f g. P(f) \<and> P(g) \<Longrightarrow> P(\<lambda>x. f x + g x)"  "\<And>f g. P(f) \<and> P(g) \<Longrightarrow> P(\<lambda>x. f x * g x)"
-          "\<And>x y. x \<in> S \<and> y \<in> S \<and> ~(x = y) \<Longrightarrow> \<exists>f. P(f) \<and> ~(f x = f y)"
+          "\<And>x y. x \<in> S \<and> y \<in> S \<and> x \<noteq> y \<Longrightarrow> \<exists>f. P(f) \<and> f x \<noteq> f y"
           "continuous_on S f"
        "0 < e"
     shows "\<exists>g. P(g) \<and> (\<forall>x \<in> S. \<bar>f x - g x\<bar> < e)"