src/HOL/HOL.thy
changeset 37264 8b931fb51cc6
parent 36945 9bec62c10714
child 37421 6cde0764bc03
--- a/src/HOL/HOL.thy	Tue Jun 01 15:37:14 2010 +0200
+++ b/src/HOL/HOL.thy	Tue Jun 01 15:38:47 2010 +0200
@@ -2033,11 +2033,6 @@
   val name = "nitpick_psimp"
   val description = "partial equational specification of constants as needed by Nitpick"
 )
-structure Nitpick_Intros = Named_Thms
-(
-  val name = "nitpick_intro"
-  val description = "introduction rules for (co)inductive predicates as needed by Nitpick"
-)
 structure Nitpick_Choice_Specs = Named_Thms
 (
   val name = "nitpick_choice_spec"
@@ -2049,7 +2044,6 @@
   Nitpick_Defs.setup
   #> Nitpick_Simps.setup
   #> Nitpick_Psimps.setup
-  #> Nitpick_Intros.setup
   #> Nitpick_Choice_Specs.setup
 *}