aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/micromega/MExtraction.v
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-04-02 19:26:59 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-04-02 19:26:59 +0200
commitaec237038d300ce7c81dddd154cbdc93fed5b226 (patch)
tree010cbf00cf80b51f53e5a44c6345844775ca52c3 /plugins/micromega/MExtraction.v
parent4226e7ac76ee8a292b717a3c0c12ef0c60495e90 (diff)
Fix some typos.
Diffstat (limited to 'plugins/micromega/MExtraction.v')
-rw-r--r--plugins/micromega/MExtraction.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/micromega/MExtraction.v b/plugins/micromega/MExtraction.v
index 22ddd549e..8b959c278 100644
--- a/plugins/micromega/MExtraction.v
+++ b/plugins/micromega/MExtraction.v
@@ -34,7 +34,7 @@ Extract Inductive sumor => option [ Some None ].
- rightmost choice (Inright) is (None) *)
-(** To preserve its laziness, andb is normally expansed.
+(** To preserve its laziness, andb is normally expanded.
Let's rather use the ocaml && *)
Extract Inlined Constant andb => "(&&)".