src/HOLCF/Library/Stream.thy
changeset 40002 c5b5f7a3a3b1
parent 37110 7ffdbc24b27f
child 40025 876689e6bbdf
--- a/src/HOLCF/Library/Stream.thy	Mon Oct 11 16:24:44 2010 -0700
+++ b/src/HOLCF/Library/Stream.thy	Mon Oct 11 21:35:31 2010 -0700
@@ -508,7 +508,7 @@
 by (insert sfilter_def [where 'a='a, THEN eq_reflection, THEN fix_eq2], auto)
 
 lemma strict_sfilter: "sfilter\<cdot>\<bottom> = \<bottom>"
-apply (rule ext_cfun)
+apply (rule cfun_eqI)
 apply (subst sfilter_unfold, auto)
 apply (case_tac "x=UU", auto)
 by (drule stream_exhaust_eq [THEN iffD1], auto)