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