--- a/src/HOL/Library/Code_Lazy.thy Sun Jan 15 16:28:03 2023 +0100
+++ b/src/HOL/Library/Code_Lazy.thy Sun Jan 15 18:30:18 2023 +0100
@@ -15,7 +15,7 @@
begin
text \<open>
- This theory and the CodeLazy tool described in @{cite "LochbihlerStoop2018"}.
+ This theory and the CodeLazy tool described in \<^cite>\<open>"LochbihlerStoop2018"\<close>.
It hooks into Isabelle's code generator such that the generated code evaluates a user-specified
set of type constructors lazily, even in target languages with eager evaluation.