summaryrefslogtreecommitdiff
path: root/theories/Relations/Relation_Operators.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Relations/Relation_Operators.v')
-rw-r--r--theories/Relations/Relation_Operators.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Relations/Relation_Operators.v b/theories/Relations/Relation_Operators.v
index 4c5a6519..87cd1e6f 100644
--- a/theories/Relations/Relation_Operators.v
+++ b/theories/Relations/Relation_Operators.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id: Relation_Operators.v 9610 2007-02-07 14:45:18Z herbelin $ i*)
+(*i $Id: Relation_Operators.v 10681 2008-03-16 13:40:45Z msozeau $ i*)
(****************************************************************************)
(* Bruno Barras, Cristina Cornes *)
@@ -83,9 +83,9 @@ Variable leA : A -> A -> Prop.
Variable leB : B -> B -> Prop.
Inductive le_AsB : A + B -> A + B -> Prop :=
- | le_aa : forall x y:A, leA x y -> le_AsB (inl B x) (inl B y)
- | le_ab : forall (x:A) (y:B), le_AsB (inl B x) (inr A y)
- | le_bb : forall x y:B, leB x y -> le_AsB (inr A x) (inr A y).
+ | le_aa : forall x y:A, leA x y -> le_AsB (inl _ x) (inl _ y)
+ | le_ab : forall (x:A) (y:B), le_AsB (inl _ x) (inr _ y)
+ | le_bb : forall x y:B, leB x y -> le_AsB (inr _ x) (inr _ y).
End Disjoint_Union.