src/HOL/Inductive.thy
changeset 33966 b863967f23ea
parent 33934 25d6a8982e37
parent 33963 977b94b64905
child 33968 f94fb13ecbb3
--- a/src/HOL/Inductive.thy	Fri Nov 27 08:42:50 2009 +0100
+++ b/src/HOL/Inductive.thy	Mon Nov 30 08:08:31 2009 +0100
@@ -261,18 +261,13 @@
 theorems basic_monos =
   subset_refl imp_refl disj_mono conj_mono ex_mono all_mono if_bool_eq_conj
   Collect_mono in_mono vimage_mono
-  imp_conv_disj not_not de_Morgan_disj de_Morgan_conj
-  not_all not_ex
-  Ball_def Bex_def
-  induct_rulify_fallback
 
 use "Tools/inductive.ML"
 setup Inductive.setup
 
 theorems [mono] =
   imp_refl disj_mono conj_mono ex_mono all_mono if_bool_eq_conj
-  imp_conv_disj not_not de_Morgan_disj de_Morgan_conj
-  not_all not_ex
+  imp_mono not_mono
   Ball_def Bex_def
   induct_rulify_fallback