src/Doc/Prog_Prove/Logic.thy
changeset 58620 7435b6a3f72e
parent 58605 9d5013661ac6
child 58962 e3491acee50f
--- a/src/Doc/Prog_Prove/Logic.thy	Tue Oct 07 21:44:41 2014 +0200
+++ b/src/Doc/Prog_Prove/Logic.thy	Tue Oct 07 22:35:11 2014 +0200
@@ -139,7 +139,7 @@
 @{thm image_def}\index{$IMP042@@{term"f ` A"}} & is the image of a function over a set
 \end{tabular}
 \end{center}
-See \cite{Nipkow-Main} for the wealth of further predefined functions in theory
+See @{cite "Nipkow-Main"} for the wealth of further predefined functions in theory
 @{theory Main}.
 
 
@@ -399,7 +399,7 @@
   {\mbox{@{text"?P = ?Q"}}}
 \]
 These rules are part of the logical system of \concept{natural deduction}
-(e.g., \cite{HuthRyan}). Although we intentionally de-emphasize the basic rules
+(e.g., @{cite HuthRyan}). Although we intentionally de-emphasize the basic rules
 of logic in favour of automatic proof methods that allow you to take bigger
 steps, these rules are helpful in locating where and why automation fails.
 When applied backwards, these rules decompose the goal:
@@ -486,7 +486,7 @@
 %
 %Command \isacom{find{\isacharunderscorekeyword}theorems} searches for specific theorems in the current
 %theory. Search criteria include pattern matching on terms and on names.
-%For details see the Isabelle/Isar Reference Manual~\cite{IsarRef}.
+%For details see the Isabelle/Isar Reference Manual~@{cite IsarRef}.
 %\bigskip
 
 \begin{warn}