src/HOLCF/Bifinite.thy
changeset 35525 fa231b86cb1e
parent 33808 31169fdc5ae7
child 37678 0040bafffdef
--- a/src/HOLCF/Bifinite.thy	Tue Mar 02 17:20:03 2010 -0800
+++ b/src/HOLCF/Bifinite.thy	Tue Mar 02 17:21:10 2010 -0800
@@ -295,7 +295,7 @@
     by (rule finite_range_imp_finite_fixes)
 qed
 
-instantiation "->" :: (profinite, profinite) profinite
+instantiation cfun :: (profinite, profinite) profinite
 begin
 
 definition
@@ -325,7 +325,7 @@
 
 end
 
-instance "->" :: (profinite, bifinite) bifinite ..
+instance cfun :: (profinite, bifinite) bifinite ..
 
 lemma approx_cfun: "approx n\<cdot>f\<cdot>x = approx n\<cdot>(f\<cdot>(approx n\<cdot>x))"
 by (simp add: approx_cfun_def)