src/HOL/Wfrec.thy
changeset 69593 3dda49e08b9d
parent 63572 c0cbfd2b5a45
child 71544 66bc4b668d6e
--- a/src/HOL/Wfrec.thy	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/HOL/Wfrec.thy	Fri Jan 04 23:22:53 2019 +0100
@@ -89,7 +89,7 @@
 
 definition same_fst :: "('a \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> ('b \<times> 'b) set) \<Rightarrow> (('a \<times> 'b) \<times> ('a \<times> 'b)) set"
   where "same_fst P R = {((x', y'), (x, y)) . x' = x \<and> P x \<and> (y',y) \<in> R x}"
-   \<comment> \<open>For @{const wfrec} declarations where the first n parameters
+   \<comment> \<open>For \<^const>\<open>wfrec\<close> declarations where the first n parameters
        stay unchanged in the recursive call.\<close>
 
 lemma same_fstI [intro!]: "P x \<Longrightarrow> (y', y) \<in> R x \<Longrightarrow> ((x, y'), (x, y)) \<in> same_fst P R"