aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Ranalysis5.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-04-16 12:15:42 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-04-16 12:16:32 +0200
commit635f559018f6a16caf5c6a75a1d38bb807e6a4c8 (patch)
tree7e40a2a638f0247984b2dea6b883f8b5ce32d10b /theories/Reals/Ranalysis5.v
parent5fb2050e424062540ffbf22de0838fafe4de0a41 (diff)
Fixing missing headers.
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 ba19e0a53..d876b5d8e 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-2012 *)
+(* \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.