diff -r 9b6a0fb85fa3 -r c3658c18b7bc src/HOL/Library/Groups_Big_Fun.thy --- a/src/HOL/Library/Groups_Big_Fun.thy Tue Oct 13 09:21:14 2015 +0200 +++ b/src/HOL/Library/Groups_Big_Fun.thy Tue Oct 13 09:21:15 2015 +0200 @@ -183,7 +183,7 @@ have bij: "bij (\(a, b, c). ((a, b), c))" by (auto intro!: bijI injI simp add: image_def) have "{p. \c. g (fst p) (snd p) c \ 1} \ {c. \p. g (fst p) (snd p) c \ 1} \ D" - by auto (insert subset, auto) + by auto (insert subset, blast) with fin have "G (\p. G (g (fst p) (snd p))) = G (\(p, c). g (fst p) (snd p) c)" by (rule cartesian_product) then have "G (\(a, b). G (g a b)) = G (\((a, b), c). g a b c)"