aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-14 07:19:02 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-14 07:19:02 +0000
commit8ddd9ba6efcd32a13b4517a4e80c5fc035a951a8 (patch)
tree576a3ab530c2753ff4f9d1c0a149948e0722dfd8
parent172ee7f67a3aa8f8888905bee3c153cae543fcd5 (diff)
Deplacement de le_minus de fast_integer vers Minus
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4162 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--theories/ZArith/fast_integer.v8
1 files changed, 0 insertions, 8 deletions
diff --git a/theories/ZArith/fast_integer.v b/theories/ZArith/fast_integer.v
index 4026ba222..334dc050f 100644
--- a/theories/ZArith/fast_integer.v
+++ b/theories/ZArith/fast_integer.v
@@ -1224,14 +1224,6 @@ Intros x y;Split; [
Trivial with arith Orelse (Intros H2;Discriminate H2)]))].
Qed.
-Theorem le_minus: (i,h:nat) (le (minus i h) i).
-Proof.
-Intros i h;Pattern i h; Apply nat_double_ind; [
- Auto with arith
-| Auto with arith
-| Intros m n H; Simpl; Apply le_trans with m:=m; Auto with arith ].
-Qed.
-
Lemma ZL16: (p,q:positive)(lt (minus (convert p) (convert q)) (convert p)).
Proof.
Intros p q; Elim (ZL4 p);Elim (ZL4 q); Intros h H1 i H2;