aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-19 12:41:04 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-19 12:41:04 +0000
commit4a816963c315007576bfaba3e87df0c7091e1402 (patch)
tree9b32d023e23b3c9cfa2b11382c34796aa3630b87 /theories/Lists/Streams.v
parentbdbbb1bea47909ad5d0daffd77e090ef9b59d826 (diff)
Mise de (*i autour CVS info
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1620 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rwxr-xr-xtheories/Lists/Streams.v8
1 files changed, 3 insertions, 5 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 5bc9dc97e..9dc01f0a1 100755
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -6,9 +6,9 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
-(* $Id$ *)
+(*i $Id$ i*)
-Implicit Arguments On.
+Set Implicit Arguments.
Section Streams. (* The set of streams : definition *)
@@ -166,6 +166,4 @@ Variable a : A.
CoFixpoint const : (Stream A) := (Cons a const).
End Constant_Stream.
-
-
-Implicit Arguments Off.
+Unset Implicit Arguments.