src/Doc/Functions/Functions.thy
changeset 58620 7435b6a3f72e
parent 58310 91ea607a34d8
child 59005 1c54ebc68394
--- a/src/Doc/Functions/Functions.thy	Tue Oct 07 21:44:41 2014 +0200
+++ b/src/Doc/Functions/Functions.thy	Tue Oct 07 22:35:11 2014 +0200
@@ -278,7 +278,7 @@
 text {*
   To see how the automatic termination proofs work, let's look at an
   example where it fails\footnote{For a detailed discussion of the
-  termination prover, see \cite{bulwahnKN07}}:
+  termination prover, see @{cite bulwahnKN07}}:
 
 \end{isamarkuptext}  
 \cmd{fun} @{text "fails :: \"nat \<Rightarrow> nat list \<Rightarrow> nat\""}\\%
@@ -334,7 +334,7 @@
   more powerful @{text size_change} method, which uses a variant of
   the size-change principle, together with some other
   techniques. While the details are discussed
-  elsewhere\cite{krauss_phd},
+  elsewhere @{cite krauss_phd},
   here are a few typical situations where
   @{text lexicographic_order} has difficulties and @{text size_change}
   may be worth a try: