DEBSOURCES
Skip Quicknav
sources / coq / 8.16.1%2Bdfsg-1 / test-suite / coq-makefile / template / theories / test.v
123456789
Declare ML Module "coq-test-suite.test". TestCommand. Goal True. Proof. test_tactic. exact I. Qed. Definition foo := 4 + 4.