src/HOL/Imperative_HOL/Ref.thy
changeset 54703 499f92dc6e45
parent 52435 6646bb548c6b
child 58889 5b7a9633cfa8
--- a/src/HOL/Imperative_HOL/Ref.thy	Mon Dec 09 12:16:52 2013 +0100
+++ b/src/HOL/Imperative_HOL/Ref.thy	Mon Dec 09 12:22:23 2013 +0100
@@ -10,8 +10,8 @@
 
 text {*
   Imperative reference operations; modeled after their ML counterparts.
-  See http://caml.inria.fr/pub/docs/manual-caml-light/node14.15.html
-  and http://www.smlnj.org/doc/Conversion/top-level-comparison.html
+  See @{url "http://caml.inria.fr/pub/docs/manual-caml-light/node14.15.html"}
+  and @{url "http://www.smlnj.org/doc/Conversion/top-level-comparison.html"}
 *}
 
 subsection {* Primitives *}