add simp rule LAM_strict
authorhuffman
Sun, 07 Mar 2010 16:12:01 -0800
changeset 35641 a17bc4cec23a
parent 35640 9617aeca7147
child 35642 f478d5a9d238
add simp rule LAM_strict
src/HOLCF/Cfun.thy
--- a/src/HOLCF/Cfun.thy	Sun Mar 07 13:34:53 2010 -0800
+++ b/src/HOLCF/Cfun.thy	Sun Mar 07 16:12:01 2010 -0800
@@ -126,9 +126,12 @@
 lemma Rep_CFun_strict1 [simp]: "\<bottom>\<cdot>x = \<bottom>"
 by (simp add: Rep_CFun_strict)
 
+lemma LAM_strict [simp]: "(\<Lambda> x. \<bottom>) = \<bottom>"
+by (simp add: inst_fun_pcpo [symmetric] Abs_CFun_strict)
+
 text {* for compatibility with old HOLCF-Version *}
 lemma inst_cfun_pcpo: "\<bottom> = (\<Lambda> x. \<bottom>)"
-by (simp add: inst_fun_pcpo [symmetric] Abs_CFun_strict)
+by simp
 
 subsection {* Basic properties of continuous functions *}