src/HOL/HOLCF/Library/List_Predomain.thy
changeset 41323 ae1c227534f5
parent 41321 4e72b6fc9dd4
child 41437 5bc117c382ec
equal deleted inserted replaced
41322:43a5b9a0ee8a 41323:ae1c227534f5
   137 
   137 
   138 abbreviation list_map :: "('a::cpo \<rightarrow> 'b::cpo) \<Rightarrow> 'a list \<rightarrow> 'b list"
   138 abbreviation list_map :: "('a::cpo \<rightarrow> 'b::cpo) \<Rightarrow> 'a list \<rightarrow> 'b list"
   139   where "list_map f \<equiv> Abs_cfun (map (Rep_cfun f))"
   139   where "list_map f \<equiv> Abs_cfun (map (Rep_cfun f))"
   140 
   140 
   141 lemma list_map_ID [domain_map_ID]: "list_map ID = ID"
   141 lemma list_map_ID [domain_map_ID]: "list_map ID = ID"
   142 by (simp add: ID_def cfun_eq_iff Abs_cfun_inverse2)
   142 by (simp add: ID_def)
   143 
   143 
   144 lemma deflation_list_map [domain_deflation]:
   144 lemma deflation_list_map [domain_deflation]:
   145   "deflation d \<Longrightarrow> deflation (list_map d)"
   145   "deflation d \<Longrightarrow> deflation (list_map d)"
   146 apply default
   146 apply default
   147 apply (induct_tac x, simp_all add: deflation.idem)
   147 apply (induct_tac x, simp_all add: deflation.idem)