DEBSOURCES
Skip Quicknav
sources / coq / 8.20.1%2Bdfsg-1 / test-suite / bugs / bug_2854.v
123456789
Section foo. Let foo := Type. Definition bar : foo -> foo := @id _. Goal False. subst foo. Fail pose bar as f. (* simpl in f. *) Abort. End foo.