DEBSOURCES
Skip Quicknav
sources / coq / 8.20.1%2Bdfsg-1 / test-suite / micromega / bug_12790.v
12345678
Require Import Lia. Goal forall (a b c d x: nat), S c = a - b -> x <= x + (S c) * d. Proof. intros a b c d x H. lia. Qed.