aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/micromega/rexample.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/micromega/rexample.v')
-rw-r--r--test-suite/micromega/rexample.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/micromega/rexample.v b/test-suite/micromega/rexample.v
index d7386a4ec..c957add69 100644
--- a/test-suite/micromega/rexample.v
+++ b/test-suite/micromega/rexample.v
@@ -12,7 +12,7 @@ Require Import Ring_normalize.
Open Scope R_scope.
-Lemma yplus_minus : forall x y,
+Lemma yplus_minus : forall x y,
0 = x + y -> 0 = x -y -> 0 = x /\ 0 = y.
Proof.
intros.
@@ -34,7 +34,7 @@ Proof.
Qed.
-Lemma vcgen_25 : forall
+Lemma vcgen_25 : forall
(n : R)
(m : R)
(jt : R)