src/HOL/Predicate_Compile.thy
changeset 47506 cde737f9c911
parent 46321 dc2236b19a3d
child 47509 fc315796794e
     1.1 --- a/src/HOL/Predicate_Compile.thy	Thu Feb 23 21:16:54 2012 +0100
     1.2 +++ b/src/HOL/Predicate_Compile.thy	Thu Feb 23 21:25:59 2012 +0100
     1.3 @@ -5,7 +5,7 @@
     1.4  header {* A compiler for predicates defined by introduction rules *}
     1.5  
     1.6  theory Predicate_Compile
     1.7 -imports New_Random_Sequence Quickcheck_Exhaustive
     1.8 +imports Predicate New_Random_Sequence Quickcheck_Exhaustive
     1.9  uses
    1.10    "Tools/Predicate_Compile/predicate_compile_aux.ML"
    1.11    "Tools/Predicate_Compile/predicate_compile_compilations.ML"