aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-09 16:29:56 +0000
committerGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-09 16:29:56 +0000
commitdfe152b89af9239899e32b2a31adbfda44af5efe (patch)
treef515b9503c4ee2f74ae8f2bbef38946000de37ec /theories/Lists/Streams.v
parentdb18bce6e5da22294b33e93e114a71e8c08fc8ee (diff)
Meta Definition -> Tactic Definition
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1239 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rwxr-xr-xtheories/Lists/Streams.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 297a888eb..5962e0ed2 100755
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -61,7 +61,7 @@ CoInductive EqSt : Stream->Stream->Prop :=
(* A coinduction principle *)
-Meta Definition CoInduction proof :=
+Tactic Definition CoInduction proof :=
Cofix proof; Intros; Constructor;
[Clear proof | Try (Apply proof;Clear proof)].