aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-07 10:27:44 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-07 10:27:44 +0000
commit30de194fa897bb44858c92dd458041bb2d2df9fe (patch)
tree2c0c4b00f00e20632a7938d98837b619498d1760 /theories/Lists/Streams.v
parent7f0812b0a29ea508f90949856866cee5fd0ea8ea (diff)
Orthographe
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@813 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rwxr-xr-xtheories/Lists/Streams.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 9895af8ae..e94bb0ee4 100755
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -154,8 +154,8 @@ CoFixpoint map : (Stream A)->(Stream B) :=
End Map.
Section Constant_Stream.
-Variables A : Set.
-Variable a : A.
+Variable A : Set.
+Variable a : A.
CoFixpoint const : (Stream A) := (Cons a const).
End Constant_Stream.