aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Num/Params.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
commit67f72c93f5f364591224a86c52727867e02a8f71 (patch)
treeecf630daf8346e77e6620233d8f3e6c18a0c9b3c /theories/Num/Params.v
parentb239b208eb9a66037b0c629cf7ccb6e4b110636a (diff)
option -dump-glob pour coqdoc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2474 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Num/Params.v')
-rw-r--r--theories/Num/Params.v15
1 files changed, 12 insertions, 3 deletions
diff --git a/theories/Num/Params.v b/theories/Num/Params.v
index a7be171b8..91c132095 100644
--- a/theories/Num/Params.v
+++ b/theories/Num/Params.v
@@ -1,7 +1,16 @@
-(*i $Id $ i*)
+(***********************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
+(* \VV/ *************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(***********************************************************************)
-(*s
+(*i $Id$ i*)
+
+(**
Axiomatisation of a numerical set
+
It will be instantiated by Z and R later on
We choose to introduce many operation to allow flexibility in definition
([S] is primitive in the definition of [nat] while [add] and [one]
@@ -14,7 +23,7 @@ Parameter one:N.
Parameter add:N->N->N.
Parameter S:N->N.
-(*s Relations, equality is defined separately *)
+(** Relations, equality is defined separately *)
Parameter lt,le,gt,ge:N->N->Prop.