aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-04 17:27:00 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-04 17:27:00 +0200
commit7accc9b6e22a0f511cb36f6ab8563b811e0e0167 (patch)
treea5d6fff43be7d7f923d9f22a721f0336c4464704 /theories/Reals
parentdbada2989e334756971c7bf69578c93b2e45643e (diff)
Remove spurious Show in script.
Diffstat (limited to 'theories/Reals')
-rw-r--r--theories/Reals/Rfunctions.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Reals/Rfunctions.v b/theories/Reals/Rfunctions.v
index 604160834..9beee06c5 100644
--- a/theories/Reals/Rfunctions.v
+++ b/theories/Reals/Rfunctions.v
@@ -741,7 +741,6 @@ Qed.
Lemma R_dist_sym : forall x y:R, R_dist x y = R_dist y x.
Proof.
unfold R_dist; intros; split_Rabs; try ring.
-Show.
generalize (Ropp_gt_lt_0_contravar (y - x) Hlt0); intro;
rewrite (Ropp_minus_distr y x) in H; generalize (Rlt_asym (x - y) 0 Hlt);
intro; unfold Rgt in H; exfalso; auto.