aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/SeqProp.v
diff options
context:
space:
mode:
authorGravatar Pierre Boutillier <pierre.boutillier@ens-lyon.org>2014-04-10 15:45:49 +0200
committerGravatar Pierre Boutillier <pierre.boutillier@ens-lyon.org>2014-04-10 16:25:08 +0200
commit6e66d8c551b5edcb33a9f3fbf744b2f82d944c50 (patch)
treed23b63653b8b2d58f20661fd5691ccac42e687fb /theories/Reals/SeqProp.v
parentf705a0b0ae587e323199c43e9669b4f96adf4d77 (diff)
No more Coersion in Init.
Diffstat (limited to 'theories/Reals/SeqProp.v')
-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 5254ff2cc..52657b401 100644
--- a/theories/Reals/SeqProp.v
+++ b/theories/Reals/SeqProp.v
@@ -27,7 +27,7 @@ Lemma growing_cv :
forall Un:nat -> R, Un_growing Un -> has_ub Un -> { l:R | Un_cv Un l }.
Proof.
intros Un Hug Heub.
- exists (projT1 (completeness (EUn Un) Heub (EUn_noempty Un))).
+ exists (proj1_sig (completeness (EUn Un) Heub (EUn_noempty Un))).
destruct (completeness _ Heub (EUn_noempty Un)) as (l, H).
now apply Un_cv_crit_lub.
Qed.