src/HOL/Algebra/Divisibility.thy
changeset 68604 57721285d4ef
parent 68551 b680e74eb6f2
child 68664 bd0df72c16d5
--- a/src/HOL/Algebra/Divisibility.thy	Sun Jul 08 11:00:20 2018 +0100
+++ b/src/HOL/Algebra/Divisibility.thy	Sun Jul 08 16:07:26 2018 +0100
@@ -1654,8 +1654,10 @@
     by (clarsimp simp add: map_eq_Cons_conv) blast
 next
   case (trans xs ys zs)
+  then obtain as' where " as <~~> as' \<and> map (assocs G) as' = ys"
+    by (metis (no_types, lifting) ex_map_conv mset_eq_perm set_mset_mset)
   then show ?case
-    by (smt ex_map_conv perm.trans perm_setP)
+    using trans.IH(2) trans.prems(2) by blast
 qed auto
 
 lemma (in comm_monoid_cancel) fmset_ee: