| author | wenzelm | 
| Tue, 25 Mar 2025 23:05:15 +0100 | |
| changeset 82407 | fcc0f74ac086 | 
| parent 74844 | 90242c744a1a | 
| permissions | -rw-r--r-- | 
| 33197 | 1  | 
(* Title: HOL/Nitpick_Examples/Tests_Nits.thy  | 
2  | 
Author: Jasmin Blanchette, TU Muenchen  | 
|
| 45035 | 3  | 
Copyright 2009-2011  | 
| 33197 | 4  | 
|
5  | 
Nitpick tests.  | 
|
6  | 
*)  | 
|
7  | 
||
| 63167 | 8  | 
section \<open>Nitpick Tests\<close>  | 
| 33197 | 9  | 
|
10  | 
theory Tests_Nits  | 
|
11  | 
imports Main  | 
|
12  | 
begin  | 
|
13  | 
||
| 
74844
 
90242c744a1a
maintain option kodkod_scala within theory context, to allow local modification;
 
wenzelm 
parents: 
63167 
diff
changeset
 | 
14  | 
ML \<open>if getenv "KODKODI" = "" then () else Nitpick_Tests.run_all_tests \<^context>\<close>  | 
| 33197 | 15  | 
|
16  | 
end  |