src/HOL/Algebra/Group.thy
changeset 69597 ff784d5a5bfb
parent 69272 15e9ed5b28fb
child 69700 7a92cbec7030
--- a/src/HOL/Algebra/Group.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Algebra/Group.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -625,7 +625,7 @@
 qed
 
 text \<open>
-  Since @{term H} is nonempty, it contains some element @{term x}.  Since
+  Since \<^term>\<open>H\<close> is nonempty, it contains some element \<^term>\<open>x\<close>.  Since
   it is closed under inverse, it contains \<open>inv x\<close>.  Since
   it is closed under product, it contains \<open>x \<otimes> inv x = \<one>\<close>.
 \<close>
@@ -1021,8 +1021,8 @@
   using DirProd_iso_set_trans assms unfolding is_iso_def by blast
 
 
-text\<open>Basis for homomorphism proofs: we assume two groups @{term G} and
-  @{term H}, with a homomorphism @{term h} between them\<close>
+text\<open>Basis for homomorphism proofs: we assume two groups \<^term>\<open>G\<close> and
+  \<^term>\<open>H\<close>, with a homomorphism \<^term>\<open>h\<close> between them\<close>
 locale group_hom = G?: group G + H?: group H for G (structure) and H (structure) +
   fixes h
   assumes homh: "h \<in> hom G H"