src/HOL/Inductive.thy
changeset 61337 4645502c3c64
parent 61076 bdc1e2f0a86a
child 61799 4cf66f21b764
--- a/src/HOL/Inductive.thy	Tue Oct 06 13:31:44 2015 +0200
+++ b/src/HOL/Inductive.thy	Tue Oct 06 15:14:28 2015 +0200
@@ -343,13 +343,13 @@
 
 text \<open>Package setup.\<close>
 
-theorems basic_monos =
+lemmas basic_monos =
   subset_refl imp_refl disj_mono conj_mono ex_mono all_mono if_bool_eq_conj
   Collect_mono in_mono vimage_mono
 
 ML_file "Tools/inductive.ML"
 
-theorems [mono] =
+lemmas [mono] =
   imp_refl disj_mono conj_mono ex_mono all_mono if_bool_eq_conj
   imp_mono not_mono
   Ball_def Bex_def