src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy
changeset 66453 cc19f7ca2ed6
parent 63167 0909deb8059b
child 67399 eab6ce8368fa
--- a/src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -1,8 +1,8 @@
 theory Hotel_Example_Prolog
 imports
   Hotel_Example
-  "~~/src/HOL/Library/Predicate_Compile_Alternative_Defs"
-  "~~/src/HOL/Library/Code_Prolog"
+  "HOL-Library.Predicate_Compile_Alternative_Defs"
+  "HOL-Library.Code_Prolog"
 begin
 
 declare Let_def[code_pred_inline]