add required type annotation
authorhuffman
Sat, 16 Sep 2006 02:32:48 +0200
changeset 20550 5a925ad63f4d
parent 20549 c643984eb94b
child 20551 ba543692bfa1
add required type annotation
src/HOL/Complex/ex/BigO_Complex.thy
--- a/src/HOL/Complex/ex/BigO_Complex.thy	Fri Sep 15 22:56:17 2006 +0200
+++ b/src/HOL/Complex/ex/BigO_Complex.thy	Sat Sep 16 02:32:48 2006 +0200
@@ -13,7 +13,7 @@
   Additional lemmas that require the \texttt{HOL-Complex} logic image.
 *}
 
-lemma bigo_LIMSEQ1: "f =o O(g) ==> g ----> 0 ==> f ----> 0"
+lemma bigo_LIMSEQ1: "f =o O(g) ==> g ----> 0 ==> f ----> (0::real)"
   apply (simp add: LIMSEQ_def bigo_alt_def)
   apply clarify
   apply (drule_tac x = "r / c" in spec)
@@ -38,7 +38,7 @@
 done
 
 lemma bigo_LIMSEQ2: "f =o g +o O(h) ==> h ----> 0 ==> f ----> a 
-    ==> g ----> a"
+    ==> g ----> (a::real)"
   apply (drule set_plus_imp_minus)
   apply (drule bigo_LIMSEQ1)
   apply assumption