rule subrelI (for nice Isar proofs of relation inequalities)
authorkrauss
Fri, 07 May 2010 15:03:53 +0200
changeset 36728 ae397b810c8b
parent 36726 47ba1770da8e
child 36729 f5b63d2bd8fa
rule subrelI (for nice Isar proofs of relation inequalities)
src/HOL/Relation.thy
--- a/src/HOL/Relation.thy	Fri May 07 09:59:59 2010 +0200
+++ b/src/HOL/Relation.thy	Fri May 07 15:03:53 2010 +0200
@@ -639,9 +639,16 @@
   done
 
 
-subsection {* Version of @{text lfp_induct} for binary relations *}
+subsection {* Miscellaneous *}
+
+text {* Version of @{thm[source] lfp_induct} for binary relations *}
 
 lemmas lfp_induct2 = 
   lfp_induct_set [of "(a, b)", split_format (complete)]
 
+text {* Version of @{thm[source] subsetI} for binary relations *}
+
+lemma subrelI: "(\<And>x y. (x, y) \<in> r \<Longrightarrow> (x, y) \<in> s) \<Longrightarrow> r \<subseteq> s"
+by auto
+
 end