diff options
author | Samuel Mimram <smimram@debian.org> | 2008-07-25 15:12:53 +0200 |
---|---|---|
committer | Samuel Mimram <smimram@debian.org> | 2008-07-25 15:12:53 +0200 |
commit | a0cfa4f118023d35b767a999d5a2ac4b082857b4 (patch) | |
tree | dabcac548e299fee1da464c93b3dba98484f45b1 /theories/Wellfounded | |
parent | 2281410e38ef99d025ea77194585a9bc019fdaa9 (diff) |
Imported Upstream version 8.2~beta3+dfsgupstream/8.2.beta3+dfsg
Diffstat (limited to 'theories/Wellfounded')
-rw-r--r-- | theories/Wellfounded/Disjoint_Union.v | 6 | ||||
-rw-r--r-- | theories/Wellfounded/Inclusion.v | 6 | ||||
-rw-r--r-- | theories/Wellfounded/Inverse_Image.v | 4 | ||||
-rw-r--r-- | theories/Wellfounded/Lexicographic_Exponentiation.v | 3 | ||||
-rw-r--r-- | theories/Wellfounded/Lexicographic_Product.v | 2 | ||||
-rw-r--r-- | theories/Wellfounded/Transitive_Closure.v | 2 | ||||
-rw-r--r-- | theories/Wellfounded/Union.v | 6 | ||||
-rw-r--r-- | theories/Wellfounded/Well_Ordering.v | 2 |
8 files changed, 15 insertions, 16 deletions
diff --git a/theories/Wellfounded/Disjoint_Union.v b/theories/Wellfounded/Disjoint_Union.v index 1e22730b..6adf629d 100644 --- a/theories/Wellfounded/Disjoint_Union.v +++ b/theories/Wellfounded/Disjoint_Union.v @@ -6,7 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Disjoint_Union.v 9245 2006-10-17 12:53:34Z notin $ i*) +(*i $Id: Disjoint_Union.v 10681 2008-03-16 13:40:45Z msozeau $ i*) (** Author: Cristina Cornes From : Constructing Recursion Operators in Type Theory @@ -15,7 +15,7 @@ Require Import Relation_Operators. Section Wf_Disjoint_Union. - Variables A B : Set. + Variables A B : Type. Variable leA : A -> A -> Prop. Variable leB : B -> B -> Prop. @@ -52,4 +52,4 @@ Section Wf_Disjoint_Union. apply (H0 b). Qed. -End Wf_Disjoint_Union.
\ No newline at end of file +End Wf_Disjoint_Union. diff --git a/theories/Wellfounded/Inclusion.v b/theories/Wellfounded/Inclusion.v index 44e07d0b..e5ef4a70 100644 --- a/theories/Wellfounded/Inclusion.v +++ b/theories/Wellfounded/Inclusion.v @@ -6,14 +6,14 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Inclusion.v 9245 2006-10-17 12:53:34Z notin $ i*) +(*i $Id: Inclusion.v 9642 2007-02-12 10:31:53Z herbelin $ i*) (** Author: Bruno Barras *) Require Import Relation_Definitions. Section WfInclusion. - Variable A : Set. + Variable A : Type. Variables R1 R2 : A -> A -> Prop. Lemma Acc_incl : inclusion A R1 R2 -> forall z:A, Acc R2 z -> Acc R1 z. @@ -29,4 +29,4 @@ Section WfInclusion. unfold well_founded in |- *; auto with sets. Qed. -End WfInclusion.
\ No newline at end of file +End WfInclusion. diff --git a/theories/Wellfounded/Inverse_Image.v b/theories/Wellfounded/Inverse_Image.v index 210cc757..29fe7bb2 100644 --- a/theories/Wellfounded/Inverse_Image.v +++ b/theories/Wellfounded/Inverse_Image.v @@ -6,13 +6,13 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Inverse_Image.v 9245 2006-10-17 12:53:34Z notin $ i*) +(*i $Id: Inverse_Image.v 9642 2007-02-12 10:31:53Z herbelin $ i*) (** Author: Bruno Barras *) Section Inverse_Image. - Variables A B : Set. + Variables A B : Type. Variable R : B -> B -> Prop. Variable f : A -> B. diff --git a/theories/Wellfounded/Lexicographic_Exponentiation.v b/theories/Wellfounded/Lexicographic_Exponentiation.v index efdf0495..4dfcb24b 100644 --- a/theories/Wellfounded/Lexicographic_Exponentiation.v +++ b/theories/Wellfounded/Lexicographic_Exponentiation.v @@ -6,14 +6,13 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Lexicographic_Exponentiation.v 9610 2007-02-07 14:45:18Z herbelin $ i*) +(*i $Id: Lexicographic_Exponentiation.v 9609 2007-02-07 14:42:26Z herbelin $ i*) (** Author: Cristina Cornes From : Constructing Recursion Operators in Type Theory L. Paulson JSC (1986) 2, 325-355 *) -Require Import Eqdep. Require Import List. Require Import Relation_Operators. Require Import Transitive_Closure. diff --git a/theories/Wellfounded/Lexicographic_Product.v b/theories/Wellfounded/Lexicographic_Product.v index 051c8127..818084b2 100644 --- a/theories/Wellfounded/Lexicographic_Product.v +++ b/theories/Wellfounded/Lexicographic_Product.v @@ -6,7 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Lexicographic_Product.v 9597 2007-02-06 19:44:05Z herbelin $ i*) +(*i $Id: Lexicographic_Product.v 9598 2007-02-06 19:45:52Z herbelin $ i*) (** Authors: Bruno Barras, Cristina Cornes *) diff --git a/theories/Wellfounded/Transitive_Closure.v b/theories/Wellfounded/Transitive_Closure.v index bd4e4fec..e552598c 100644 --- a/theories/Wellfounded/Transitive_Closure.v +++ b/theories/Wellfounded/Transitive_Closure.v @@ -6,7 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Transitive_Closure.v 9597 2007-02-06 19:44:05Z herbelin $ i*) +(*i $Id: Transitive_Closure.v 9598 2007-02-06 19:45:52Z herbelin $ i*) (** Author: Bruno Barras *) diff --git a/theories/Wellfounded/Union.v b/theories/Wellfounded/Union.v index 634576ad..8589c18f 100644 --- a/theories/Wellfounded/Union.v +++ b/theories/Wellfounded/Union.v @@ -6,7 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Union.v 9245 2006-10-17 12:53:34Z notin $ i*) +(*i $Id: Union.v 9642 2007-02-12 10:31:53Z herbelin $ i*) (** Author: Bruno Barras *) @@ -15,7 +15,7 @@ Require Import Relation_Definitions. Require Import Transitive_Closure. Section WfUnion. - Variable A : Set. + Variable A : Type. Variables R1 R2 : relation A. Notation Union := (union A R1 R2). @@ -72,4 +72,4 @@ Section WfUnion. apply Acc_union; auto with sets. Qed. -End WfUnion.
\ No newline at end of file +End WfUnion. diff --git a/theories/Wellfounded/Well_Ordering.v b/theories/Wellfounded/Well_Ordering.v index f691f2b7..af8832ec 100644 --- a/theories/Wellfounded/Well_Ordering.v +++ b/theories/Wellfounded/Well_Ordering.v @@ -6,7 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Well_Ordering.v 9597 2007-02-06 19:44:05Z herbelin $ i*) +(*i $Id: Well_Ordering.v 9598 2007-02-06 19:45:52Z herbelin $ i*) (** Author: Cristina Cornes. From: Constructing Recursion Operators in Type Theory |