src/HOL/ex/Adhoc_Overloading_Examples.thy
changeset 69597 ff784d5a5bfb
parent 66453 cc19f7ca2ed6
child 69745 aec42cee2521
--- a/src/HOL/ex/Adhoc_Overloading_Examples.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/ex/Adhoc_Overloading_Examples.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -82,7 +82,7 @@
 subsection \<open>Adhoc Overloading inside Locales\<close>
 
 text \<open>As example we use permutations that are parametrized over an
-atom type @{typ "'a"}.\<close>
+atom type \<^typ>\<open>'a\<close>.\<close>
 
 definition perms :: "('a \<Rightarrow> 'a) set" where
   "perms = {f. bij f \<and> finite {x. f x \<noteq> x}}"
@@ -178,7 +178,7 @@
 
 consts PERMUTE :: "'a perm \<Rightarrow> 'b \<Rightarrow> 'b" (infixr "\<bullet>" 75)
 
-text \<open>Then we add a locale for types @{typ 'b} that support
+text \<open>Then we add a locale for types \<^typ>\<open>'b\<close> that support
 appliciation of permutations.\<close>
 locale permute =
   fixes permute :: "'a perm \<Rightarrow> 'b \<Rightarrow> 'b"