src/HOL/Analysis/Uniform_Limit.thy
changeset 70136 f03a01a18c6e
parent 69597 ff784d5a5bfb
child 70817 dd675800469d
--- a/src/HOL/Analysis/Uniform_Limit.thy	Fri Apr 12 19:48:29 2019 +0200
+++ b/src/HOL/Analysis/Uniform_Limit.thy	Fri Apr 12 22:09:25 2019 +0200
@@ -12,10 +12,10 @@
 
 subsection \<open>Definition\<close>
 
-definition%important uniformly_on :: "'a set \<Rightarrow> ('a \<Rightarrow> 'b::metric_space) \<Rightarrow> ('a \<Rightarrow> 'b) filter"
+definition\<^marker>\<open>tag important\<close> uniformly_on :: "'a set \<Rightarrow> ('a \<Rightarrow> 'b::metric_space) \<Rightarrow> ('a \<Rightarrow> 'b) filter"
   where "uniformly_on S l = (INF e\<in>{0 <..}. principal {f. \<forall>x\<in>S. dist (f x) (l x) < e})"
 
-abbreviation%important
+abbreviation\<^marker>\<open>tag important\<close>
   "uniform_limit S f l \<equiv> filterlim f (uniformly_on S l)"
 
 definition uniformly_convergent_on where
@@ -366,7 +366,7 @@
 qed
 
 text\<open>Alternative version, formulated as in HOL Light\<close>
-corollary%unimportant series_comparison_uniform:
+corollary\<^marker>\<open>tag unimportant\<close> series_comparison_uniform:
   fixes f :: "_ \<Rightarrow> nat \<Rightarrow> _ :: banach"
   assumes g: "summable g" and le: "\<And>n x. N \<le> n \<and> x \<in> A \<Longrightarrow> norm(f x n) \<le> g n"
     shows "\<exists>l. \<forall>e. 0 < e \<longrightarrow> (\<exists>N. \<forall>n x. N \<le> n \<and> x \<in> A \<longrightarrow> dist(sum (f x) {..<n}) (l x) < e)"
@@ -379,20 +379,20 @@
     done
 qed
 
-corollary%unimportant Weierstrass_m_test:
+corollary\<^marker>\<open>tag unimportant\<close> Weierstrass_m_test:
   fixes f :: "_ \<Rightarrow> _ \<Rightarrow> _ :: banach"
   assumes "\<And>n x. x \<in> A \<Longrightarrow> norm (f n x) \<le> M n"
   assumes "summable M"
   shows "uniform_limit A (\<lambda>n x. \<Sum>i<n. f i x) (\<lambda>x. suminf (\<lambda>i. f i x)) sequentially"
   using assms by (intro Weierstrass_m_test_ev always_eventually) auto
 
-corollary%unimportant Weierstrass_m_test'_ev:
+corollary\<^marker>\<open>tag unimportant\<close> Weierstrass_m_test'_ev:
   fixes f :: "_ \<Rightarrow> _ \<Rightarrow> _ :: banach"
   assumes "eventually (\<lambda>n. \<forall>x\<in>A. norm (f n x) \<le> M n) sequentially" "summable M"
   shows   "uniformly_convergent_on A (\<lambda>n x. \<Sum>i<n. f i x)"
   unfolding uniformly_convergent_on_def by (rule exI, rule Weierstrass_m_test_ev[OF assms])
 
-corollary%unimportant Weierstrass_m_test':
+corollary\<^marker>\<open>tag unimportant\<close> Weierstrass_m_test':
   fixes f :: "_ \<Rightarrow> _ \<Rightarrow> _ :: banach"
   assumes "\<And>n x. x \<in> A \<Longrightarrow> norm (f n x) \<le> M n" "summable M"
   shows   "uniformly_convergent_on A (\<lambda>n x. \<Sum>i<n. f i x)"
@@ -402,7 +402,7 @@
   by simp
 
 
-subsection%unimportant \<open>Structural introduction rules\<close>
+subsection\<^marker>\<open>tag unimportant\<close> \<open>Structural introduction rules\<close>
 
 named_theorems uniform_limit_intros "introduction rules for uniform_limit"
 setup \<open>