src/HOL/Algebra/Divisibility.thy
changeset 63793 e68a0b651eb5
parent 63633 2accfb71e33b
child 63832 a400b127853c
equal deleted inserted replaced
63792:4ccb7e635477 63793:e68a0b651eb5
  2049         and a: "a = assocs G c"
  2049         and a: "a = assocs G c"
  2050         by auto
  2050         by auto
  2051     from cP csP
  2051     from cP csP
  2052         have tP: "\<forall>x\<in>set (c#cs). P x" by simp
  2052         have tP: "\<forall>x\<in>set (c#cs). P x" by simp
  2053     from mset a
  2053     from mset a
  2054     have "mset (map (assocs G) (c#cs)) = mset Cs' + {#a#}" by simp
  2054     have "mset (map (assocs G) (c#cs)) = add_mset a (mset Cs')" by simp
  2055     from tP this
  2055     from tP this
  2056     show "\<exists>cs. (\<forall>x\<in>set cs. P x) \<and>
  2056     show "\<exists>cs. (\<forall>x\<in>set cs. P x) \<and>
  2057                mset (map (assocs G) cs) =
  2057                mset (map (assocs G) cs) =
  2058                mset Cs' + {#a#}" by fast
  2058                add_mset a (mset Cs')" by fast
  2059   qed
  2059   qed
  2060   thus ?thesis by (simp add: fmset_def)
  2060   thus ?thesis by (simp add: fmset_def)
  2061 qed
  2061 qed
  2062 
  2062 
  2063 lemma (in monoid) mset_wfactorsEx:
  2063 lemma (in monoid) mset_wfactorsEx: