aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Wellfounded
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-21 16:41:05 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-21 16:41:05 +0000
commit05b6e6ae8247b047b96f50dfcde59d619500d50d (patch)
tree4d05ad2b650267b8bd68eca8309fc20c0e31ee9b /theories/Wellfounded
parent2e364ae6c6c3fd99636d5d99104d0d01fda2a438 (diff)
Nettoyage
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@903 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Wellfounded')
-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.