DEBSOURCES
Skip Quicknav
sources / coq / 8.20.1%2Bdfsg-1 / test-suite / bugs / bug_18006.v
12345678
Lemma foo : nat -> nat. Proof. fix f 1. intros n. epose (fun a:nat => _). exact (f n). Fail Guarded. Abort.