src/HOL/Nitpick_Examples/Tests_Nits.thy
author boehmes
Thu, 27 May 2010 17:09:06 +0200
changeset 37155 e3f18cfc9829
parent 35076 cc19e2aef17e
child 37495 650fae5eea93
permissions -rw-r--r--
sort signature in SMT-LIB output (improves sharing of SMT certificates: goals of the same logical structure are translated into equal SMT-LIB benchmarks)

(*  Title:      HOL/Nitpick_Examples/Tests_Nits.thy
    Author:     Jasmin Blanchette, TU Muenchen
    Copyright   2009, 2010

Nitpick tests.
*)

header {* Nitpick Tests *}

theory Tests_Nits
imports Main
begin

ML {* Nitpick_Tests.run_all_tests () *}

end