src/HOLCF/Deflation.thy
changeset 27681 8cedebf55539
parent 27401 4edc81f93e35
child 28611 983c1855a7af
equal deleted inserted replaced
27680:5a557a5afc48 27681:8cedebf55539
   321   apply (rule monofun_cfun_arg)
   321   apply (rule monofun_cfun_arg)
   322   apply (erule ep_pair.e_p_less)
   322   apply (erule ep_pair.e_p_less)
   323  apply (erule ep_pair.e_p_less)
   323  apply (erule ep_pair.e_p_less)
   324 done
   324 done
   325 
   325 
   326 locale (open) pcpo_ep_pair = ep_pair +
   326 locale pcpo_ep_pair = ep_pair +
   327   constrains e :: "'a::pcpo \<rightarrow> 'b::pcpo"
   327   constrains e :: "'a::pcpo \<rightarrow> 'b::pcpo"
   328   constrains p :: "'b::pcpo \<rightarrow> 'a::pcpo"
   328   constrains p :: "'b::pcpo \<rightarrow> 'a::pcpo"
   329 begin
   329 begin
   330 
   330 
   331 lemma e_strict [simp]: "e\<cdot>\<bottom> = \<bottom>"
   331 lemma e_strict [simp]: "e\<cdot>\<bottom> = \<bottom>"