aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Wellfounded
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/Wellfounded
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/Wellfounded')
-rw-r--r--theories/Wellfounded/Disjoint_Union.v9
-rw-r--r--theories/Wellfounded/Inclusion.v4
-rw-r--r--theories/Wellfounded/Inverse_Image.v4
-rw-r--r--theories/Wellfounded/Lexicographic_Exponentiation.v10
-rw-r--r--theories/Wellfounded/Lexicographic_Product.v11
-rw-r--r--theories/Wellfounded/Transitive_Closure.v4
-rw-r--r--theories/Wellfounded/Union.v4
-rw-r--r--theories/Wellfounded/Well_Ordering.v14
8 files changed, 21 insertions, 39 deletions
diff --git a/theories/Wellfounded/Disjoint_Union.v b/theories/Wellfounded/Disjoint_Union.v
index 7de40a413..5cb4b79d5 100644
--- a/theories/Wellfounded/Disjoint_Union.v
+++ b/theories/Wellfounded/Disjoint_Union.v
@@ -8,12 +8,9 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Cristina Cornes *)
-(* *)
-(* From : Constructing Recursion Operators in Type Theory *)
-(* L. Paulson JSC (1986) 2, 325-355 *)
-(****************************************************************************)
+(** Author: Cristina Cornes
+ From : Constructing Recursion Operators in Type Theory
+ L. Paulson JSC (1986) 2, 325-355 *)
Require Relation_Operators.
diff --git a/theories/Wellfounded/Inclusion.v b/theories/Wellfounded/Inclusion.v
index 66ef2346e..db9cfe227 100644
--- a/theories/Wellfounded/Inclusion.v
+++ b/theories/Wellfounded/Inclusion.v
@@ -8,9 +8,7 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Bruno Barras *)
-(****************************************************************************)
+(** Author: Bruno Barras *)
Require Relation_Definitions.
diff --git a/theories/Wellfounded/Inverse_Image.v b/theories/Wellfounded/Inverse_Image.v
index bc87acd98..3e4bca83f 100644
--- a/theories/Wellfounded/Inverse_Image.v
+++ b/theories/Wellfounded/Inverse_Image.v
@@ -8,9 +8,7 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Bruno Barras *)
-(****************************************************************************)
+(** Author: Bruno Barras *)
Section Inverse_Image.
diff --git a/theories/Wellfounded/Lexicographic_Exponentiation.v b/theories/Wellfounded/Lexicographic_Exponentiation.v
index 4ccc9e68d..ad157ea9d 100644
--- a/theories/Wellfounded/Lexicographic_Exponentiation.v
+++ b/theories/Wellfounded/Lexicographic_Exponentiation.v
@@ -8,12 +8,10 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Cristina Cornes *)
-(* *)
-(* From : Constructing Recursion Operators in Type Theory *)
-(* L. Paulson JSC (1986) 2, 325-355 *)
-(****************************************************************************)
+(** Author: Cristina Cornes
+
+ From : Constructing Recursion Operators in Type Theory
+ L. Paulson JSC (1986) 2, 325-355 *)
Require Eqdep.
Require PolyList.
diff --git a/theories/Wellfounded/Lexicographic_Product.v b/theories/Wellfounded/Lexicographic_Product.v
index 01b442a85..c57a75133 100644
--- a/theories/Wellfounded/Lexicographic_Product.v
+++ b/theories/Wellfounded/Lexicographic_Product.v
@@ -8,18 +8,15 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Bruno Barras Cristina Cornes *)
-(* *)
-(****************************************************************************)
+(** Authors: Bruno Barras,Cristina Cornes *)
Require Eqdep.
Require Relation_Operators.
Require Transitive_Closure.
-(* From : Constructing Recursion Operators in Type Theory
- L. Paulson JSC (1986) 2, 325-355
-*)
+(** From : Constructing Recursion Operators in Type Theory
+ L. Paulson JSC (1986) 2, 325-355 *)
+
Section WfLexicographic_Product.
Variable A:Set.
Variable B:A->Set.
diff --git a/theories/Wellfounded/Transitive_Closure.v b/theories/Wellfounded/Transitive_Closure.v
index 992099809..1cb9848f6 100644
--- a/theories/Wellfounded/Transitive_Closure.v
+++ b/theories/Wellfounded/Transitive_Closure.v
@@ -8,9 +8,7 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Bruno Barras *)
-(****************************************************************************)
+(** Author: Bruno Barras *)
Require Relation_Definitions.
Require Relation_Operators.
diff --git a/theories/Wellfounded/Union.v b/theories/Wellfounded/Union.v
index 1a3625b01..576c83cb4 100644
--- a/theories/Wellfounded/Union.v
+++ b/theories/Wellfounded/Union.v
@@ -8,9 +8,7 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Bruno Barras *)
-(****************************************************************************)
+(** Author: Bruno Barras *)
Require Relation_Operators.
Require Relation_Definitions.
diff --git a/theories/Wellfounded/Well_Ordering.v b/theories/Wellfounded/Well_Ordering.v
index ba9910440..ebd4925d1 100644
--- a/theories/Wellfounded/Well_Ordering.v
+++ b/theories/Wellfounded/Well_Ordering.v
@@ -8,12 +8,9 @@
(*i $Id$ i*)
-(****************************************************************************)
-(* Cristina Cornes *)
-(* *)
-(* From: Constructing Recursion Operators in Type Theory *)
-(* L. Paulson JSC (1986) 2, 325-355 *)
-(****************************************************************************)
+(** Author: Cristina Cornes.
+ From: Constructing Recursion Operators in Type Theory
+ L. Paulson JSC (1986) 2, 325-355 *)
Require Eqdep.
@@ -51,8 +48,9 @@ End WellOrdering.
Section Characterisation_wf_relations.
-(* wellfounded relations are the inverse image of wellordering types *)
-(* in course of development *)
+
+(** Wellfounded relations are the inverse image of wellordering types *)
+(* in course of development *)
Variable A:Set.