src/HOL/HOLCF/Library/Option_Cpo.thy
changeset 41393 17bf4ddd0833
parent 41325 b27e5c9f5c10
child 41436 480978f80eae
equal deleted inserted replaced
41392:d1ff42a70f77 41393:17bf4ddd0833
   263 
   263 
   264 abbreviation option_map
   264 abbreviation option_map
   265   where "option_map f \<equiv> Abs_cfun (Option.map (Rep_cfun f))"
   265   where "option_map f \<equiv> Abs_cfun (Option.map (Rep_cfun f))"
   266 
   266 
   267 lemma option_map_ID [domain_map_ID]: "option_map ID = ID"
   267 lemma option_map_ID [domain_map_ID]: "option_map ID = ID"
   268 by (simp add: ID_def cfun_eq_iff Option.map.identity)
   268 by (simp add: ID_def cfun_eq_iff Option.map.identity id_def)
   269 
   269 
   270 lemma deflation_option_map [domain_deflation]:
   270 lemma deflation_option_map [domain_deflation]:
   271   "deflation d \<Longrightarrow> deflation (option_map d)"
   271   "deflation d \<Longrightarrow> deflation (option_map d)"
   272 apply default
   272 apply default
   273 apply (induct_tac x, simp_all add: deflation.idem)
   273 apply (induct_tac x, simp_all add: deflation.idem)