DEBSOURCES
Skip Quicknav
sources / coq / 8.20.1%2Bdfsg-1 / test-suite / bugs / bug_16278_load.v
12345678
Set Nested Proofs Allowed. Lemma outer : True. Proof. Lemma inner : True. Proof. constructor. Qed. exact inner. Qed.