Fixed a presentation error
authorpaulson <lp15@cam.ac.uk>
Tue, 28 Feb 2023 11:19:47 +0000
changeset 77407 02af8a1b97f6
parent 77406 c2013f617a70
child 77408 8fe30123aaab
Fixed a presentation error
src/HOL/Algebra/Coset.thy
--- a/src/HOL/Algebra/Coset.thy	Mon Feb 27 17:09:59 2023 +0000
+++ b/src/HOL/Algebra/Coset.thy	Tue Feb 28 11:19:47 2023 +0000
@@ -1609,7 +1609,7 @@
   shows "H <#> N = H"
   using group.set_mult_carrier_idem[OF subgroup.subgroup_is_group[OF HG group_axioms] NG] by simp
 
-text \<open>A normal subgroup is commutative with set_mult\<close>
+text \<open>A normal subgroup is commutative with set multiplication\<close>
 lemma (in group) commut_normal:
   assumes "subgroup H G" and "N\<lhd>G"
   shows "H<#>N = N<#>H"