src/HOL/Inductive.thy
changeset 22218 30a8890d2967
parent 21018 e6b8d6784792
child 22783 e5f947e0ade8
--- a/src/HOL/Inductive.thy	Wed Jan 31 14:03:31 2007 +0100
+++ b/src/HOL/Inductive.thy	Wed Jan 31 16:05:10 2007 +0100
@@ -64,7 +64,7 @@
 setup OldInductivePackage.setup
 
 theorems basic_monos [mono] =
-  subset_refl imp_refl disj_mono conj_mono ex_mono all_mono if_def2
+  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
@@ -75,7 +75,7 @@
 setup InductivePackage.setup
 
 theorems [mono2] =
-  imp_refl disj_mono conj_mono ex_mono all_mono if_def2
+  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
   Ball_def Bex_def