src/HOL/Analysis/Operator_Norm.thy
changeset 70136 f03a01a18c6e
parent 69607 7cd977863194
--- a/src/HOL/Analysis/Operator_Norm.thy	Fri Apr 12 19:48:29 2019 +0200
+++ b/src/HOL/Analysis/Operator_Norm.thy	Fri Apr 12 22:09:25 2019 +0200
@@ -11,8 +11,8 @@
 
 text \<open>This formulation yields zero if \<open>'a\<close> is the trivial vector space.\<close>
 
-text%important \<open>%whitespace\<close>
-definition%important
+text\<^marker>\<open>tag important\<close> \<open>%whitespace\<close>
+definition\<^marker>\<open>tag important\<close>
 onorm :: "('a::real_normed_vector \<Rightarrow> 'b::real_normed_vector) \<Rightarrow> real" where
 "onorm f = (SUP x. norm (f x) / norm x)"