src/HOL/Analysis/Riemann_Mapping.thy
changeset 70136 f03a01a18c6e
parent 69922 4a9167f377b0
child 70365 4df0628e8545
--- a/src/HOL/Analysis/Riemann_Mapping.thy	Fri Apr 12 19:48:29 2019 +0200
+++ b/src/HOL/Analysis/Riemann_Mapping.thy	Fri Apr 12 22:09:25 2019 +0200
@@ -10,7 +10,7 @@
 
 subsection\<open>Moebius functions are biholomorphisms of the unit disc\<close>
 
-definition%important Moebius_function :: "[real,complex,complex] \<Rightarrow> complex" where
+definition\<^marker>\<open>tag important\<close> 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)"
 
 lemma Moebius_function_simple:
@@ -1411,7 +1411,7 @@
 qed
 
 
-subsection%unimportant \<open>More Borsukian results\<close>
+subsection\<^marker>\<open>tag unimportant\<close> \<open>More Borsukian results\<close>
 
 lemma Borsukian_componentwise_eq:
   fixes S :: "'a::euclidean_space set"