DEBSOURCES
Skip Quicknav
sources / coq / 8.16.1%2Bdfsg-1 / test-suite / misc / vio_checking.v
123456789
Lemma foo : Type. Proof. exact Type. Qed. Lemma foo1 : Type. Proof. exact Type. Qed. Lemma foo2 : Type. Proof. exact foo1. Qed.