From 7accc9b6e22a0f511cb36f6ab8563b811e0e0167 Mon Sep 17 00:00:00 2001 From: Matthieu Sozeau Date: Wed, 4 Jun 2014 17:27:00 +0200 Subject: Remove spurious Show in script. --- theories/Reals/Rfunctions.v | 1 - 1 file changed, 1 deletion(-) (limited to 'theories/Reals') 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. -- cgit v1.2.3