src/HOL/Analysis/Riemann_Mapping.thy
changeset 67968 a5ad4c015d1c
parent 67685 bdff8bf0a75b
child 68634 db0980691ef4
--- a/src/HOL/Analysis/Riemann_Mapping.thy	Sun Apr 08 12:31:08 2018 +0200
+++ b/src/HOL/Analysis/Riemann_Mapping.thy	Mon Apr 09 16:20:23 2018 +0200
@@ -8,7 +8,7 @@
 imports Great_Picard
 begin
 
-subsection\<open>Moebius functions are biholomorphisms of the unit disc.\<close>
+subsection\<open>Moebius functions are biholomorphisms of the unit disc\<close>
 
 definition Moebius_function :: "[real,complex,complex] \<Rightarrow> complex" where
   "Moebius_function \<equiv> \<lambda>t w z. exp(\<i> * of_real t) * (z - w) / (1 - cnj w * z)"
@@ -853,7 +853,7 @@
   using convex_imp_contractible homeomorphic_contractible_eq simply_connected_eq_homeomorphic_to_disc by auto
 
 
-subsection\<open>A further chain of equivalences about components of the complement of a simply connected set.\<close>
+subsection\<open>A further chain of equivalences about components of the complement of a simply connected set\<close>
 
 text\<open>(following 1.35 in Burckel'S book)\<close>