src/HOL/Analysis/Derivative.thy
changeset 69553 2c2e2b3e19b7
parent 69529 4ab9657b3257
child 69597 ff784d5a5bfb
--- a/src/HOL/Analysis/Derivative.thy	Sun Dec 30 17:44:33 2018 +0100
+++ b/src/HOL/Analysis/Derivative.thy	Mon Dec 31 12:25:21 2018 +0100
@@ -2193,7 +2193,7 @@
   using assms(2-3) vector_derivative_works
   by auto
 
-subsection\<open>The notion of being field differentiable\<close>
+subsection \<open>Field differentiability\<close>
 
 definition%important field_differentiable :: "['a \<Rightarrow> 'a::real_normed_field, 'a filter] \<Rightarrow> bool"
            (infixr "(field'_differentiable)" 50)