src/Doc/Tutorial/Sets/Recur.thy
changeset 69597 ff784d5a5bfb
parent 67406 23307fd33906
--- a/src/Doc/Tutorial/Sets/Recur.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/Doc/Tutorial/Sets/Recur.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -34,14 +34,14 @@
 
 The HOL library formalizes
 some of the theory of wellfounded relations. For example
-@{prop"wf r"}\index{*wf|bold} means that relation @{term[show_types]"r::('a*'a)set"} is
+\<^prop>\<open>wf r\<close>\index{*wf|bold} means that relation @{term[show_types]"r::('a*'a)set"} is
 wellfounded.
 Finally we should mention that HOL already provides the mother of all
 inductions, \textbf{wellfounded
 induction}\indexbold{induction!wellfounded}\index{wellfounded
 induction|see{induction, wellfounded}} (@{thm[source]wf_induct}):
 @{thm[display]wf_induct[no_vars]}
-where @{term"wf r"} means that the relation @{term r} is wellfounded
+where \<^term>\<open>wf r\<close> means that the relation \<^term>\<open>r\<close> is wellfounded
 
 \<close>