src/Doc/Typeclass_Hierarchy/Typeclass_Hierarchy.thy
changeset 67299 ba52a058942f
parent 66453 cc19f7ca2ed6
child 68484 59793df7f853
--- a/src/Doc/Typeclass_Hierarchy/Typeclass_Hierarchy.thy	Fri Dec 29 18:09:38 2017 +0100
+++ b/src/Doc/Typeclass_Hierarchy/Typeclass_Hierarchy.thy	Fri Dec 29 19:17:52 2017 +0100
@@ -28,8 +28,8 @@
   instantiating type-classes, adding relationships between
   locales (@{command sublocale}) and type-classes
   (@{command subclass}).  Handy introductions are the
-  respective tutorials \cite{isabelle-locale}
-  \cite{isabelle-classes}.
+  respective tutorials @{cite "isabelle-locale"}
+  @{cite "isabelle-classes"}.
 \<close>
 
 subsection \<open>Strengths and restrictions of type classes\<close>
@@ -48,7 +48,7 @@
   to the numerical type on the right hand side.
 
   How to accomplish this given the quite restrictive type system
-  of {Isabelle/HOL}?  Paulson \cite{paulson-numerical} explains
+  of {Isabelle/HOL}?  Paulson @{cite "paulson-numerical"} explains
   that each numerical type has some characteristic properties
   which define an characteristic algebraic structure;  @{text \<sqsubset>}
   then corresponds to specialization of the corresponding
@@ -122,7 +122,7 @@
   optionally showing the logical content for each class also.
   Optional parameters restrict the graph to a particular segment
   which is useful to get a graspable view.  See
-  the Isar reference manual \cite{isabelle-isar-ref} for details.
+  the Isar reference manual @{cite "isabelle-isar-ref"} for details.
 \<close>
 
 
@@ -144,7 +144,7 @@
     \<^item> @{command class} @{class one} with @{term [source] "1::'a::one"}
 
   \noindent Before the introduction of the @{command class} statement in
-  Isabelle \cite{Haftmann-Wenzel:2006:classes} it was impossible
+  Isabelle @{cite "Haftmann-Wenzel:2006:classes"} it was impossible
   to define operations with associated axioms in the same class,
   hence there were always pairs of syntactic and logical type
   classes.  This restriction is lifted nowadays, but there are