src/HOL/Library/Multiset.thy
changeset 73052 c03a148110cc
parent 73047 ab9e27da0e85
child 73270 e2d03448d5b5
equal deleted inserted replaced
73051:6ba08ec184a1 73052:c03a148110cc
  2468   shows "x dvd prod_mset A"
  2468   shows "x dvd prod_mset A"
  2469   using assms prod_mset_subset_imp_dvd [of "{#x#}" A] by simp
  2469   using assms prod_mset_subset_imp_dvd [of "{#x#}" A] by simp
  2470 
  2470 
  2471 end
  2471 end
  2472 
  2472 
       
  2473 notation prod_mset ("\<Prod>\<^sub>#")
       
  2474 
  2473 syntax (ASCII)
  2475 syntax (ASCII)
  2474   "_prod_mset_image" :: "pttrn \<Rightarrow> 'b set \<Rightarrow> 'a \<Rightarrow> 'a::comm_monoid_mult"  ("(3PROD _:#_. _)" [0, 51, 10] 10)
  2476   "_prod_mset_image" :: "pttrn \<Rightarrow> 'b set \<Rightarrow> 'a \<Rightarrow> 'a::comm_monoid_mult"  ("(3PROD _:#_. _)" [0, 51, 10] 10)
  2475 syntax
  2477 syntax
  2476   "_prod_mset_image" :: "pttrn \<Rightarrow> 'b set \<Rightarrow> 'a \<Rightarrow> 'a::comm_monoid_mult"  ("(3\<Prod>_\<in>#_. _)" [0, 51, 10] 10)
  2478   "_prod_mset_image" :: "pttrn \<Rightarrow> 'b set \<Rightarrow> 'a \<Rightarrow> 'a::comm_monoid_mult"  ("(3\<Prod>_\<in>#_. _)" [0, 51, 10] 10)
  2477 translations
  2479 translations