DEBSOURCES
Skip Quicknav
sources / coq / 8.20.1%2Bdfsg-1 / test-suite / bugs / bug_10560.v
123456789
From Coq Require Import Uint63. Open Scope uint63_scope. Lemma foo : let n := opp 0 in add n 0 = n. Proof. cbv. apply eq_refl. Qed.