diff -r 450cefec7c11 -r cc19f7ca2ed6 src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy --- a/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Fri Aug 18 13:55:05 2017 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Fri Aug 18 20:47:47 2017 +0200 @@ -1,7 +1,7 @@ theory Reg_Exp_Example imports - "~~/src/HOL/Library/Predicate_Compile_Quickcheck" - "~~/src/HOL/Library/Code_Prolog" + "HOL-Library.Predicate_Compile_Quickcheck" + "HOL-Library.Code_Prolog" begin text \An example from the experiments from SmallCheck (\<^url>\http://www.cs.york.ac.uk/fp/smallcheck\)\