| changeset 33197 | de6285ebcc05 |
| child 34126 | 8a2c5d7aff51 |
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Nitpick_Examples/Nitpick_Examples.thy Fri Oct 23 18:59:24 2009 +0200 @@ -0,0 +1,14 @@ +(* Title: HOL/Nitpick_Examples/Nitpick_Examples.thy + Author: Jasmin Blanchette, TU Muenchen + Copyright 2009 + +Nitpick examples. +*) + +theory Nitpick_Examples +imports Core_Nits Datatype_Nits Induct_Nits Manual_Nits Mini_Nits Mono_Nits + Pattern_Nits Record_Nits Refute_Nits Special_Nits Tests_Nits + Typedef_Nits +begin + +end