src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy
changeset 51599 1559e9266280
parent 48013 44de84112a67
child 57544 8840fa17e17c
equal deleted inserted replaced
51598:5dbe537087aa 51599:1559e9266280
     4 *)
     4 *)
     5 
     5 
     6 header {* Examples for the 'quickcheck' command *}
     6 header {* Examples for the 'quickcheck' command *}
     7 
     7 
     8 theory Quickcheck_Examples
     8 theory Quickcheck_Examples
     9 imports Complex_Main "~~/src/HOL/Library/Dlist" "~~/src/HOL/Library/Multiset"
     9 imports Complex_Main "~~/src/HOL/Library/Dlist" "~~/src/HOL/Library/DAList_Multiset"
    10 begin
    10 begin
    11 
    11 
    12 text {*
    12 text {*
    13 The 'quickcheck' command allows to find counterexamples by evaluating
    13 The 'quickcheck' command allows to find counterexamples by evaluating
    14 formulae.
    14 formulae.