src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy
changeset 41956 c15ef1b85035
parent 41413 64cd30d6b0b8
child 43885 7caa1139b4e5
--- 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]