aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
commit67f72c93f5f364591224a86c52727867e02a8f71 (patch)
treeecf630daf8346e77e6620233d8f3e6c18a0c9b3c /theories/Lists/Streams.v
parentb239b208eb9a66037b0c629cf7ccb6e4b110636a (diff)
option -dump-glob pour coqdoc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2474 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rwxr-xr-xtheories/Lists/Streams.v11
1 files changed, 5 insertions, 6 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 16c88e598..f5f15d889 100755
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -58,7 +58,7 @@ Lemma Str_nth_plus
Intros; Unfold Str_nth; Rewrite Str_nth_tl_plus; Trivial with datatypes.
Save.
-(* Extensional Equality between two streams *)
+(** Extensional Equality between two streams *)
CoInductive EqSt : Stream->Stream->Prop :=
eqst : (s1,s2:Stream)
@@ -66,14 +66,14 @@ CoInductive EqSt : Stream->Stream->Prop :=
(EqSt (tl s1) (tl s2))
->(EqSt s1 s2).
-(* A coinduction principle *)
+(** A coinduction principle *)
Meta Definition CoInduction proof :=
Cofix proof; Intros; Constructor;
[Clear proof | Try (Apply proof;Clear proof)].
-(* Extensional equality is an equivalence relation *)
+(** Extensional equality is an equivalence relation *)
Theorem EqSt_reflex : (s:Stream)(EqSt s s).
(CoInduction EqSt_reflex).
@@ -99,9 +99,8 @@ Case H; Trivial with datatypes.
Case H0; Trivial with datatypes.
Qed.
-(*
-The definition given is equivalent to require the elements at each position to be equal
-*)
+(** The definition given is equivalent to require the elements at each
+ position to be equal *)
Theorem eqst_ntheq :
(n:nat)(s1,s2:Stream)(EqSt s1 s2)->(Str_nth n s1)=(Str_nth n s2).