summaryrefslogtreecommitdiff
path: root/theories/Reals/Ranalysis5.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Reals/Ranalysis5.v')
-rw-r--r--theories/Reals/Ranalysis5.v10
1 files changed, 9 insertions, 1 deletions
diff --git a/theories/Reals/Ranalysis5.v b/theories/Reals/Ranalysis5.v
index c8a2e1a8..5c3b03fa 100644
--- a/theories/Reals/Ranalysis5.v
+++ b/theories/Reals/Ranalysis5.v
@@ -1,3 +1,11 @@
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2014 *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
+
Require Import Rbase.
Require Import Ranalysis_reg.
Require Import Rfunctions.
@@ -1345,4 +1353,4 @@ assert (Main : Rabs ((f (x+h) - fn N (x+h)) - (f x - fn N x) + (fn N (x+h) - fn
field ; apply Rgt_not_eq ; apply Rabs_pos_lt ; assumption.
assumption.
field. assumption.
-Qed. \ No newline at end of file
+Qed.