src/HOL/Relation.thy
changeset 61630 608520e0e8e2
parent 61424 c3658c18b7bc
child 61799 4cf66f21b764
--- a/src/HOL/Relation.thy	Wed Nov 11 09:21:56 2015 +0100
+++ b/src/HOL/Relation.thy	Wed Nov 11 09:48:24 2015 +0100
@@ -219,6 +219,9 @@
 lemma reflp_equality [simp]: "reflp op ="
 by(simp add: reflp_def)
 
+lemma reflp_mono: "\<lbrakk> reflp R; \<And>x y. R x y \<longrightarrow> Q x y \<rbrakk> \<Longrightarrow> reflp Q"
+by(auto intro: reflpI dest: reflpD)
+
 subsubsection \<open>Irreflexivity\<close>
 
 definition irrefl :: "'a rel \<Rightarrow> bool"
@@ -676,6 +679,8 @@
 lemma eq_OO: "op= OO R = R"
 by blast
 
+lemma OO_eq: "R OO op = = R"
+by blast
 
 subsubsection \<open>Converse\<close>