| author | huffman | 
| Wed, 24 Aug 2011 11:56:57 -0700 | |
| changeset 44514 | d02b01e5ab8f | 
| parent 39221 | 70fd4a3c41ed | 
| child 45035 | 60d2c03d5c70 | 
| permissions | -rw-r--r-- | 
| 33197 | 1 | (* Title: HOL/Nitpick_Examples/Nitpick_Examples.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: 
34126diff
changeset | 3 | Copyright 2009, 2010 | 
| 33197 | 4 | |
| 5 | Nitpick examples. | |
| 6 | *) | |
| 7 | ||
| 8 | theory Nitpick_Examples | |
| 35076 
cc19e2aef17e
added hotel key card example for Nitpick, and renumber atoms in Nitpick's output for increased readability
 blanchet parents: 
34126diff
changeset | 9 | imports Core_Nits Datatype_Nits Hotel_Nits Induct_Nits Integer_Nits Manual_Nits | 
| 39221 
70fd4a3c41ed
remove "minipick" (the toy version of Nitpick) and some tests;
 blanchet parents: 
35076diff
changeset | 10 | Mono_Nits Pattern_Nits Record_Nits Refute_Nits Special_Nits Tests_Nits | 
| 
70fd4a3c41ed
remove "minipick" (the toy version of Nitpick) and some tests;
 blanchet parents: 
35076diff
changeset | 11 | Typedef_Nits | 
| 33197 | 12 | begin | 
| 13 | end |