aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-19 17:57:40 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-19 17:57:40 +0000
commita3958897600963d2529772f43b029f1579524e95 (patch)
tree010493f2b0028d6510f952c3b6eb0c425bcbfa05
parent0bec25a0f6e90429d59d20e42cacac3a9bee72a6 (diff)
Restauration compatibilite 7.4 pour le Hint Unfold Rgt
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4951 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--theories/Reals/RIneq.v1
-rw-r--r--theories/Reals/Rdefinitions.v2
2 files changed, 1 insertions, 2 deletions
diff --git a/theories/Reals/RIneq.v b/theories/Reals/RIneq.v
index 1ada96892..313e22560 100644
--- a/theories/Reals/RIneq.v
+++ b/theories/Reals/RIneq.v
@@ -1407,6 +1407,7 @@ Lemma eq_IZR_R0:(z:Z)``(IZR z)==0``->`z=0`.
NewDestruct z; Simpl; Intros; Auto with zarith.
Case (Rlt_not_eq ``0`` (INR (convert p))); Auto with real.
Case (Rlt_not_eq ``-(INR (convert p))`` ``0`` ); Auto with real.
+Apply Rgt_RoppO. Unfold Rgt; Apply INR_pos.
Qed.
(**********)
diff --git a/theories/Reals/Rdefinitions.v b/theories/Reals/Rdefinitions.v
index fc1e36631..75a082cfc 100644
--- a/theories/Reals/Rdefinitions.v
+++ b/theories/Reals/Rdefinitions.v
@@ -67,5 +67,3 @@ V8Notation "x <= y <= z" := (Rle x y)/\(Rle y z) : R_scope.
V8Notation "x <= y < z" := (Rle x y)/\(Rlt y z) : R_scope.
V8Notation "x < y < z" := (Rlt x y)/\(Rlt y z) : R_scope.
V8Notation "x < y <= z" := (Rlt x y)/\(Rle y z) : R_scope.
-
-Hints Unfold Rgt : real.