aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/TheoryList.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-05-28 16:21:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-05-28 16:21:04 +0000
commit10fa54f60acdfc8de6b59659f9fa8bc1ed3c18e6 (patch)
tree3cba1b1fb761818bb593e4c5d118e0ce9e49792d /theories/Lists/TheoryList.v
parentfd65ef00907710b3b036abf263516cfa872feb33 (diff)
- Déplacement des types paramétriques prod, sum, option, identity,
sig, sig2, sumor, list et vector dans Type - Branchement de prodT/listT vers les nouveaux prod/list - Abandon sigS/sigS2 au profit de sigT et du nouveau sigT2 - Changements en conséquence dans les théories (notamment Field_Tactic), ainsi que dans les modules ML Coqlib/Equality/Hipattern/Field git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8866 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/TheoryList.v')
-rw-r--r--theories/Lists/TheoryList.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Lists/TheoryList.v b/theories/Lists/TheoryList.v
index 26eae1a05..226d07149 100644
--- a/theories/Lists/TheoryList.v
+++ b/theories/Lists/TheoryList.v
@@ -14,7 +14,7 @@ Require Export List.
Set Implicit Arguments.
Section Lists.
-Variable A : Set.
+Variable A : Type.
(**********************)
(** The null function *)
@@ -325,7 +325,7 @@ Realizer find.
*)
Qed.
-Variable B : Set.
+Variable B : Type.
Variable T : A -> B -> Prop.
Variable TS_dec : forall a:A, {c : B | T a c} + {P a}.
@@ -358,7 +358,7 @@ End Find_sec.
Section Assoc_sec.
-Variable B : Set.
+Variable B : Type.
Fixpoint assoc (a:A) (l:list (A * B)) {struct l} :
Exc B :=
match l with