merged
authornipkow
Sat, 08 Feb 2025 17:46:10 +0100
changeset 82117 0c54f3c06174
parent 82115 bb6a3b379f6a (current diff)
parent 82116 ab0030db61fd (diff)
child 82118 f798a913d729
merged
--- a/src/HOL/Transitive_Closure.thy	Sat Feb 08 17:44:04 2025 +0100
+++ b/src/HOL/Transitive_Closure.thy	Sat Feb 08 17:46:10 2025 +0100
@@ -676,6 +676,9 @@
 lemma rtrancl_empty [simp]: "{}\<^sup>* = Id"
   by (rule subst [OF reflcl_trancl]) simp
 
+lemma rtrancl__Id[simp]: "Id\<^sup>* = Id"
+using rtrancl_empty rtrancl_idemp[of "{}"] by (simp)
+
 lemma rtranclpD: "R\<^sup>*\<^sup>* a b \<Longrightarrow> a = b \<or> a \<noteq> b \<and> R\<^sup>+\<^sup>+ a b"
   by (force simp: reflclp_tranclp [symmetric] simp del: reflclp_tranclp)