aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Relations
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-06-01 12:02:49 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-06-04 18:42:22 +0200
commit90fc6f45fa1a4ef5251046d8b4e4249164afa60b (patch)
tree48be98a97cb2f3c4d0fb66dcf4079c87f9ff80b4 /theories/Relations
parent7accc9b6e22a0f511cb36f6ab8563b811e0e0167 (diff)
Small lemma about Relations.
Diffstat (limited to 'theories/Relations')
-rw-r--r--theories/Relations/Operators_Properties.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/theories/Relations/Operators_Properties.v b/theories/Relations/Operators_Properties.v
index e599669f8..c2cd9628b 100644
--- a/theories/Relations/Operators_Properties.v
+++ b/theories/Relations/Operators_Properties.v
@@ -403,6 +403,13 @@ Section Properties.
End Equivalences.
+ Lemma clos_trans_transp_permute : forall x y,
+ transp _ (clos_trans R) x y <-> clos_trans (transp _ R) x y.
+ Proof.
+ split; induction 1;
+ (apply t_step; assumption) || eapply t_trans; eassumption.
+ Qed.
+
End Properties.
(* begin hide *)