aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:03 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:03 +0200
commit18512ba12400e30858ae19e5ef69b9590b96de06 (patch)
treed85d73110a1eb95b8873375cee0bd35821996657 /theories/Reals
parent3011cbfb224b3b2dfb72afd05094614b97a2128b (diff)
Revert "Temporary hack to compensate missing comma while re-printing tactic"
Diffstat (limited to 'theories/Reals')
-rw-r--r--theories/Reals/PSeries_reg.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Reals/PSeries_reg.v b/theories/Reals/PSeries_reg.v
index 3d29a5bbf..03ac6582b 100644
--- a/theories/Reals/PSeries_reg.v
+++ b/theories/Reals/PSeries_reg.v
@@ -54,7 +54,7 @@ rewrite Rplus_comm; apply Rplus_lt_compat_l, Rmult_lt_compat_r.
apply Rlt_trans with z; assumption.
destruct (boule_of_interval _ _ cmp) as [c [r [P1 P2]]].
assert (0 < /2) by (apply Rinv_0_lt_compat, Rlt_0_2).
-exists c; exists r; split.
+exists c, r; split.
destruct h; unfold Boule; simpl; apply Rabs_def1.
apply Rplus_lt_reg_l with c; rewrite P2;
replace (c + (z - c)) with (z * / 2 + z * / 2) by field.