add type annotation to avoid warning
authorhuffman
Thu, 14 Oct 2010 09:28:05 -0700
changeset 40012 f13341a45407
parent 40011 b974cf829099
child 40013 9db8fb58fddc
add type annotation to avoid warning
src/HOLCF/Bifinite.thy
--- a/src/HOLCF/Bifinite.thy	Wed Oct 13 10:56:42 2010 -0700
+++ b/src/HOLCF/Bifinite.thy	Thu Oct 14 09:28:05 2010 -0700
@@ -440,7 +440,7 @@
 
 lemma finite_deflation_lift_approx: "finite_deflation (lift_approx i)"
 proof
-  fix x
+  fix x :: "'a lift"
   show "lift_approx i\<cdot>x \<sqsubseteq> x"
     unfolding lift_approx_def
     by (cases x, simp, simp)