From 90fc6f45fa1a4ef5251046d8b4e4249164afa60b Mon Sep 17 00:00:00 2001 From: Hugo Herbelin Date: Sun, 1 Jun 2014 12:02:49 +0200 Subject: Small lemma about Relations. --- theories/Relations/Operators_Properties.v | 7 +++++++ 1 file changed, 7 insertions(+) (limited to 'theories/Relations') 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 *) -- cgit v1.2.3