src/HOL/Nitpick_Examples/Tests_Nits.thy
author blanchet
Tue, 27 Oct 2009 14:40:24 +0100
changeset 33224 f93390060bbe
parent 33197 de6285ebcc05
child 35073 cc19e2aef17e
permissions -rw-r--r--
internal renaming in Nitpick and fixed Kodkodi invokation on Linux;
renamed Nitpick's ML structures from NitpickXxx to Nitpick_Xxx and added KODKODI_JAVA_LIBRARY_PATH to LD_LIBRARY_PATH before invoking Kodkodi
     1 (*  Title:      HOL/Nitpick_Examples/Tests_Nits.thy
     2     Author:     Jasmin Blanchette, TU Muenchen
     3     Copyright   2009
     4 
     5 Nitpick tests.
     6 *)
     7 
     8 header {* Nitpick Tests *}
     9 
    10 theory Tests_Nits
    11 imports Main
    12 begin
    13 
    14 ML {* Nitpick_Tests.run_all_tests () *}
    15 
    16 end