src/HOL/Transitive_Closure.thy
changeset 76750 f70a7ff13b10
parent 76675 0d7a9e4e1d61
child 76751 66f17783913b
--- a/src/HOL/Transitive_Closure.thy	Mon Dec 19 16:00:49 2022 +0100
+++ b/src/HOL/Transitive_Closure.thy	Mon Dec 19 16:05:57 2022 +0100
@@ -85,8 +85,8 @@
 lemma trans_reflclI[simp]: "trans r \<Longrightarrow> trans (r\<^sup>=)"
   unfolding trans_def by blast
 
-lemma transp_reflclp[simp]: "transp R \<Longrightarrow> transp R\<^sup>=\<^sup>="
-  unfolding transp_def by blast
+lemma transp_on_reflclp[simp]: "transp_on A R \<Longrightarrow> transp_on A R\<^sup>=\<^sup>="
+  by (auto intro: transp_onI dest: transp_onD)
 
 lemma reflclp_idemp [simp]: "(P\<^sup>=\<^sup>=)\<^sup>=\<^sup>= = P\<^sup>=\<^sup>="
   by blast