src/HOL/Quickcheck.thy
changeset 41928 05abcee548a1
parent 41923 f05fc0711bc7
child 41935 d786a8a3dc47
equal deleted inserted replaced
41927:8759e9d043f9 41928:05abcee548a1
     2 
     2 
     3 header {* A simple counterexample generator performing random testing *}
     3 header {* A simple counterexample generator performing random testing *}
     4 
     4 
     5 theory Quickcheck
     5 theory Quickcheck
     6 imports Random Code_Evaluation Enum
     6 imports Random Code_Evaluation Enum
     7 uses ("Tools/Quickcheck/random_generators.ML")
     7 uses
       
     8   "Tools/Quickcheck/quickcheck_common.ML"
       
     9   ("Tools/Quickcheck/random_generators.ML")
     8 begin
    10 begin
     9 
    11 
    10 notation fcomp (infixl "\<circ>>" 60)
    12 notation fcomp (infixl "\<circ>>" 60)
    11 notation scomp (infixl "\<circ>\<rightarrow>" 60)
    13 notation scomp (infixl "\<circ>\<rightarrow>" 60)
    12 
    14