diff -r 703ea96b13c6 -r c15ef1b85035 src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy --- a/src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy Sun Mar 13 20:56:00 2011 +0100 +++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy Sun Mar 13 21:21:48 2011 +0100 @@ -1,5 +1,8 @@ theory Hotel_Example_Prolog -imports Hotel_Example "~~/src/HOL/Library/Predicate_Compile_Alternative_Defs" Code_Prolog +imports + Hotel_Example + "~~/src/HOL/Library/Predicate_Compile_Alternative_Defs" + "~~/src/HOL/Library/Code_Prolog" begin declare Let_def[code_pred_inline]