aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/micromega/Refl.v
diff options
context:
space:
mode:
Diffstat (limited to 'plugins/micromega/Refl.v')
-rw-r--r--plugins/micromega/Refl.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/micromega/Refl.v b/plugins/micromega/Refl.v
index 801d8b212..c86fe8fb6 100644
--- a/plugins/micromega/Refl.v
+++ b/plugins/micromega/Refl.v
@@ -107,7 +107,7 @@ Proof.
Qed.
Lemma not_make_conj_app : forall (A:Type) (t:list A) a eval
- (no_middle_eval : forall d, eval d \/ ~ eval d) ,
+ (no_middle_eval : forall d, eval d \/ ~ eval d) ,
~ make_conj eval (t ++ a) -> (~ make_conj eval t) \/ (~ make_conj eval a).
Proof.
induction t.