aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Cauchy_prod.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Reals/Cauchy_prod.v')
-rw-r--r--theories/Reals/Cauchy_prod.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/Reals/Cauchy_prod.v b/theories/Reals/Cauchy_prod.v
index cf962a0e2..c6926ec18 100644
--- a/theories/Reals/Cauchy_prod.v
+++ b/theories/Reals/Cauchy_prod.v
@@ -12,6 +12,7 @@ Require Rbase.
Require Rfunctions.
Require Rseries.
Require PartSum.
+Import R_scope.
(**********)
Lemma sum_N_predN : (An:nat->R;N:nat) (lt O N) -> (sum_f_R0 An N)==``(sum_f_R0 An (pred N)) + (An N)``.
@@ -342,4 +343,4 @@ Simpl; Symmetry; Apply S_pred with O; Assumption.
Inversion H.
Left; Reflexivity.
Right; Apply lt_le_trans with (1); [Apply lt_n_Sn | Exact H1].
-Qed. \ No newline at end of file
+Qed.