aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-05-23 10:40:51 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-06-14 07:33:11 +0200
commit7668037a8daaef7bc8f1fc3225c2e6cc26cac0aa (patch)
tree2607253dc63558a4c8545a53e32ad140221e0560 /theories/Reals
parent180b3739bb6601ff9aaf951e4b87e0bb45341b77 (diff)
Remove deprecated options from the standard library.
Diffstat (limited to 'theories/Reals')
-rw-r--r--theories/Reals/SeqProp.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Reals/SeqProp.v b/theories/Reals/SeqProp.v
index 3697999f7..6a5233b64 100644
--- a/theories/Reals/SeqProp.v
+++ b/theories/Reals/SeqProp.v
@@ -150,7 +150,7 @@ Definition sequence_lb (Un:nat -> R) (pr:has_lb Un)
(* Compatibility *)
Notation sequence_majorant := sequence_ub (only parsing).
Notation sequence_minorant := sequence_lb (only parsing).
-Unset Standard Proposition Elimination Names.
+
Lemma Wn_decreasing :
forall (Un:nat -> R) (pr:has_ub Un), Un_decreasing (sequence_ub Un pr).
Proof.