diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/Nitpick_Examples/Refute_Nits.thy --- a/src/HOL/Nitpick_Examples/Refute_Nits.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/Nitpick_Examples/Refute_Nits.thy Sat Jan 05 17:24:33 2019 +0100 @@ -408,7 +408,7 @@ nitpick [expect = genuine] oops -subsubsection \@{const undefined}\ +subsubsection \\<^const>\undefined\\ lemma "undefined" nitpick [expect = genuine] @@ -426,7 +426,7 @@ nitpick [expect = genuine] oops -subsubsection \@{const The}\ +subsubsection \\<^const>\The\\ lemma "The P" nitpick [expect = genuine] @@ -448,7 +448,7 @@ nitpick [expect = genuine] oops -subsubsection \@{const Eps}\ +subsubsection \\<^const>\Eps\\ lemma "Eps P" nitpick [expect = genuine] @@ -525,7 +525,7 @@ subsubsection \Subtypes (typedef), typedecl\ -text \A completely unspecified non-empty subset of @{typ "'a"}:\ +text \A completely unspecified non-empty subset of \<^typ>\'a\:\ definition "myTdef = insert (undefined::'a) (undefined::'a set)"