aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/ring/ZArithRing.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-06-25 10:49:06 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-06-25 10:49:06 +0000
commit4aa7a14528a016a18831eb18e5085ecfca2adf3e (patch)
tree64d0c0974316c2a57032b0f00da3a88497abdf58 /contrib/ring/ZArithRing.v
parent571e258f8327b3e889a433043c9044f328ec9c9c (diff)
eq and eqT are the same
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5825 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/ring/ZArithRing.v')
-rw-r--r--contrib/ring/ZArithRing.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/contrib/ring/ZArithRing.v b/contrib/ring/ZArithRing.v
index e6a7bf2af..8981a46a5 100644
--- a/contrib/ring/ZArithRing.v
+++ b/contrib/ring/ZArithRing.v
@@ -27,10 +27,10 @@ Lemma Zeq_prop : forall x y:Z, Is_true (Zeq x y) -> x = y.
Qed.
Definition ZTheory : Ring_Theory Zplus Zmult 1%Z 0%Z Zopp Zeq.
- split; intros; apply eq2eqT; eauto with zarith.
- apply eqT2eq; apply Zeq_prop; assumption.
+ split; intros; eauto with zarith.
+ apply Zeq_prop; assumption.
Qed.
(* NatConstants and NatTheory are defined in Ring_theory.v *)
Add Ring Z Zplus Zmult 1%Z 0%Z Zopp Zeq ZTheory
- [ Zpos Zneg 0%Z xO xI 1%positive ]. \ No newline at end of file
+ [ Zpos Zneg 0%Z xO xI 1%positive ].