src/HOLCF/Cfun.thy
changeset 15641 b389f108c485
parent 15600 a59f07556a8d
child 16055 58186c507750
--- a/src/HOLCF/Cfun.thy	Thu Mar 31 03:01:21 2005 +0200
+++ b/src/HOLCF/Cfun.thy	Thu Mar 31 03:03:22 2005 +0200
@@ -70,6 +70,11 @@
 lemma beta_cfun: "cont(c1) ==> (LAM x .c1 x)$u = c1 u"
 by (rule Cfunapp2)
 
+text {* Eta - equality for continuous functions *}
+
+lemma eta_cfun: "(LAM x. f$x) = f"
+by (rule Rep_CFun_inverse)
+
 subsection {* Type @{typ "'a -> 'b"} is a partial order *}
 
 instance "->"  :: (cpo, cpo) sq_ord ..
@@ -424,6 +429,11 @@
 apply (erule p2 [THEN cont2contlub, THEN contlubE, THEN spec, THEN mp])
 done
 
+text {* cont2cont Lemma for @{term "%x. LAM y. c1 x$y"} *}
+
+lemma cont2cont_eta: "cont c1 ==> cont (%x. LAM y. c1 x$y)"
+by (simp only: eta_cfun)
+
 text {* cont2cont tactic *}
 
 lemmas cont_lemmas1 = cont_const cont_id cont_Rep_CFun2