aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-09 15:23:08 +0000
committerGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-09 15:23:08 +0000
commit43f76860196296aa180e27d90f64a05ed7edf9d7 (patch)
treecc7f954fa633a55136db4a7c66d3058ef9e1590c /theories
parentbeed52ca495d7cceac9abba5722576a6d9f15ed2 (diff)
Tactic Definition -> Meta Definition
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1237 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rwxr-xr-xtheories/Lists/Streams.v2
-rw-r--r--theories/Zarith/zarith_aux.v2
2 files changed, 2 insertions, 2 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 5962e0ed2..297a888eb 100755
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -61,7 +61,7 @@ CoInductive EqSt : Stream->Stream->Prop :=
(* A coinduction principle *)
-Tactic Definition CoInduction proof :=
+Meta Definition CoInduction proof :=
Cofix proof; Intros; Constructor;
[Clear proof | Try (Apply proof;Clear proof)].
diff --git a/theories/Zarith/zarith_aux.v b/theories/Zarith/zarith_aux.v
index 113a59347..b67bf39f5 100644
--- a/theories/Zarith/zarith_aux.v
+++ b/theories/Zarith/zarith_aux.v
@@ -11,7 +11,7 @@
Require Arith.
Require Export fast_integer.
-Tactic Definition ElimCompare com1 com2:=
+Meta Definition ElimCompare com1 com2:=
Elim (Dcompare (Zcompare com1 com2)); [
Idtac
| Intro hidden_auxiliary; Elim hidden_auxiliary;