From 596f0f2b5ab76305447ed1ef3999fd7d9939fbef Mon Sep 17 00:00:00 2001 From: mohring Date: Wed, 30 Nov 2005 10:05:53 +0000 Subject: changement parametres inductifs dans les theories git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7630 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Lists/Streams.v | 13 ++++++------- 1 file changed, 6 insertions(+), 7 deletions(-) (limited to 'theories/Lists') diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v index f69041eb8..366172381 100755 --- a/theories/Lists/Streams.v +++ b/theories/Lists/Streams.v @@ -71,9 +71,8 @@ Qed. (** Extensional Equality between two streams *) -CoInductive EqSt : Stream -> Stream -> Prop := +CoInductive EqSt (s1 s2: Stream) : Prop := eqst : - forall s1 s2:Stream, hd s1 = hd s2 -> EqSt (tl s1) (tl s2) -> EqSt s1 s2. (** A coinduction principle *) @@ -140,12 +139,12 @@ Inductive Exists : Stream -> Prop := | Further : forall x:Stream, ~ P x -> Exists (tl x) -> Exists x. i*) -Inductive Exists : Stream -> Prop := - | Here : forall x:Stream, P x -> Exists x - | Further : forall x:Stream, Exists (tl x) -> Exists x. +Inductive Exists ( x: Stream ) : Prop := + | Here : P x -> Exists x + | Further : Exists (tl x) -> Exists x. -CoInductive ForAll : Stream -> Prop := - HereAndFurther : forall x:Stream, P x -> ForAll (tl x) -> ForAll x. +CoInductive ForAll (x: Stream) : Prop := + HereAndFurther : P x -> ForAll (tl x) -> ForAll x. Section Co_Induction_ForAll. -- cgit v1.2.3