src/Doc/Tutorial/Advanced/simp2.thy
changeset 58620 7435b6a3f72e
parent 57512 cc97b347b301
child 67406 23307fd33906
--- a/src/Doc/Tutorial/Advanced/simp2.thy	Tue Oct 07 21:44:41 2014 +0200
+++ b/src/Doc/Tutorial/Advanced/simp2.thy	Tue Oct 07 22:35:11 2014 +0200
@@ -123,7 +123,7 @@
 rewrite rules. This is not quite true.  For reasons of feasibility,
 the simplifier expects the
 left-hand side of each rule to be a so-called \emph{higher-order
-pattern}~\cite{nipkow-patterns}\indexbold{patterns!higher-order}. 
+pattern}~@{cite "nipkow-patterns"}\indexbold{patterns!higher-order}. 
 This restricts where
 unknowns may occur.  Higher-order patterns are terms in $\beta$-normal
 form.  (This means there are no subterms of the form $(\lambda x. M)(N)$.)