aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-07-11 15:25:03 +0000
committerGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-07-11 15:25:03 +0000
commit2ed747a81ed14d91112b9b3360c6e5ab4ff897eb (patch)
treeab7199f3977d3efd160e2f24fb7c7e0b205f154f /theories/Lists/Streams.v
parent78a52468777ab14cb88a9acd5b26f549177762fa (diff)
Added ForAll_Str_nth_tl
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9967 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rw-r--r--theories/Lists/Streams.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 909c6b49f..472265f3e 100644
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -146,6 +146,15 @@ Inductive Exists ( x: Stream ) : Prop :=
CoInductive ForAll (x: Stream) : Prop :=
HereAndFurther : P x -> ForAll (tl x) -> ForAll x.
+Lemma ForAll_Str_nth_tl : forall m x, ForAll x -> ForAll (Str_nth_tl m x).
+Proof.
+induction m.
+ tauto.
+intros x [_ H].
+simpl.
+apply IHm.
+assumption.
+Qed.
Section Co_Induction_ForAll.
Variable Inv : Stream -> Prop.