aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 19:19:05 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 19:19:05 +0000
commit49898a533578846598c7d8a62e8de2f1fcca84c0 (patch)
tree57f1ec2af840f41730cf5254422da2c330503777 /theories/Lists/Streams.v
parent626b27bd1955c1a071d607fbf35706155df5e229 (diff)
MAJ commentaires
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4583 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rwxr-xr-xtheories/Lists/Streams.v10
1 files changed, 6 insertions, 4 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 35d67e568..9bbbe0e46 100755
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -10,7 +10,9 @@
Set Implicit Arguments.
-Section Streams. (* The set of streams : definition *)
+(** Streams *)
+
+Section Streams.
Variable A : Set.
@@ -125,9 +127,9 @@ Section Stream_Properties.
Variable P : Stream->Prop.
(*i
-Inductive Exists : Stream -> Prop :=
- Here : (x:Stream)(P x) ->(Exists x) |
- Further : (x:Stream)~(P x)->(Exists (tl x))->(Exists x).
+Inductive Exists : Stream -> Prop :=
+ | Here : forall x:Stream, P x -> Exists x
+ | Further : forall x:Stream, ~ P x -> Exists (tl x) -> Exists x.
i*)
Inductive Exists : Stream -> Prop :=