add monotonicity rule for rtranclp
authorhoelzl
Tue, 07 Jul 2015 18:01:30 +0200
changeset 60681 9ce7463350a9
parent 60680 589ed01b94fe
child 60682 5a6cd2560549
add monotonicity rule for rtranclp
src/HOL/Transitive_Closure.thy
--- a/src/HOL/Transitive_Closure.thy	Tue Jul 07 00:48:42 2015 +0200
+++ b/src/HOL/Transitive_Closure.thy	Tue Jul 07 18:01:30 2015 +0200
@@ -104,6 +104,10 @@
    apply (rule_tac [2] rtranclp.rtrancl_into_rtrancl, blast+)
   done
 
+lemma mono_rtranclp[mono]:
+   "(\<And>a b. x a b \<longrightarrow> y a b) \<Longrightarrow> x^** a b \<longrightarrow> y^** a b"
+   using rtranclp_mono[of x y] by auto
+
 lemmas rtrancl_mono = rtranclp_mono [to_set]
 
 theorem rtranclp_induct [consumes 1, case_names base step, induct set: rtranclp]: