lemma deflation_strict
authorhuffman
Thu, 05 Nov 2009 11:36:30 -0800
changeset 33503 3496616b2171
parent 33439 f5d95787224f
child 33504 b4210cc3ac97
lemma deflation_strict
src/HOLCF/Deflation.thy
--- a/src/HOLCF/Deflation.thy	Thu Nov 05 14:37:39 2009 +0100
+++ b/src/HOLCF/Deflation.thy	Thu Nov 05 11:36:30 2009 -0800
@@ -55,6 +55,9 @@
 
 end
 
+lemma deflation_strict: "deflation d \<Longrightarrow> d\<cdot>\<bottom> = \<bottom>"
+by (rule deflation.below [THEN UU_I])
+
 lemma adm_deflation: "adm (\<lambda>d. deflation d)"
 by (simp add: deflation_def)