src/HOL/Predicate_Compile.thy
changeset 58823 513268cb2178
parent 55543 f0ef75c6c0d8
child 58889 5b7a9633cfa8
equal deleted inserted replaced
58822:90a5e981af3e 58823:513268cb2178
    19 ML_file "Tools/Predicate_Compile/predicate_compile_fun.ML"
    19 ML_file "Tools/Predicate_Compile/predicate_compile_fun.ML"
    20 ML_file "Tools/Predicate_Compile/predicate_compile_pred.ML"
    20 ML_file "Tools/Predicate_Compile/predicate_compile_pred.ML"
    21 ML_file "Tools/Predicate_Compile/predicate_compile_specialisation.ML"
    21 ML_file "Tools/Predicate_Compile/predicate_compile_specialisation.ML"
    22 ML_file "Tools/Predicate_Compile/predicate_compile.ML"
    22 ML_file "Tools/Predicate_Compile/predicate_compile.ML"
    23 
    23 
    24 setup Predicate_Compile.setup
       
    25 
    24 
    26 subsection {* Set membership as a generator predicate *}
    25 subsection {* Set membership as a generator predicate *}
    27 
    26 
    28 text {* 
    27 text {* 
    29   Introduce a new constant for membership to allow 
    28   Introduce a new constant for membership to allow