| author | wenzelm |
| Tue, 04 May 2010 20:26:53 +0200 | |
| changeset 36650 | d65f07abfa7c |
| parent 35076 | cc19e2aef17e |
| child 37495 | 650fae5eea93 |
| 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 |
||
|
33232
f93390060bbe
internal renaming in Nitpick and fixed Kodkodi invokation on Linux;
blanchet
parents:
33197
diff
changeset
|
14 |
ML {* Nitpick_Tests.run_all_tests () *}
|
| 33197 | 15 |
|
16 |
end |