aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
Diffstat (limited to 'theories')
-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.