src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy
changeset 41956 c15ef1b85035
parent 41413 64cd30d6b0b8
child 43953 3b69f057ef2e
--- 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/) *}