--- a/src/HOL/Isar_Examples/Structured_Statements.thy Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Isar_Examples/Structured_Statements.thy Sat Jan 05 17:24:33 2019 +0100
@@ -152,9 +152,9 @@
have C
proof -
- show ?thesis when "A x" (is ?A) for x :: 'a \<comment> \<open>abstract @{term x}\<close>
+ show ?thesis when "A x" (is ?A) for x :: 'a \<comment> \<open>abstract \<^term>\<open>x\<close>\<close>
using that \<proof>
- show "?A a" \<comment> \<open>concrete @{term a}\<close>
+ show "?A a" \<comment> \<open>concrete \<^term>\<open>a\<close>\<close>
\<proof>
qed
end