diff options
author | 2000-03-21 18:11:57 +0000 | |
---|---|---|
committer | 2000-03-21 18:11:57 +0000 | |
commit | 5c83e9be8a66f67628c022f2dec283a5b159b648 (patch) | |
tree | efc37a096236e763695a1885b616f3098cc2ab0a | |
parent | dd1601c0c197fb7601812717eb76aa98fb97308a (diff) |
Retour sur les anciens noms
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@348 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r-- | theories/Zarith/fast_integer.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Zarith/fast_integer.v b/theories/Zarith/fast_integer.v index 444d5e9a1..93b78f9e4 100644 --- a/theories/Zarith/fast_integer.v +++ b/theories/Zarith/fast_integer.v @@ -258,7 +258,7 @@ Theorem compare_convert1 : ~(compare x y SUPERIEUR) = EGAL /\ ~(compare x y INFERIEUR) = EGAL. Proof. Induction x;Induction y;Split;Simpl;Auto with arith; - (Discriminate Orelse (Elim (H y0); Auto with arith)). + (Discriminate Orelse (Elim (H p0); Auto with arith)). Save. Theorem compare_convert_EGAL : (x,y:positive) (compare x y EGAL) = EGAL -> x=y. |