diff -r 1e31ddcab458 -r 4c275405faae src/HOL/Library/Code_Lazy.thy --- 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 \ - This theory and the CodeLazy tool described in @{cite "LochbihlerStoop2018"}. + This theory and the CodeLazy tool described in \<^cite>\"LochbihlerStoop2018"\. 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.