Skip to Content.
Sympa Menu

coq-club - [Coq-Club] a coqdoc issue

coq-club AT inria.fr

Subject: The Coq mailing list

List archive

[Coq-Club] a coqdoc issue


chronological Thread 
  • From: Vladimir Voevodsky <vladimir AT ias.edu>
  • To: Coq Club <coq-club AT inria.fr>
  • Subject: [Coq-Club] a coqdoc issue
  • Date: Wed, 3 Nov 2010 10:18:44 -0400

Hello,

I have used coqdoc with --html option to get "documentation" for my file and the output, when viewed with a browser, has strange coloring behavior. Here is an example:




Theorem isapropneg (X:UU): isaprop (X -> empty).
Proofintroapply (impredfun (S OX empty isapropempty). Qed.

Corollary isapropdneg (X:UU): isaprop (dneg X).
Proofintroapply (isapropneg (neg X)). Defined.

Definition isaninvprop (X:UU):= isweq _ _ (todneg X).

Theorem isaninvpropneg (X:UU): isaninvprop (neg X).
Proofintros.
set (f:= todneg (neg X)). set (g:= negf _ _ (todneg X)). set (is1:= isapropneg X). set (is2:= isapropneg (dneg X)). apply(isweqimplimpl _ _ f g is1 is2). Defined.



 Any ideas on how to make it behave properly?

Thanks!
Vladimir.



Archive powered by MhonArc 2.6.16.

Top of Page