aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rtrigo_reg.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Reals/Rtrigo_reg.v')
-rw-r--r--theories/Reals/Rtrigo_reg.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Reals/Rtrigo_reg.v b/theories/Reals/Rtrigo_reg.v
index 2fdf96d0c..5a34dd7af 100644
--- a/theories/Reals/Rtrigo_reg.v
+++ b/theories/Reals/Rtrigo_reg.v
@@ -8,7 +8,7 @@
(*i $Id$ i*)
-Require RealsB.
+Require Rbase.
Require Rfunctions.
Require SeqSeries.
Require Rtrigo.
@@ -491,4 +491,4 @@ Qed.
Lemma derive_pt_cos : (x:R) ``(derive_pt cos x (derivable_pt_cos ?))==-(sin x)``.
Intros; Apply derive_pt_eq_0.
Apply derivable_pt_lim_cos.
-Qed. \ No newline at end of file
+Qed.