aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-04-17 14:18:25 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-04-17 14:18:25 +0000
commite6dc3d26de0fbd4d0b09dd692432e2cd14774118 (patch)
tree7b59d151da0de78736103c2dc2a487b9b5a0ab7b /theories/Lists/Streams.v
parent1c16b71834633aa11003b664757969255c0c65e5 (diff)
Correction du bug #1510
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9777 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rw-r--r--theories/Lists/Streams.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index a8b55fb3e..4e8be48a4 100644
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -162,13 +162,13 @@ End Stream_Properties.
End Streams.
Section Map.
-Variables A B : Set.
+Variables A B : Type.
Variable f : A -> B.
CoFixpoint map (s:Stream A) : Stream B := Cons (f (hd s)) (map (tl s)).
End Map.
Section Constant_Stream.
-Variable A : Set.
+Variable A : Type.
Variable a : A.
CoFixpoint const : Stream A := Cons a const.
End Constant_Stream.