src/HOL/Nitpick_Examples/Nitpick_Examples.thy
author huffman
Wed, 24 Aug 2011 11:56:57 -0700
changeset 44514 d02b01e5ab8f
parent 39221 70fd4a3c41ed
child 45035 60d2c03d5c70
permissions -rw-r--r--
move geometric progression lemmas from Linear_Algebra.thy to Integration.thy where they are used

(*  Title:      HOL/Nitpick_Examples/Nitpick_Examples.thy
    Author:     Jasmin Blanchette, TU Muenchen
    Copyright   2009, 2010

Nitpick examples.
*)

theory Nitpick_Examples
imports Core_Nits Datatype_Nits Hotel_Nits Induct_Nits Integer_Nits Manual_Nits
        Mono_Nits Pattern_Nits Record_Nits Refute_Nits Special_Nits Tests_Nits
        Typedef_Nits
begin
end