src/HOL/Tools/Predicate_Compile/predicate_compile_quickcheck.ML
changeset 61140 78ece168f5b5
parent 59154 68ca25931dce
child 69593 3dda49e08b9d
equal deleted inserted replaced
61130:8e736ce4c6f4 61140:78ece168f5b5
    24     (unit -> Code_Numeral.natural -> term list Lazy_Sequence.lazy_sequence) ->
    24     (unit -> Code_Numeral.natural -> term list Lazy_Sequence.lazy_sequence) ->
    25     Proof.context -> Proof.context
    25     Proof.context -> Proof.context
    26   val put_cps_result : (unit -> Code_Numeral.natural -> (bool * term list) option) ->
    26   val put_cps_result : (unit -> Code_Numeral.natural -> (bool * term list) option) ->
    27     Proof.context -> Proof.context
    27     Proof.context -> Proof.context
    28   val test_goals : (Predicate_Compile_Aux.compilation * bool) ->
    28   val test_goals : (Predicate_Compile_Aux.compilation * bool) ->
    29     Proof.context -> bool * bool -> (string * typ) list -> (term * term list) list ->
    29     Proof.context -> bool -> (string * typ) list -> (term * term list) list ->
    30     Quickcheck.result list
    30     Quickcheck.result list
    31   val nrandom : int Unsynchronized.ref
    31   val nrandom : int Unsynchronized.ref
    32   val debug : bool Unsynchronized.ref
    32   val debug : bool Unsynchronized.ref
    33   val no_higher_order_predicate : string list Unsynchronized.ref
    33   val no_higher_order_predicate : string list Unsynchronized.ref
    34 end;
    34 end;