DEBSOURCES
Skip Quicknav
sources / coq-doc / 8.16.1-1 / test-suite / bugs / bug_3260.v
12345678
Require Import Setoid. Goal forall m n, n = m -> n+n = m+m. intros. replace n with m at 2. lazymatch goal with |- n + m = m + m => idtac end. Abort.