| author | huffman |
| Wed, 10 Aug 2011 18:02:16 -0700 | |
| changeset 44142 | 8e27e0177518 |
| parent 37495 | 650fae5eea93 |
| child 45035 | 60d2c03d5c70 |
| permissions | -rw-r--r-- |
| 33197 | 1 |
(* Title: HOL/Nitpick_Examples/Tests_Nits.thy |
2 |
Author: Jasmin Blanchette, TU Muenchen |
|
|
35076
cc19e2aef17e
added hotel key card example for Nitpick, and renumber atoms in Nitpick's output for increased readability
blanchet
parents:
33232
diff
changeset
|
3 |
Copyright 2009, 2010 |
| 33197 | 4 |
|
5 |
Nitpick tests. |
|
6 |
*) |
|
7 |
||
8 |
header {* Nitpick Tests *}
|
|
9 |
||
10 |
theory Tests_Nits |
|
11 |
imports Main |
|
12 |
begin |
|
13 |
||
|
37495
650fae5eea93
make the Nitpick_Example theory processable even when Kodkodi is not installed;
blanchet
parents:
35076
diff
changeset
|
14 |
ML {* () |> getenv "KODKODI" <> "" ? Nitpick_Tests.run_all_tests *}
|
| 33197 | 15 |
|
16 |
end |