src/HOL/Tools/Quickcheck/quickcheck_common.ML
changeset 45039 632a033616e9
parent 44241 7943b69f0188
child 45159 3f1d1ce024cb
equal deleted inserted replaced
45038:e24bf05dd273 45039:632a033616e9
    16       -> string list -> string -> string list * string list -> typ list * typ list -> theory -> theory)
    16       -> string list -> string -> string list * string list -> typ list * typ list -> theory -> theory)
    17     -> Datatype.config -> string list -> theory -> theory
    17     -> Datatype.config -> string list -> theory -> theory
    18   val gen_mk_parametric_generator_expr :
    18   val gen_mk_parametric_generator_expr :
    19    (((Proof.context -> term * term list -> term) * term) * typ)
    19    (((Proof.context -> term * term list -> term) * term) * typ)
    20      -> Proof.context -> (term * term list) list -> term
    20      -> Proof.context -> (term * term list) list -> term
       
    21   val mk_fun_upd : typ -> typ -> term * term -> term -> term
    21   val post_process_term : term -> term
    22   val post_process_term : term -> term
    22 end;
    23 end;
    23 
    24 
    24 structure Quickcheck_Common : QUICKCHECK_COMMON =
    25 structure Quickcheck_Common : QUICKCHECK_COMMON =
    25 struct
    26 struct