From 2f2b225969cf4b06ff60d4a5862cf8404bb11268 Mon Sep 17 00:00:00 2001 From: herbelin Date: Wed, 9 Apr 2003 10:55:08 +0000 Subject: Suppression de l'étage "Import nat/Z/R_scope". "Open Scope" remplace "Import". MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3877 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Reals/Cos_plus.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/Reals/Cos_plus.v') diff --git a/theories/Reals/Cos_plus.v b/theories/Reals/Cos_plus.v index e366adb38..ae650225f 100644 --- a/theories/Reals/Cos_plus.v +++ b/theories/Reals/Cos_plus.v @@ -14,8 +14,8 @@ Require SeqSeries. Require Rtrigo_def. Require Cos_rel. Require Max. -Import nat_scope. -Import R_scope. +V7only [Import nat_scope.]. +V7only [Import R_scope.]. Definition Majxy [x,y:R] : nat->R := [n:nat](Rdiv (pow (Rmax R1 (Rmax (Rabsolu x) (Rabsolu y))) (mult (4) (S n))) (INR (fact n))). -- cgit v1.2.3