We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 9a2f939 commit 71ec953Copy full SHA for 71ec953
theories/additions/Dichotomy.v
@@ -171,7 +171,7 @@ Proof.
171
intros p H; unfold dicho; generalize (dicho_aux_lt p H).
172
intro H0; assert (2 <= N.pos p / (N.pos (dicho_aux p)) )%N.
173
- replace 2%N with (2%N * Npos (dicho_aux p) / Npos (dicho_aux p))%N.
174
- + apply N.Div0.div_le_mono.
+ + apply (* N.Div0.div_le_mono. *) N.div_le_mono; try discriminate.
175
* replace 2%N with (Npos 2%positive); cbn;auto.
176
+ rewrite N.div_mul; [auto | discriminate].
177
- case_eq (N.pos p / N.pos (dicho_aux p))%N.
0 commit comments