aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/ring/NArithRing.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:19:56 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:19:56 +0000
commit634d52825790d8818883549616b3c8807655d2b8 (patch)
treebef68618f7decd0f401931adc1f1043de3634c22 /contrib/ring/NArithRing.v
parentae8dadbbc2c96f50e80e952171396dd683b2d01f (diff)
Noms/énoncés plus canoniques
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4875 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/ring/NArithRing.v')
-rw-r--r--contrib/ring/NArithRing.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/contrib/ring/NArithRing.v b/contrib/ring/NArithRing.v
index 63483e5b1..018503dc8 100644
--- a/contrib/ring/NArithRing.v
+++ b/contrib/ring/NArithRing.v
@@ -30,13 +30,13 @@ Save.
Definition NTheory : (Semi_Ring_Theory Nplus Nmult (Pos xH) Nul Neq).
Split.
Apply Nplus_comm.
- Symmetry; Apply Nplus_assoc_l.
+ Symmetry; Apply Nplus_assoc.
Apply Nmult_comm.
- Symmetry; Apply Nmult_assoc_l.
+ Symmetry; Apply Nmult_assoc.
Apply Nplus_0_l.
Apply Nmult_1_l.
Apply Nmult_0_l.
- Apply Nmult_Nplus_distr_l.
+ Apply Nmult_plus_distr_r.
Apply Nplus_reg_l.
Apply Neq_prop.
Save.