src/HOL/Set.thy
changeset 13421 8fcdf4a26468
parent 13113 5eb9be7b72a5
child 13462 56610e2ba220
--- a/src/HOL/Set.thy	Wed Jul 24 22:14:42 2002 +0200
+++ b/src/HOL/Set.thy	Wed Jul 24 22:15:55 2002 +0200
@@ -960,16 +960,16 @@
 
 text {* \medskip Monotonicity. *}
 
-lemma mono_Un: "mono f ==> f A \<union> f B \<subseteq> f (A \<union> B)"
+lemma mono_Un: includes mono shows "f A \<union> f B \<subseteq> f (A \<union> B)"
   apply (rule Un_least)
-   apply (erule Un_upper1 [THEN [2] monoD])
-  apply (erule Un_upper2 [THEN [2] monoD])
+   apply (rule Un_upper1 [THEN mono])
+  apply (rule Un_upper2 [THEN mono])
   done
 
-lemma mono_Int: "mono f ==> f (A \<inter> B) \<subseteq> f A \<inter> f B"
+lemma mono_Int: includes mono shows "f (A \<inter> B) \<subseteq> f A \<inter> f B"
   apply (rule Int_greatest)
-   apply (erule Int_lower1 [THEN [2] monoD])
-  apply (erule Int_lower2 [THEN [2] monoD])
+   apply (rule Int_lower1 [THEN mono])
+  apply (rule Int_lower2 [THEN mono])
   done