src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy
changeset 54703 499f92dc6e45
parent 52666 391913d17d15
child 56927 4044a7d1720f
--- a/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy	Mon Dec 09 12:16:52 2013 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy	Mon Dec 09 12:22:23 2013 +0100
@@ -4,7 +4,7 @@
   "~~/src/HOL/Library/Code_Prolog"
 begin
 
-text {* An example from the experiments from SmallCheck (http://www.cs.york.ac.uk/fp/smallcheck/) *}
+text {* An example from the experiments from SmallCheck (@{url "http://www.cs.york.ac.uk/fp/smallcheck/"}) *}
 text {* The example (original in Haskell) was imported with Haskabelle and
   manually slightly adapted.
 *}