src/HOLCF/ConvexPD.thy
changeset 40577 5c6225a1c2c0
parent 40576 fa5e0cacd5e7
child 40589 0e77e45d2ffc
equal deleted inserted replaced
40576:fa5e0cacd5e7 40577:5c6225a1c2c0
   373 
   373 
   374 lemma convex_map_plus [simp]:
   374 lemma convex_map_plus [simp]:
   375   "convex_map\<cdot>f\<cdot>(xs +\<natural> ys) = convex_map\<cdot>f\<cdot>xs +\<natural> convex_map\<cdot>f\<cdot>ys"
   375   "convex_map\<cdot>f\<cdot>(xs +\<natural> ys) = convex_map\<cdot>f\<cdot>xs +\<natural> convex_map\<cdot>f\<cdot>ys"
   376 unfolding convex_map_def by simp
   376 unfolding convex_map_def by simp
   377 
   377 
       
   378 lemma convex_map_bottom [simp]: "convex_map\<cdot>f\<cdot>\<bottom> = {f\<cdot>\<bottom>}\<natural>"
       
   379 unfolding convex_map_def by simp
       
   380 
   378 lemma convex_map_ident: "convex_map\<cdot>(\<Lambda> x. x)\<cdot>xs = xs"
   381 lemma convex_map_ident: "convex_map\<cdot>(\<Lambda> x. x)\<cdot>xs = xs"
   379 by (induct xs rule: convex_pd_induct, simp_all)
   382 by (induct xs rule: convex_pd_induct, simp_all)
   380 
   383 
   381 lemma convex_map_ID: "convex_map\<cdot>ID = ID"
   384 lemma convex_map_ID: "convex_map\<cdot>ID = ID"
   382 by (simp add: cfun_eq_iff ID_def convex_map_ident)
   385 by (simp add: cfun_eq_iff ID_def convex_map_ident)
   515 
   518 
   516 lemma convex_join_plus [simp]:
   519 lemma convex_join_plus [simp]:
   517   "convex_join\<cdot>(xss +\<natural> yss) = convex_join\<cdot>xss +\<natural> convex_join\<cdot>yss"
   520   "convex_join\<cdot>(xss +\<natural> yss) = convex_join\<cdot>xss +\<natural> convex_join\<cdot>yss"
   518 unfolding convex_join_def by simp
   521 unfolding convex_join_def by simp
   519 
   522 
       
   523 lemma convex_join_bottom [simp]: "convex_join\<cdot>\<bottom> = \<bottom>"
       
   524 unfolding convex_join_def by simp
       
   525 
   520 lemma convex_join_map_unit:
   526 lemma convex_join_map_unit:
   521   "convex_join\<cdot>(convex_map\<cdot>convex_unit\<cdot>xs) = xs"
   527   "convex_join\<cdot>(convex_map\<cdot>convex_unit\<cdot>xs) = xs"
   522 by (induct xs rule: convex_pd_induct, simp_all)
   528 by (induct xs rule: convex_pd_induct, simp_all)
   523 
   529 
   524 lemma convex_join_map_join:
   530 lemma convex_join_map_join: