changeset 47937 | 70375fa2679d |
parent 47436 | d8fad618a67a |
child 48253 | 4410a709913c |
--- a/src/HOL/Relation.thy Wed May 16 19:15:45 2012 +0200 +++ b/src/HOL/Relation.thy Wed May 16 19:17:20 2012 +0200 @@ -173,6 +173,11 @@ obtains "r x x" using assms by (auto dest: refl_onD simp add: reflp_def) +lemma reflpD: + assumes "reflp r" + shows "r x x" + using assms by (auto elim: reflpE) + lemma refl_on_Int: "refl_on A r ==> refl_on B s ==> refl_on (A \<inter> B) (r \<inter> s)" by (unfold refl_on_def) blast