aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Wellfounded/Disjoint_Union.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Wellfounded/Disjoint_Union.v')
-rw-r--r--theories/Wellfounded/Disjoint_Union.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Wellfounded/Disjoint_Union.v b/theories/Wellfounded/Disjoint_Union.v
index f6ce84f98..a86d19c09 100644
--- a/theories/Wellfounded/Disjoint_Union.v
+++ b/theories/Wellfounded/Disjoint_Union.v
@@ -21,7 +21,7 @@ Section Wf_Disjoint_Union.
Notation Le_AsB := (le_AsB A B leA leB).
- Lemma acc_A_sum : forall x:A, Acc leA x -> Acc Le_AsB (inl B x).
+ Lemma acc_A_sum : forall x:A, Acc leA x -> Acc Le_AsB (inl x).
Proof.
induction 1.
apply Acc_intro; intros y H2.
@@ -30,7 +30,7 @@ Section Wf_Disjoint_Union.
Qed.
Lemma acc_B_sum :
- well_founded leA -> forall x:B, Acc leB x -> Acc Le_AsB (inr A x).
+ well_founded leA -> forall x:B, Acc leB x -> Acc Le_AsB (inr x).
Proof.
induction 2.
apply Acc_intro; intros y H3.