more automation
authornipkow
Thu, 18 Jan 2018 08:08:36 +0100
changeset 67453 afefc45ed4e9
parent 67452 aab817885622
child 67454 867d7e91af65
more automation
src/HOL/Topological_Spaces.thy
--- a/src/HOL/Topological_Spaces.thy	Wed Jan 17 12:27:06 2018 +0100
+++ b/src/HOL/Topological_Spaces.thy	Thu Jan 18 08:08:36 2018 +0100
@@ -760,7 +760,7 @@
     and "y < a \<Longrightarrow> eventually (\<lambda>x. f x < a) F"
   using assms by (auto simp: order_tendsto_iff)
 
-lemma (in linorder_topology) tendsto_max:
+lemma (in linorder_topology) tendsto_max[tendsto_intros]:
   assumes X: "(X \<longlongrightarrow> x) net"
     and Y: "(Y \<longlongrightarrow> y) net"
   shows "((\<lambda>x. max (X x) (Y x)) \<longlongrightarrow> max x y) net"
@@ -778,7 +778,7 @@
     by (auto simp: eventually_conj_iff)
 qed
 
-lemma (in linorder_topology) tendsto_min:
+lemma (in linorder_topology) tendsto_min[tendsto_intros]:
   assumes X: "(X \<longlongrightarrow> x) net"
     and Y: "(Y \<longlongrightarrow> y) net"
   shows "((\<lambda>x. min (X x) (Y x)) \<longlongrightarrow> min x y) net"