src/HOL/NSA/HSEQ.thy
changeset 51474 1e9e68247ad1
parent 44568 e6f291cb5810
child 51525 d3d170a2887f
--- a/src/HOL/NSA/HSEQ.thy	Fri Mar 22 10:41:43 2013 +0100
+++ b/src/HOL/NSA/HSEQ.thy	Fri Mar 22 10:41:43 2013 +0100
@@ -343,7 +343,7 @@
 text{*Standard Version: easily now proved using equivalence of NS and
  standard definitions *}
 
-lemma convergent_Bseq: "convergent X ==> Bseq X"
+lemma convergent_Bseq: "convergent X ==> Bseq (X::nat \<Rightarrow> _::real_normed_vector)"
 by (simp add: NSconvergent_NSBseq convergent_NSconvergent_iff Bseq_NSBseq_iff)
 
 subsubsection{*Upper Bounds and Lubs of Bounded Sequences*}