changeset 58889 | 5b7a9633cfa8 |
parent 58826 | 2ed2eaabe3df |
child 59484 | a130ae7a9398 |
--- a/src/HOL/Quickcheck_Exhaustive.thy Sun Nov 02 18:21:14 2014 +0100 +++ b/src/HOL/Quickcheck_Exhaustive.thy Sun Nov 02 18:21:45 2014 +0100 @@ -1,6 +1,6 @@ (* Author: Lukas Bulwahn, TU Muenchen *) -header {* A simple counterexample generator performing exhaustive testing *} +section {* A simple counterexample generator performing exhaustive testing *} theory Quickcheck_Exhaustive imports Quickcheck_Random