diff -r 10fe23659be3 -r e8f4ce87012b src/HOL/Algebra/Group.thy --- a/src/HOL/Algebra/Group.thy Tue Apr 09 15:31:14 2019 +0100 +++ b/src/HOL/Algebra/Group.thy Tue Apr 09 21:05:32 2019 +0100 @@ -913,6 +913,9 @@ "\h \ hom G H; bij_betw h (carrier G) (carrier H)\ \ h \ iso G H" by (auto simp: iso_def) +lemma is_isoI: "h \ iso G H \ G \ H" + using is_iso_def by auto + lemma epi_iff_subset: "f \ epi G G' \ f \ hom G G' \ carrier G' \ f ` carrier G" by (auto simp: epi_def hom_def)