diff options
Diffstat (limited to 'theories/Relations/Relation_Operators.v')
-rw-r--r-- | theories/Relations/Relation_Operators.v | 6 |
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Relations/Relation_Operators.v b/theories/Relations/Relation_Operators.v index 8d76b4f4e..61b70ba68 100644 --- a/theories/Relations/Relation_Operators.v +++ b/theories/Relations/Relation_Operators.v @@ -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. |