src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy
changeset 69508 2a4c8a2a3f8e
parent 69325 4b6ddc5989fc
child 69597 ff784d5a5bfb
--- a/src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy	Wed Dec 26 20:57:23 2018 +0100
+++ b/src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy	Thu Dec 27 19:48:28 2018 +0100
@@ -1195,8 +1195,8 @@
   proof (rule starlike_negligible [OF \<open>closed S\<close>, of a])
     fix c x
     assume cx: "a + c *\<^sub>R x \<in> S" "0 \<le> c" "a + x \<in> S"
-    with star have "~ (c < 1)" by auto
-    moreover have "~ (c > 1)"
+    with star have "\<not> (c < 1)" by auto
+    moreover have "\<not> (c > 1)"
       using star [of "1/c" "c *\<^sub>R x"] cx by force
     ultimately show "c = 1" by arith
   qed