src/HOL/Tools/Quickcheck/quickcheck_common.ML
changeset 42361 23f352990944
parent 42287 d98eb048a2e4
child 42793 88bee9f6eec7
equal deleted inserted replaced
42360:da8817d01e7c 42361:23f352990944
    63       #> apfst fst) (names ~~ Ts)
    63       #> apfst fst) (names ~~ Ts)
    64     #> (fn (consts, lthy) =>
    64     #> (fn (consts, lthy) =>
    65       let
    65       let
    66         val eqs_t = mk_equations consts
    66         val eqs_t = mk_equations consts
    67         val eqs = map (fn eq => Goal.prove lthy argnames [] eq
    67         val eqs = map (fn eq => Goal.prove lthy argnames [] eq
    68           (fn _ => Skip_Proof.cheat_tac (ProofContext.theory_of lthy))) eqs_t
    68           (fn _ => Skip_Proof.cheat_tac (Proof_Context.theory_of lthy))) eqs_t
    69       in
    69       in
    70         fold (fn (name, eq) => Local_Theory.note
    70         fold (fn (name, eq) => Local_Theory.note
    71         ((Binding.conceal (Binding.qualify true prfx
    71         ((Binding.conceal (Binding.qualify true prfx
    72            (Binding.qualify true name (Binding.name "simps"))),
    72            (Binding.qualify true name (Binding.name "simps"))),
    73            Code.add_default_eqn_attrib :: map (Attrib.internal o K)
    73            Code.add_default_eqn_attrib :: map (Attrib.internal o K)