From b22125319bf7ba65b0c5ce00124285351277895a Mon Sep 17 00:00:00 2001 From: herbelin Date: Fri, 19 Nov 2004 22:12:33 +0000 Subject: Généralisation à Type de certaines propriétés des relations MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@6331 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Relations/Relation_Operators.v | 12 ++++++------ 1 file changed, 6 insertions(+), 6 deletions(-) (limited to 'theories/Relations') diff --git a/theories/Relations/Relation_Operators.v b/theories/Relations/Relation_Operators.v index 1933655c9..86cd92b85 100755 --- a/theories/Relations/Relation_Operators.v +++ b/theories/Relations/Relation_Operators.v @@ -22,7 +22,7 @@ Require Import List. (** Some operators to build relations *) Section Transitive_Closure. - Variable A : Set. + Variable A : Type. Variable R : relation A. Inductive clos_trans : A -> A -> Prop := @@ -33,7 +33,7 @@ End Transitive_Closure. Section Reflexive_Transitive_Closure. - Variable A : Set. + Variable A : Type. Variable R : relation A. Inductive clos_refl_trans : relation A := @@ -46,7 +46,7 @@ End Reflexive_Transitive_Closure. Section Reflexive_Symetric_Transitive_Closure. - Variable A : Set. + Variable A : Type. Variable R : relation A. Inductive clos_refl_sym_trans : relation A := @@ -62,7 +62,7 @@ End Reflexive_Symetric_Transitive_Closure. Section Transposee. - Variable A : Set. + Variable A : Type. Variable R : relation A. Definition transp (x y:A) := R y x. @@ -70,7 +70,7 @@ End Transposee. Section Union. - Variable A : Set. + Variable A : Type. Variables R1 R2 : relation A. Definition union (x y:A) := R1 x y \/ R2 x y. @@ -164,4 +164,4 @@ End Lexicographic_Exponentiation. Hint Unfold transp union: sets v62. Hint Resolve t_step rt_step rt_refl rst_step rst_refl: sets v62. -Hint Immediate rst_sym: sets v62. \ No newline at end of file +Hint Immediate rst_sym: sets v62. -- cgit v1.2.3