src/HOL/ex/While_Combinator_Example.thy
changeset 69597 ff784d5a5bfb
parent 67613 ce654b0e6d69
--- a/src/HOL/ex/While_Combinator_Example.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/ex/While_Combinator_Example.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -9,7 +9,7 @@
 imports "HOL-Library.While_Combinator"
 begin
 
-text \<open>Computation of the @{term lfp} on finite sets via 
+text \<open>Computation of the \<^term>\<open>lfp\<close> on finite sets via 
   iteration.\<close>
 
 theorem lfp_conv_while: