src/Doc/Codegen/Evaluation.thy
changeset 58620 7435b6a3f72e
parent 58310 91ea607a34d8
child 59334 f0141b991c8f
--- a/src/Doc/Codegen/Evaluation.thy	Tue Oct 07 21:44:41 2014 +0200
+++ b/src/Doc/Codegen/Evaluation.thy	Tue Oct 07 22:35:11 2014 +0200
@@ -53,7 +53,7 @@
 subsubsection {* Normalization by evaluation (@{text nbe}) *}
 
 text {*
-  Normalization by evaluation \cite{Aehlig-Haftmann-Nipkow:2008:nbe}
+  Normalization by evaluation @{cite "Aehlig-Haftmann-Nipkow:2008:nbe"}
   provides a comparably fast partially symbolic evaluation which
   permits also normalization of functions and uninterpreted symbols;
   the stack of code to be trusted is considerable.