diff -r 35f30e07fe0d -r 64cd30d6b0b8 src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy --- a/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Wed Dec 29 13:51:17 2010 +0100 +++ b/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Wed Dec 29 17:34:41 2010 +0100 @@ -1,5 +1,5 @@ theory Reg_Exp_Example -imports Predicate_Compile_Quickcheck Code_Prolog +imports "~~/src/HOL/Library/Predicate_Compile_Quickcheck" Code_Prolog begin text {* An example from the experiments from SmallCheck (http://www.cs.york.ac.uk/fp/smallcheck/) *}