added lemma
authornipkow
Sat, 08 Feb 2025 17:45:49 +0100
changeset 82116 ab0030db61fd
parent 82103 eebb8270b3cc
child 82117 0c54f3c06174
added lemma
src/HOL/Transitive_Closure.thy
--- a/src/HOL/Transitive_Closure.thy	Sat Feb 08 11:18:30 2025 +0100
+++ b/src/HOL/Transitive_Closure.thy	Sat Feb 08 17:45:49 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)