--- a/src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy Sun Mar 13 20:56:00 2011 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy Sun Mar 13 21:21:48 2011 +0100
@@ -1,5 +1,5 @@
theory Code_Prolog_Examples
-imports Code_Prolog
+imports "~~/src/HOL/Library/Code_Prolog"
begin
section {* Example append *}
--- a/src/HOL/Predicate_Compile_Examples/Context_Free_Grammar_Example.thy Sun Mar 13 20:56:00 2011 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Context_Free_Grammar_Example.thy Sun Mar 13 21:21:48 2011 +0100
@@ -1,5 +1,5 @@
theory Context_Free_Grammar_Example
-imports Code_Prolog
+imports "~~/src/HOL/Library/Code_Prolog"
begin
declare mem_def[code_pred_inline]
--- 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]
--- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Sun Mar 13 20:56:00 2011 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Sun Mar 13 21:21:48 2011 +0100
@@ -1,5 +1,5 @@
theory Lambda_Example
-imports Code_Prolog
+imports "~~/src/HOL/Library/Code_Prolog"
begin
subsection {* Lambda *}
--- a/src/HOL/Predicate_Compile_Examples/List_Examples.thy Sun Mar 13 20:56:00 2011 +0100
+++ b/src/HOL/Predicate_Compile_Examples/List_Examples.thy Sun Mar 13 21:21:48 2011 +0100
@@ -1,5 +1,8 @@
theory List_Examples
-imports Main "~~/src/HOL/Library/Predicate_Compile_Quickcheck" "Code_Prolog"
+imports
+ Main
+ "~~/src/HOL/Library/Predicate_Compile_Quickcheck"
+ "~~/src/HOL/Library/Code_Prolog"
begin
setup {* Context.theory_map (Quickcheck.add_generator ("prolog", Code_Prolog.quickcheck)) *}
--- a/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Sun Mar 13 20:56:00 2011 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Sun Mar 13 21:21:48 2011 +0100
@@ -1,5 +1,7 @@
theory Reg_Exp_Example
-imports "~~/src/HOL/Library/Predicate_Compile_Quickcheck" Code_Prolog
+imports
+ "~~/src/HOL/Library/Predicate_Compile_Quickcheck"
+ "~~/src/HOL/Library/Code_Prolog"
begin
text {* An example from the experiments from SmallCheck (http://www.cs.york.ac.uk/fp/smallcheck/) *}