merged
authorwenzelm
Tue, 12 Mar 2024 15:31:44 +0100
changeset 79872 85ff8d62c414
parent 79865 53d0d2860ed8 (diff)
parent 79871 630a82f87310 (current diff)
child 79873 6c19c29ddcbe
merged
--- a/src/HOL/Complex_Analysis/Meromorphic.thy	Tue Mar 12 15:30:32 2024 +0100
+++ b/src/HOL/Complex_Analysis/Meromorphic.thy	Tue Mar 12 15:31:44 2024 +0100
@@ -59,7 +59,7 @@
   shows   "(\<lambda>y. \<Prod>x\<in>#I. f x y) has_laurent_expansion (\<Prod>x\<in>#I. F x)"
   using assms by (induction I) (auto intro!: laurent_expansion_intros)
 
-subsection \<open>Remove singular points: remove_sings\<close>
+subsection \<open>Remove singular points\<close>
 
 definition remove_sings :: "(complex \<Rightarrow> complex) \<Rightarrow> complex \<Rightarrow> complex" where
   "remove_sings f z = (if \<exists>c. f \<midarrow>z\<rightarrow> c then Lim (at z) f else 0)"