src/HOLCF/Fix.thy
changeset 40004 9f6ed6840e8d
parent 36452 d37c6eed8117
child 40321 d065b195ec89
--- a/src/HOLCF/Fix.thy	Tue Oct 12 05:25:21 2010 -0700
+++ b/src/HOLCF/Fix.thy	Tue Oct 12 05:48:15 2010 -0700
@@ -60,13 +60,7 @@
 text {* direct connection between @{term fix} and iteration *}
 
 lemma fix_def2: "fix\<cdot>F = (\<Squnion>i. iterate i\<cdot>F\<cdot>\<bottom>)"
-apply (unfold fix_def)
-apply (rule beta_cfun)
-apply (rule cont2cont_lub)
-apply (rule ch2ch_lambda)
-apply (rule chain_iterate)
-apply simp
-done
+unfolding fix_def by simp
 
 lemma iterate_below_fix: "iterate n\<cdot>f\<cdot>\<bottom> \<sqsubseteq> fix\<cdot>f"
   unfolding fix_def2