src/HOL/Library/Multiset.thy
changeset 40968 a6fcd305f7dc
parent 40950 a370b0fb6f09
child 41069 6fabc0414055
equal deleted inserted replaced
40965:54b6c9e1c157 40968:a6fcd305f7dc
  1629   but also images like @{term "{#x+x. x:#M #}"} and @{term [source]
  1629   but also images like @{term "{#x+x. x:#M #}"} and @{term [source]
  1630   "{#x+x|x:#M. x<c#}"}, where the latter is currently displayed as
  1630   "{#x+x|x:#M. x<c#}"}, where the latter is currently displayed as
  1631   @{term "{#x+x|x:#M. x<c#}"}.
  1631   @{term "{#x+x|x:#M. x<c#}"}.
  1632 *}
  1632 *}
  1633 
  1633 
  1634 type_mapper image_mset proof -
  1634 type_lifting image_mset proof -
  1635   fix f g A show "image_mset f (image_mset g A) = image_mset (\<lambda>x. f (g x)) A"
  1635   fix f g A show "image_mset f (image_mset g A) = image_mset (\<lambda>x. f (g x)) A"
  1636     by (induct A) simp_all
  1636     by (induct A) simp_all
  1637 next
  1637 next
  1638   fix A show "image_mset (\<lambda>x. x) A = A"
  1638   fix A show "image_mset (\<lambda>x. x) A = A"
  1639     by (induct A) simp_all
  1639     by (induct A) simp_all