aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Relations/Operators_Properties.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-10-19 13:43:38 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-10-19 13:43:38 +0000
commitadd39fd4566c0e00293c2082077d08fb21178607 (patch)
treef0e0036098c54d9972c24b77581f587a1059068d /theories/Relations/Operators_Properties.v
parentcad1432683f0fa93efaf64f26803a44f64fd1bd0 (diff)
Retour en arrière sur la mise en paramètre du premier argument de
Coq.Relation.Relation_Operators.clos_refl_sym_trans car cela échange les arguments de rst_sym et casse la compatibilité (cf p.ex. Rocq/PTS). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11471 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Relations/Operators_Properties.v')
-rw-r--r--theories/Relations/Operators_Properties.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Relations/Operators_Properties.v b/theories/Relations/Operators_Properties.v
index 22582f75d..2ced22298 100644
--- a/theories/Relations/Operators_Properties.v
+++ b/theories/Relations/Operators_Properties.v
@@ -70,7 +70,7 @@ Section Properties.
apply Build_equivalence.
exact (rst_refl A R).
exact (rst_trans A R).
- exact (fun x y => rst_sym A R y x).
+ exact (rst_sym A R).
Qed.
(** Idempotency of the reflexive-symmetric-transitive closure operator *)