tuned exhaustive_generators
authorbulwahn
Mon, 14 Mar 2011 12:34:12 +0100
changeset 41966 d65835c381dd
parent 41965 328371f4f927
child 41967 6aa69999da8f
child 41969 1cf3e4107a2a
tuned exhaustive_generators
src/HOL/Tools/Quickcheck/exhaustive_generators.ML
--- a/src/HOL/Tools/Quickcheck/exhaustive_generators.ML	Mon Mar 14 12:34:11 2011 +0100
+++ b/src/HOL/Tools/Quickcheck/exhaustive_generators.ML	Mon Mar 14 12:34:12 2011 +0100
@@ -193,7 +193,7 @@
         #> apfst fst) (exhaustivesN ~~ (Ts @ Us))
       #> (fn (exhaustives, lthy) =>
         let
-          val eqs_t = mk_equations thy descr vs tycos exhaustives (Ts, Us)
+          val eqs_t = mk_equations descr vs tycos exhaustives (Ts, Us)
           val eqs = map (fn eq => Goal.prove lthy ["f", "i"] [] eq
             (fn _ => Skip_Proof.cheat_tac (ProofContext.theory_of lthy))) eqs_t
         in