aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/SeqProp.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Reals/SeqProp.v')
-rw-r--r--theories/Reals/SeqProp.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Reals/SeqProp.v b/theories/Reals/SeqProp.v
index 6f489f37f..e64d9cc4f 100644
--- a/theories/Reals/SeqProp.v
+++ b/theories/Reals/SeqProp.v
@@ -13,6 +13,7 @@ Require Rfunctions.
Require Rseries.
Require Classical.
Require Max.
+Import R_scope.
Definition Un_decreasing [Un:nat->R] : Prop := (n:nat) (Rle (Un (S n)) (Un n)).
Definition opp_seq [Un:nat->R] : nat->R := [n:nat]``-(Un n)``.