src/HOLCF/Cfun.thy
changeset 19709 78cd5f6af8e8
parent 18092 2c5d5da79a1e
child 23152 9497234a2743
equal deleted inserted replaced
19708:a508bde37a81 19709:78cd5f6af8e8
   453 lemma cfcomp1: "(f oo g) = (\<Lambda> x. f\<cdot>(g\<cdot>x))"
   453 lemma cfcomp1: "(f oo g) = (\<Lambda> x. f\<cdot>(g\<cdot>x))"
   454 by (simp add: oo_def)
   454 by (simp add: oo_def)
   455 
   455 
   456 lemma cfcomp2 [simp]: "(f oo g)\<cdot>x = f\<cdot>(g\<cdot>x)"
   456 lemma cfcomp2 [simp]: "(f oo g)\<cdot>x = f\<cdot>(g\<cdot>x)"
   457 by (simp add: cfcomp1)
   457 by (simp add: cfcomp1)
       
   458 
       
   459 lemma cfcomp_strict [simp]: "\<bottom> oo f = \<bottom>"
       
   460 by (simp add: expand_cfun_eq)
   458 
   461 
   459 text {*
   462 text {*
   460   Show that interpretation of (pcpo,@{text "_->_"}) is a category.
   463   Show that interpretation of (pcpo,@{text "_->_"}) is a category.
   461   The class of objects is interpretation of syntactical class pcpo.
   464   The class of objects is interpretation of syntactical class pcpo.
   462   The class of arrows  between objects @{typ 'a} and @{typ 'b} is interpret. of @{typ "'a -> 'b"}.
   465   The class of arrows  between objects @{typ 'a} and @{typ 'b} is interpret. of @{typ "'a -> 'b"}.