src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy
changeset 66453 cc19f7ca2ed6
parent 63680 6e1e8b5abbfa
child 68224 1f7308050349
--- 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 \<open>An example from the experiments from SmallCheck (\<^url>\<open>http://www.cs.york.ac.uk/fp/smallcheck\<close>)\<close>