src/HOL/Library/While_Combinator.thy
changeset 50180 c6626861c31a
parent 50008 eb7f574d0303
child 50577 cfbad2d08412
--- a/src/HOL/Library/While_Combinator.thy	Fri Nov 23 18:28:00 2012 +0100
+++ b/src/HOL/Library/While_Combinator.thy	Fri Nov 23 23:07:38 2012 +0100
@@ -169,4 +169,9 @@
   show ?thesis by auto
 qed
 
+lemma lfp_while:
+  assumes "mono f" and "!!X. X \<subseteq> C \<Longrightarrow> f X \<subseteq> C" and "finite C"
+  shows "lfp f = while (\<lambda>A. f A \<noteq> A) f {}"
+unfolding while_def using assms by (rule lfp_the_while_option) blast
+
 end