aboutsummaryrefslogtreecommitdiff
path: root/theories
diff options
context:
space:
mode:
authorHugo Herbelin2020-05-28 15:38:34 +0200
committerHugo Herbelin2021-04-06 17:40:53 +0200
commit6628ed4a231b7362b033f62505eca3c899e60549 (patch)
tree9b8fb6ef754dcea3dae76b0640d5d71eea40b3ac /theories
parent2ee505630756676ded9f8eb6511ad642c80179ee (diff)
Typo in a micromega comment.
Diffstat (limited to 'theories')
-rw-r--r--theories/micromega/OrderedRing.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/theories/micromega/OrderedRing.v b/theories/micromega/OrderedRing.v
index 5fa3740ab1..bfbd6fd8d3 100644
--- a/theories/micromega/OrderedRing.v
+++ b/theories/micromega/OrderedRing.v
@@ -423,7 +423,7 @@ Qed.
(* The following theorems are used to build a morphism from Z to R and
prove its properties in ZCoeff.v. They are not used in RingMicromega.v. *)
-(* Surprisingly, multilication is needed to prove the following theorem *)
+(* Surprisingly, multiplication is needed to prove the following theorem *)
Theorem Ropp_neg_pos : forall n : R, - n < 0 <-> 0 < n.
Proof.
@@ -457,4 +457,3 @@ apply Rtimes_pos_pos. assumption. now apply -> Rlt_lt_minus.
Qed.*)
End STRICT_ORDERED_RING.
-