add type annotation to avoid warning
authorhuffman
Thu, 21 Oct 2010 15:19:07 -0700
changeset 40085 c157ff4d59a6
parent 40084 23a1cfdb5acb
child 40086 c339c0e8fdfb
add type annotation to avoid warning
src/HOLCF/Up.thy
--- a/src/HOLCF/Up.thy	Thu Oct 21 12:51:36 2010 -0700
+++ b/src/HOLCF/Up.thy	Thu Oct 21 15:19:07 2010 -0700
@@ -120,7 +120,8 @@
       by (simp add: lub_const)
     thus ?thesis ..
   next
-    fix A assume "range S <<| Iup (\<Squnion>i. A i)"
+    fix A :: "nat \<Rightarrow> 'a"
+    assume "range S <<| Iup (\<Squnion>i. A i)"
     thus ?thesis ..
   qed
 qed