src/HOL/Deriv.thy
changeset 76033 97b6daab0233
parent 75462 7448423e5dba
child 77138 c8597292cd41
--- a/src/HOL/Deriv.thy	Wed Aug 31 23:00:43 2022 +0200
+++ b/src/HOL/Deriv.thy	Wed Aug 31 23:05:12 2022 +0200
@@ -811,7 +811,7 @@
 lemma DERIV_def: "DERIV f x :> D \<longleftrightarrow> (\<lambda>h. (f (x + h) - f x) / h) \<midarrow>0\<rightarrow> D"
   unfolding field_has_derivative_at has_field_derivative_def has_field_derivative_iff ..
 
-text \<open>due to Christian Pardillo Laursen, replacing a proper epsilon-delta horror\<close>
+text \<open>due to Christian Pardillo Laursen, replacing a proper epsilon-delta horror\<close>
 lemma field_derivative_lim_unique:
   assumes f: "(f has_field_derivative df) (at z)"
     and s: "s \<longlonglongrightarrow> 0"  "\<And>n. s n \<noteq> 0"