add lemma
authorAndreas Lochbihler
Wed, 11 Feb 2015 14:07:28 +0100
changeset 59518 28cfc60dea7a
parent 59517 22c9e6cf5572
child 59519 2fb0c0fc62a3
add lemma
src/HOL/Relation.thy
--- a/src/HOL/Relation.thy	Wed Feb 11 14:03:05 2015 +0100
+++ b/src/HOL/Relation.thy	Wed Feb 11 14:07:28 2015 +0100
@@ -426,6 +426,8 @@
   "transp r \<longleftrightarrow> trans {(x, y). r x y}"
   by (simp add: trans_def transp_def)
 
+lemma transp_equality [simp]: "transp op ="
+by(auto intro: transpI)
 
 subsubsection {* Totality *}