QuickChickInterfaceQuickChick Reference Manual
From QuickChick Require Import QuickChick.
Require Import ZArith Strings.Ascii Strings.String.
From ExtLib.Structures Require Import Functor Applicative.
Require Import ZArith Strings.Ascii Strings.String.
From ExtLib.Structures Require Import Functor Applicative.
QuickChick provides a large collection of combinators and
notations for writing property-based random tests. This file
documents the entire public interface (the module type
QuickChickSig).
The Show Typeclass
Class Show (A : Type) : Type :=
{
show : A → string
}.
#[export] Declare Instance showNat : Show nat.
#[export] Declare Instance showBool : Show bool.
#[export] Declare Instance showZ : Show Z.
#[export] Declare Instance showString : Show string.
#[export] Declare Instance showList :
∀ {A : Type} `{Show A}, Show (list A).
#[export] Declare Instance showPair :
∀ {A B : Type} `{Show A} `{Show B}, Show (A × B).
#[export] Declare Instance showOpt :
∀ {A : Type} `{Show A}, Show (option A).
#[export] Declare Instance showEx :
∀ {A} `{Show A} P, Show ({x : A | P x}).
#[export] Declare Instance showBool : Show bool.
#[export] Declare Instance showZ : Show Z.
#[export] Declare Instance showString : Show string.
#[export] Declare Instance showList :
∀ {A : Type} `{Show A}, Show (list A).
#[export] Declare Instance showPair :
∀ {A B : Type} `{Show A} `{Show B}, Show (A × B).
#[export] Declare Instance showOpt :
∀ {A : Type} `{Show A}, Show (option A).
#[export] Declare Instance showEx :
∀ {A} `{Show A} P, Show ({x : A | P x}).
When defining Show instance for your own datatypes, you sometimes need to
start a new line for better printing. nl is a shorthand for it.
G A is the type of random generators for type A.
Run a generator with a size parameter (a natural number denoting
the maximum depth of the generated A) and a random seed.
The semantics of a generator is its set of possible outcomes.
Parameter semGen : ∀ {A : Type} (g : G A), set A.
Parameter semGenSize : ∀ {A : Type} (g : G A) (size : nat), set A.
Parameter semGenSize : ∀ {A : Type} (g : G A) (size : nat), set A.
Structural Combinators
#[export] Declare Instance Monad_G : Monad G.
#[export] Declare Instance Functor_G : Functor G.
#[export] Declare Instance Applicative_G : Applicative G.
#[export] Declare Instance Functor_G : Functor G.
#[export] Declare Instance Applicative_G : Applicative G.
A variant of bind for the (G (option --)) monad. Useful for
chaining generators that can fail / backtrack.
Basic Generator Combinators
Parameter listOf : ∀ {A : Type}, G A → G (list A).
Parameter vectorOf : ∀ {A : Type}, nat → G A → G (list A).
Parameter vectorOf : ∀ {A : Type}, nat → G A → G (list A).
elems_ a l constructs a generator from a list l and a
default element a. If l is non-empty, the generator picks an
element from l uniformly; otherwise it always yields a.
Similar to elems_, instead of choosing from a list of As,
oneOf_ g l returns g if l is empty; otherwise it uniformly
picks a generator for A in l.
We can also choose generators with distributions other than the
uniform one. freq_ g l returns g if l is empty;
otherwise it chooses a generator from l, where the first field
indicates the chance that the second field is chosen. For example,
freq_ z [(2, x); (3, y)] has 40% probability of choosing
x and 60% probability of choosing y.
Try all generators until one returns a Some value or all failed once with
None. The generators are picked at random according to their weights
(like frequency), and each one is run at most once.
Internally, the G monad hides a size parameter that can be accessed by
generators. The sized combinator provides such access. The resize
combinator sets it.
Generate-and-test approach to generate data with preconditions.
Parameter suchThatMaybe :
∀ {A : Type}, G A → (A → bool) → G (option A).
Parameter suchThatMaybeOpt :
∀ {A : Type}, G (option A) → (A → bool) → G (option A).
∀ {A : Type}, G A → (A → bool) → G (option A).
Parameter suchThatMaybeOpt :
∀ {A : Type}, G (option A) → (A → bool) → G (option A).
The elems_, oneOf_, and freq_ combinators all take
default values; these are only used if their list arguments are
empty, which should not normally happen. The QcDefaultNotation
sub-module exposes notation (without the underscores) to hide this default.
elems is a shorthand for elems_ without a default argument.
Notation " 'elems' [ x ] " :=
(elems_ x (cons x nil)) : qc_scope.
Notation " 'elems' [ x ; y ] " :=
(elems_ x (cons x (cons y nil))) : qc_scope.
Notation " 'elems' [ x ; y ; .. ; z ] " :=
(elems_ x (cons x (cons y .. (cons z nil) ..))) : qc_scope.
Notation " 'elems' ( x ;; l ) " :=
(elems_ x (cons x l)) (at level 1, no associativity) : qc_scope.
(elems_ x (cons x nil)) : qc_scope.
Notation " 'elems' [ x ; y ] " :=
(elems_ x (cons x (cons y nil))) : qc_scope.
Notation " 'elems' [ x ; y ; .. ; z ] " :=
(elems_ x (cons x (cons y .. (cons z nil) ..))) : qc_scope.
Notation " 'elems' ( x ;; l ) " :=
(elems_ x (cons x l)) (at level 1, no associativity) : qc_scope.
oneOf is a shorthand for oneOf_ without a default argument.
Notation " 'oneOf' [ x ] " :=
(oneOf_ x (cons x nil)) : qc_scope.
Notation " 'oneOf' [ x ; y ] " :=
(oneOf_ x (cons x (cons y nil))) : qc_scope.
Notation " 'oneOf' [ x ; y ; .. ; z ] " :=
(oneOf_ x (cons x (cons y .. (cons z nil) ..))) : qc_scope.
Notation " 'oneOf' ( x ;; l ) " :=
(oneOf_ x (cons x l)) (at level 1, no associativity) : qc_scope.
(oneOf_ x (cons x nil)) : qc_scope.
Notation " 'oneOf' [ x ; y ] " :=
(oneOf_ x (cons x (cons y nil))) : qc_scope.
Notation " 'oneOf' [ x ; y ; .. ; z ] " :=
(oneOf_ x (cons x (cons y .. (cons z nil) ..))) : qc_scope.
Notation " 'oneOf' ( x ;; l ) " :=
(oneOf_ x (cons x l)) (at level 1, no associativity) : qc_scope.
freq is a shorthand for freq_ without a default argument.
Notation " 'freq' [ x ] " :=
(freq_ x (cons x nil)) : qc_scope.
Notation " 'freq' [ ( n , x ) ; y ] " :=
(freq_ x (cons (n, x) (cons y nil))) : qc_scope.
Notation " 'freq' [ ( n , x ) ; y ; .. ; z ] " :=
(freq_ x (cons (n, x) (cons y .. (cons z nil) ..))) : qc_scope.
Notation " 'freq' ( ( n , x ) ;; l ) " :=
(freq_ x (cons (n, x) l)) (at level 1, no associativity) : qc_scope.
End QcDefaultNotation.
(freq_ x (cons x nil)) : qc_scope.
Notation " 'freq' [ ( n , x ) ; y ] " :=
(freq_ x (cons (n, x) (cons y nil))) : qc_scope.
Notation " 'freq' [ ( n , x ) ; y ; .. ; z ] " :=
(freq_ x (cons (n, x) (cons y .. (cons z nil) ..))) : qc_scope.
Notation " 'freq' ( ( n , x ) ;; l ) " :=
(freq_ x (cons (n, x) l)) (at level 1, no associativity) : qc_scope.
End QcDefaultNotation.
The original version of QuickChick used elements, oneof and frequency
as the default-argument versions of the corresponding combinators.
These have since been deprecated in favor of a more consistent
naming scheme.
Choosing from Intervals
Existing Class OrdType.
#[export] Declare Instance OrdBool : OrdType bool.
#[export] Declare Instance OrdNat : OrdType nat.
#[export] Declare Instance OrdZ : OrdType Z.
#[export] Declare Instance OrdBool : OrdType bool.
#[export] Declare Instance OrdNat : OrdType nat.
#[export] Declare Instance OrdZ : OrdType Z.
We also expect the random function to be able to pick every element in any
given interval.
Existing Class ChoosableFromInterval.
QuickChick has provided some instances for ordered data types that are
choosable from intervals, including bool, nat, and Z.
#[export] Declare Instance ChooseBool : ChoosableFromInterval bool.
#[export] Declare Instance ChooseNat : ChoosableFromInterval nat.
#[export] Declare Instance ChooseZ : ChoosableFromInterval Z.
#[export] Declare Instance ChooseNat : ChoosableFromInterval nat.
#[export] Declare Instance ChooseZ : ChoosableFromInterval Z.
choose l r generates a value between l and r, inclusive the two
extremes. It causes a runtime error if r < l.
The Gen and GenSized Typeclasses
Class GenSized (A : Type) := { arbitrarySized : nat → G A }.
Class Gen (A : Type) := { arbitrary : G A }.
Here are some basic instances for generators:
#[export] Declare Instance genBoolSized : GenSized bool.
#[export] Declare Instance genNatSized : GenSized nat.
#[export] Declare Instance genZSized : GenSized Z.
#[export] Declare Instance genListSized :
∀ {A : Type} `{GenSized A}, GenSized (list A).
#[export] Declare Instance genList :
∀ {A : Type} `{Gen A}, Gen (list A).
#[export] Declare Instance genOption :
∀ {A : Type} `{Gen A}, Gen (option A).
#[export] Declare Instance genPairSized :
∀ {A B : Type} `{GenSized A} `{GenSized B}, GenSized (A×B).
#[export] Declare Instance genPair :
∀ {A B : Type} `{Gen A} `{Gen B}, Gen (A × B).
#[export] Declare Instance genNatSized : GenSized nat.
#[export] Declare Instance genZSized : GenSized Z.
#[export] Declare Instance genListSized :
∀ {A : Type} `{GenSized A}, GenSized (list A).
#[export] Declare Instance genList :
∀ {A : Type} `{Gen A}, Gen (list A).
#[export] Declare Instance genOption :
∀ {A : Type} `{Gen A}, Gen (option A).
#[export] Declare Instance genPairSized :
∀ {A B : Type} `{GenSized A} `{GenSized B}, GenSized (A×B).
#[export] Declare Instance genPair :
∀ {A B : Type} `{Gen A} `{Gen B}, Gen (A × B).
Generators for Data Satisfying Inductive Predicates
Class GenSizedSuchThat (A : Type) (P : A → Prop) :=
{
arbitrarySizeST : nat → G (option A)
}.
Class GenSuchThat (A : Type) (P : A → Prop) :=
{
arbitraryST : G (option A)
}.
@arbitraryST _ (fun e ⇒ has_type e T) _ where the first placeholder is the type of expressions exp and the second placeholder is the actual instance to be inferred.
(*
Notation "'genST' x" := (@arbitraryST _ x _) (at level 70).
*)
Notation "'genST' x" := (@arbitraryST _ x _) (at level 70).
*)
Shrinking
The Shrink Typeclass
Class Shrink (A : Type) :=
{
shrink : A → list A
}.
#[export] Declare Instance shrinkBool : Shrink bool.
#[export] Declare Instance shrinkNat : Shrink nat.
#[export] Declare Instance shrinkZ : Shrink Z.
#[export] Declare Instance shrinkList {A : Type} `{Shrink A} : Shrink (list A).
#[export] Declare Instance shrinkPair {A B} `{Shrink A} `{Shrink B} : Shrink (A × B).
#[export] Declare Instance shrinkOption {A : Type} `{Shrink A} : Shrink (option A).
#[export] Declare Instance shrinkNat : Shrink nat.
#[export] Declare Instance shrinkZ : Shrink Z.
#[export] Declare Instance shrinkList {A : Type} `{Shrink A} : Shrink (list A).
#[export] Declare Instance shrinkPair {A B} `{Shrink A} `{Shrink B} : Shrink (A × B).
#[export] Declare Instance shrinkOption {A : Type} `{Shrink A} : Shrink (option A).
The Arbitrary Typeclass
Class Arbitrary (A : Type) `{Gen A} `{Shrink A}.
The Generator Typeclass Hierarchy
GenSized
|
|
Gen Shrink
\ /
\ /
Arbitrary
The Checkable class indicates we can check a type A.
Class Checkable (A : Type) : Type :=
{
checker : A → Checker
}.
Boolean checkers always pass or always fail.
Class Checkable (A : Type) : Type :=
{
checker : A → Checker
}.
The unit checker is always discarded (that is, it represents a
useless test). It is used, for example, in the implementation of
the "implication Checker" combinator ==>.
Given a generator for showable As, construct a Checker.
Parameter forAll :
∀ {A prop : Type} `{Checkable prop} `{Show A}
(gen : G A) (pf : A → prop), Checker.
∀ {A prop : Type} `{Checkable prop} `{Show A}
(gen : G A) (pf : A → prop), Checker.
A variant of forAll that provides evidence that the generated
values are members of the semantics of the generator. (Such evidence
can be useful when constructing dependently typed data, such as
bounded integers.)
Parameter forAllProof :
∀ {A prop : Type} `{Checkable prop} `{Show A}
(gen : G A) (pf : ∀ (x : A), semGen gen x → prop), Checker.
∀ {A prop : Type} `{Checkable prop} `{Show A}
(gen : G A) (pf : ∀ (x : A), semGen gen x → prop), Checker.
Given a generator and a shrinker for showable As, construct a
Checker.
Parameter forAllShrink :
∀ {A prop : Type} `{Checkable prop} `{Show A}
(gen : G A) (shrinker : A → list A) (pf : A → prop), Checker.
∀ {A prop : Type} `{Checkable prop} `{Show A}
(gen : G A) (shrinker : A → list A) (pf : A → prop), Checker.
Lift (Show, Gen, Shrink) instances for A
to a Checker for functions A -> prop. This is what makes it
possible to write (for some example property foo := fun x ⇒ x >?
0, say) QuickChick foo instead of QuickChick (forAllShrink
arbitrary shrink foo).
#[export] Declare Instance testFun :
∀ {A prop : Type} `{Show A} `{Arbitrary A} `{Checkable prop},
Checkable (A → prop).
∀ {A prop : Type} `{Show A} `{Arbitrary A} `{Checkable prop},
Checkable (A → prop).
Lift products similarly.
#[export] Declare Instance testProd :
∀ {A : Type} {prop : A → Type} `{Show A} `{Arbitrary A}
`{∀ x : A, Checkable (prop x)},
Checkable (∀ (x : A), prop x).
∀ {A : Type} {prop : A → Type} `{Show A} `{Arbitrary A}
`{∀ x : A, Checkable (prop x)},
Checkable (∀ (x : A), prop x).
Lift polymorphic functions by instantiating to 'nat'. :-)
#[export] Declare Instance testPolyFun :
∀ {prop : Type → Type} `{Checkable (prop nat)},
Checkable (∀ T, prop T).
∀ {prop : Type → Type} `{Checkable (prop nat)},
Checkable (∀ T, prop T).
Record an expectation that a property should fail, i.e.
the property will fail if all the tests succeed.
Collect statistics across all tests.
Set the reason for failure. Will only count shrinks as valid if
they preserve the tag.
Form the conjunction / disjunction of a list of checkers.
Parameter conjoin : ∀ (l : list Checker), Checker.
Parameter disjoin : ∀ (l : list Checker), Checker.
Parameter disjoin : ∀ (l : list Checker), Checker.
Define a checker for a conditional property. Invalid generated
inputs (ones for which the antecedent fails) are discarded.
Notation for implication. Clashes with many other notations in
other libraries, so it lives in its own module. Note that this
includes the notations for the generator combinators above
to avoid needing to import two modules.
Module QcNotation.
Export QcDefaultNotation.
Notation "x ==> y" :=
(implication x y) (at level 55, right associativity)
: Checker_scope.
End QcNotation.
Export QcDefaultNotation.
Notation "x ==> y" :=
(implication x y) (at level 55, right associativity)
: Checker_scope.
End QcNotation.
Decidability
The Dec Typeclass
Decidability typeclass using ssreflect's 'decidable'.Class Dec (P : Prop) : Type := { dec : decidable P }.
Logic Combinator instances.
#[export] Declare Instance Dec_neg {P} {H : Dec P} : Dec (¬ P).
#[export] Declare Instance Dec_conj {P Q} {H : Dec P} {I : Dec Q} : Dec (P ∧ Q).
#[export] Declare Instance Dec_disj {P Q} {H : Dec P} {I : Dec Q} : Dec (P ∨ Q).
#[export] Declare Instance Dec_conj {P Q} {H : Dec P} {I : Dec Q} : Dec (P ∧ Q).
#[export] Declare Instance Dec_disj {P Q} {H : Dec P} {I : Dec Q} : Dec (P ∨ Q).
A convenient notation for coercing a decidable proposition to a bool.
The Dec_Eq Typeclass
Class Dec_Eq (A : Type) :=
{
dec_eq : ∀ (x y : A), decidable (x = y)
}.
Since deciding equalities is a very common requirement in testing,
QuickChick provides a tactic that can define instances of the form
Dec (x = y).
Ltac dec_eq.
QuickChick also lifts common decidable instances to the Dec typeclass.
Ltac dec_eq.
#[export] Declare Instance Dec_eq_bool (x y : bool) : Dec (x = y).
#[export] Declare Instance Dec_eq_nat (m n : nat) : Dec (m = n).
#[export] Declare Instance Dec_eq_opt (A : Type) (m n : option A)
`{_ : ∀ (x y : A), Dec (x = y)} : Dec (m = n).
#[export] Declare Instance Dec_eq_prod (A B : Type) (m n : A × B)
`{_ : ∀ (x y : A), Dec (x = y)}
`{_ : ∀ (x y : B), Dec (x = y)}
: Dec (m = n).
#[export] Declare Instance Dec_eq_list (A : Type) (m n : list A)
`{_ : ∀ (x y : A), Dec (x = y)} : Dec (m = n).
#[export] Declare Instance Dec_ascii (m n : Ascii.ascii) : Dec (m = n).
#[export] Declare Instance Dec_string (m n : string) : Dec (m = n).
#[export] Declare Instance Dec_eq_nat (m n : nat) : Dec (m = n).
#[export] Declare Instance Dec_eq_opt (A : Type) (m n : option A)
`{_ : ∀ (x y : A), Dec (x = y)} : Dec (m = n).
#[export] Declare Instance Dec_eq_prod (A B : Type) (m n : A × B)
`{_ : ∀ (x y : A), Dec (x = y)}
`{_ : ∀ (x y : B), Dec (x = y)}
: Dec (m = n).
#[export] Declare Instance Dec_eq_list (A : Type) (m n : list A)
`{_ : ∀ (x y : A), Dec (x = y)} : Dec (m = n).
#[export] Declare Instance Dec_ascii (m n : Ascii.ascii) : Dec (m = n).
#[export] Declare Instance Dec_string (m n : string) : Dec (m = n).
Automatic Instance Derivation
Derive <class> for T. Here <class> must be one of GenSized, Shrink, Arbitrary, or Show, and T must be an inductive defined datatype (think Haskell/OCaml).
Derive (<class>,...,<class>) for T.
- A paper on deriving QuickChick generators for a large class of
inductive relations.
https://lemonidas.github.io/pdf/GeneratingGoodGenerators.pdf
- Leo's PhD dissertation.
https://lemonidas.github.io/pdf/Leo-PhD-Thesis.pdf
- examples/DependentTest.v
Top-level Commands and Settings
Sample g.
QuickChick prop.
Record Args :=
MkArgs
{
(* Re-execute a test. *)
(* Default: None *)
replay : option (RandomSeed × nat);
(* Maximum number of successful tests to run. *)
(* Default: 10000 *)
maxSuccess : nat;
(* Maximum number of discards to accept. *)
(* Default: 20000 *)
maxDiscard : nat;
(* Maximum number of shrinks to perform before terminating. *)
(* Default : 1000 *)
maxShrinks : nat;
(* Maximum size of terms to generate (depth). *)
(* Default : 7 *)
maxSize : nat;
(* Verbosity. Note: Doesn't do much... *)
(* Default true. *)
chatty : bool
}.
MkArgs
{
(* Re-execute a test. *)
(* Default: None *)
replay : option (RandomSeed × nat);
(* Maximum number of successful tests to run. *)
(* Default: 10000 *)
maxSuccess : nat;
(* Maximum number of discards to accept. *)
(* Default: 20000 *)
maxDiscard : nat;
(* Maximum number of shrinks to perform before terminating. *)
(* Default : 1000 *)
maxShrinks : nat;
(* Maximum size of terms to generate (depth). *)
(* Default : 7 *)
maxSize : nat;
(* Verbosity. Note: Doesn't do much... *)
(* Default true. *)
chatty : bool
}.
Instead of record updates, you should overwrite extraction constants.
Extract Constant defNumTests ⇒ "10000".
Extract Constant defNumDiscards ⇒ "(2 * defNumTests)".
Extract Constant defNumShrinks ⇒ "1000".
Extract Constant defSize ⇒ "7".
Extract Constant defNumTests ⇒ "10000".
Extract Constant defNumDiscards ⇒ "(2 * defNumTests)".
Extract Constant defNumShrinks ⇒ "1000".
Extract Constant defSize ⇒ "7".
The quickChick Command-Line Tool
- Batch processing, compilation and execution of tests
- Mutation testing
- Sectioning of tests and mutants
Test Annotations
(*! QuickChick prop. *)
Only tests that are annotated this way will be processed. Only property names are allowed.
Mutant Annotations
(*! *)
Normal code
(*!! mutant-name *)
(*! mutant 1 *)
(*! mutant 2 *)
... etc ...
Section Annotations
(*! Section section-name *)
Optionally, one can include an extends clause
(*! Section section-name *)(*! extends other-section-name *)
This signifies that the section being defined also contains all tests and mutants from other-section-name.
Command-Line Tool Flags
- -s <section>: Specify which sections properties and mutants to test
- -v: Verbose mode for debugging
- -failfast: Stop as soon as a problem is detected
- -color: Use colors on an ANSI-compatible terminal
- -cmd <command>: What compile command is used to compile the current directory if it is not make
- -top <name>: Specify the name of the top-level logical module. That should be the same as the -Q or -R directive in _CoqProject or Top which is the default
- -ocamlbuild <args>: Any arguments necessary to pass to ocamlbuild when compiling the extracted code (e.g. linked libraries)
- -nobase: Pass this option to not test the base mutant
- -m <number>: Pass this to only test a mutant with a specific id number
- -tag <name>: Pass this to only test a mutant with a specific tag
- -include <name>: Specify a to include in the compilation
- -exclude <names>: Specify files to be excluded from compilation. Must be the last argument passed.