aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/NumPrelude.v
diff options
context:
space:
mode:
authorGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-01 20:21:28 +0000
committerGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-01 20:21:28 +0000
commitc3b607d94cb14217311617919886ba404a5c3edd (patch)
treef443ce8db2d1ddc6ffd9142138fa9a5a7be37e70 /theories/Numbers/NumPrelude.v
parentbbeab5df3839652d3d81a686012256fb1ce148c7 (diff)
Added the compilation of theories/Numbers to Makefile.common. The following things compile: abstract natural numbers and integers with plus, times, minus, and order; Peano and binary implementations for natural numbers.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10161 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/NumPrelude.v')
-rw-r--r--theories/Numbers/NumPrelude.v7
1 files changed, 5 insertions, 2 deletions
diff --git a/theories/Numbers/NumPrelude.v b/theories/Numbers/NumPrelude.v
index 6d3ad55a9..7feed2b14 100644
--- a/theories/Numbers/NumPrelude.v
+++ b/theories/Numbers/NumPrelude.v
@@ -226,12 +226,15 @@ Ltac rewrite_true P H :=
setoid_replace P with True using relation iff;
[| split; intro; [constructor | apply H]].
-Tactic Notation "symmetry" constr(Eq) :=
+(*Ltac symmetry Eq :=
lazymatch Eq with
| ?E ?t1 ?t2 => setoid_replace (E t1 t2) with (E t2 t1) using relation iff;
[| split; intro; symmetry; assumption]
| _ => fail Eq "does not have the form (E t1 t2)"
-end.
+end.*)
+(* This does not work because there already is a tactic "symmetry".
+Declaring "symmetry" a tactic notation does not work because it conflicts
+with "symmetry in": it thinks that "in" is a term. *)
Theorem and_cancel_l : forall A B C : Prop,
(B -> A) -> (C -> A ) -> ((A /\ B <-> A /\ C) <-> (B <-> C)).