aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--theories/Wellfounded/Lexicographic_Product.v2
-rw-r--r--theories/Wellfounded/Well_Ordering.v2
2 files changed, 2 insertions, 2 deletions
diff --git a/theories/Wellfounded/Lexicographic_Product.v b/theories/Wellfounded/Lexicographic_Product.v
index 5fa24e2cc..157265047 100644
--- a/theories/Wellfounded/Lexicographic_Product.v
+++ b/theories/Wellfounded/Lexicographic_Product.v
@@ -45,7 +45,7 @@ Proof.
Apply H2.
Auto with sets.
- Injection H8. (*** BUG ***)
+ Injection H8.
Induction 2.
Injection H9.
Induction 2;Auto with sets.
diff --git a/theories/Wellfounded/Well_Ordering.v b/theories/Wellfounded/Well_Ordering.v
index ad616ecc0..e2da52b53 100644
--- a/theories/Wellfounded/Well_Ordering.v
+++ b/theories/Wellfounded/Well_Ordering.v
@@ -28,7 +28,7 @@ Proof.
Apply Acc_intro.
Elim a.
Intros.
- Inversion H0. (*** BUG ***)
+ Inversion H0.
Apply Acc_intro.
Generalize H4 ;Generalize H1 ;Generalize f0 ;Generalize v.
Rewrite -> H3.