aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/setoid_ring/ZArithRing.v
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-17 15:58:14 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-17 15:58:14 +0000
commit61ccbc81a2f3b4662ed4a2bad9d07d2003dda3a2 (patch)
tree961cc88c714aa91a0276ea9fbf8bc53b2b9d5c28 /plugins/setoid_ring/ZArithRing.v
parent6d3fbdf36c6a47b49c2a4b16f498972c93c07574 (diff)
Delete trailing whitespaces in all *.{v,ml*} files
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12337 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/setoid_ring/ZArithRing.v')
-rw-r--r--plugins/setoid_ring/ZArithRing.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/plugins/setoid_ring/ZArithRing.v b/plugins/setoid_ring/ZArithRing.v
index 942915abf..4cb5a05a3 100644
--- a/plugins/setoid_ring/ZArithRing.v
+++ b/plugins/setoid_ring/ZArithRing.v
@@ -21,7 +21,7 @@ Ltac Zcst t :=
end.
Ltac isZpow_coef t :=
- match t with
+ match t with
| Zpos ?p => isPcst p
| Z0 => constr:true
| _ => constr:false
@@ -41,18 +41,18 @@ Ltac Zpow_tac t :=
Ltac Zpower_neg :=
repeat match goal with
- | [|- ?G] =>
- match G with
+ | [|- ?G] =>
+ match G with
| context c [Zpower _ (Zneg _)] =>
let t := context c [Z0] in
change t
end
- end.
+ end.
Add Ring Zr : Zth
(decidable Zeq_bool_eq, constants [Zcst], preprocess [Zpower_neg;unfold Zsucc],
power_tac Zpower_theory [Zpow_tac],
- (* The two following option are not needed, it is the default chose when the set of
+ (* The two following option are not needed, it is the default chose when the set of
coefficiant is usual ring Z *)
div (InitialRing.Ztriv_div_th (@Eqsth Z) (@IDphi Z)),
sign get_signZ_th).