aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rbase.v
diff options
context:
space:
mode:
authorGravatar courant <courant@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-21 15:07:27 +0000
committerGravatar courant <courant@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-21 15:07:27 +0000
commit6de9782f097b11b023629abfebae01aa9cff98c1 (patch)
tree0ff110071d2b11dd3ba53df14e5199ac262f91ae /theories/Reals/Rbase.v
parent9bd0183e7b6faa97dbaf2d6b016f4b0dc74e1a8c (diff)
Intuition ne fait plus de Unfold des constantes (il faut les faire
soi-même si nécessaire) : l'idée est d'avoir un comportement clair et toujours aussi rapide que possible. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2559 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rbase.v')
-rw-r--r--theories/Reals/Rbase.v27
1 files changed, 17 insertions, 10 deletions
diff --git a/theories/Reals/Rbase.v b/theories/Reals/Rbase.v
index c1f0feb9a..ca1853405 100644
--- a/theories/Reals/Rbase.v
+++ b/theories/Reals/Rbase.v
@@ -70,7 +70,7 @@ Hints Resolve imp_not_Req : real.
(**********)
Lemma Req_EM:(r1,r2:R)(r1==r2)\/``r1<>r2``.
-Intros ; Generalize (total_order_T r1 r2) ; Intuition EAuto with real.
+Intros ; Generalize (total_order_T r1 r2) imp_not_Req ; Intuition EAuto 3.
Save.
Hints Resolve Req_EM : real.
@@ -91,7 +91,7 @@ Save.
(**********)
Lemma Rlt_le:(r1,r2:R)``r1<r2``-> ``r1<=r2``.
-Intuition Auto.
+Intros ; Red ; Tauto.
Save.
Hints Resolve Rlt_le : real.
@@ -107,14 +107,15 @@ Save.
(**********)
Lemma not_Rle:(r1,r2:R)~(``r1<=r2``)->``r1>r2``.
-Intros r1 r2 ; Generalize (total_order r1 r2) ; Tauto.
+Intros r1 r2 ; Generalize (total_order r1 r2) ; Unfold Rle; Tauto.
Save.
Hints Immediate Rle_ge Rge_le not_Rle : real.
(**********)
Lemma Rlt_le_not:(r1,r2:R)``r2<r1``->~(``r1<=r2``).
-Intros r1 r2 ; Generalize (Rlt_antisym r1 r2) (imp_not_Req r1 r2) ; Intuition.
+Generalize Rlt_antisym imp_not_Req ; Unfold Rle.
+Intuition EAuto 3.
Save.
Lemma Rle_not:(r1,r2:R)``r1>r2`` -> ~(``r1<=r2``).
@@ -123,12 +124,13 @@ Proof Rlt_le_not.
Hints Immediate Rlt_le_not : real.
Lemma Rle_not_lt: (r1, r2:R) ``r2 <= r1`` ->~ (``r1<r2``).
-Intros r1 r2. Generalize (Rlt_antisym r1 r2) (imp_not_Req r1 r2); Intuition.
+Intros r1 r2. Generalize (Rlt_antisym r1 r2) (imp_not_Req r1 r2).
+Unfold Rle; Intuition.
Save.
(**********)
Lemma Rlt_ge_not:(r1,r2:R)``r1<r2``->~(``r1>=r2``).
-Generalize Rlt_le_not. Intuition EAuto 3.
+Generalize Rlt_le_not. Unfold Rle Rge. Intuition EAuto 3.
Save.
Hints Immediate Rlt_ge_not : real.
@@ -155,7 +157,7 @@ Save.
Hints Immediate eq_Rge_sym : real.
Lemma Rle_antisym : (r1,r2:R)``r1<=r2`` -> ``r2<=r1``-> r1==r2.
-Intros r1 r2; Generalize (Rlt_antisym r1 r2) ; Intuition.
+Intros r1 r2; Generalize (Rlt_antisym r1 r2) ; Unfold Rle ; Intuition.
Save.
Hints Resolve Rle_antisym : real.
@@ -171,17 +173,20 @@ Save.
(**********)
Lemma Rle_trans:(r1,r2,r3:R) ``r1<=r2``->``r2<=r3``->``r1<=r3``.
Generalize trans_eqT Rlt_trans Rlt_rew.
+Unfold Rle.
Intuition EAuto 2.
Save.
(**********)
Lemma Rle_lt_trans:(r1,r2,r3:R)``r1<=r2``->``r2<r3``->``r1<r3``.
-Generalize Rlt_trans Rlt_rew. Intuition EAuto 2.
+Generalize Rlt_trans Rlt_rew.
+Unfold Rle.
+Intuition EAuto 2.
Save.
(**********)
Lemma Rlt_le_trans:(r1,r2,r3:R)``r1<r2``->``r2<=r3``->``r1<r3``.
-Generalize Rlt_trans Rlt_rew; Intuition EAuto 2.
+Generalize Rlt_trans Rlt_rew; Unfold Rle; Intuition EAuto 2.
Save.
@@ -192,7 +197,9 @@ Save.
(**********)
Lemma total_order_Rle:(r1,r2:R)(sumboolT ``r1<=r2`` ~(``r1<=r2``)).
-Intros r1 r2; Generalize (total_order_T r1 r2);Intuition EAuto with real.
+Intros r1 r2.
+Generalize (total_order_T r1 r2) (imp_not_Req r1 r2).
+Intuition EAuto 4 with real.
Save.
(**********)