diff options
-rw-r--r-- | Makefile.doc | 4 | ||||
-rw-r--r-- | theories/Logic/ChoiceFacts.v | 8 | ||||
-rw-r--r-- | theories/Logic/ClassicalUniqueChoice.v | 6 | ||||
-rw-r--r-- | tools/coqdoc/cpretty.mll | 2 | ||||
-rw-r--r-- | toplevel/vernacentries.ml | 3 |
5 files changed, 12 insertions, 11 deletions
diff --git a/Makefile.doc b/Makefile.doc index 49b377ef7..56daaa851 100644 --- a/Makefile.doc +++ b/Makefile.doc @@ -214,11 +214,11 @@ doc/stdlib/html/index.html: doc/stdlib/index-list.html doc/stdlib/index-body.htm ifdef QUICK doc/stdlib/Library.coqdoc.tex: $(COQDOC) -q -boot --gallina --body-only --latex --stdout --utf8 \ - -R theories Coq $(THEORIESLIGHTVO:.vo=.v) >> $@ + -R theories Coq $(THEORIESLIGHTVO:.vo=.v) > $@ else doc/stdlib/Library.coqdoc.tex: $(COQDOC) $(THEORIESLIGHTVO) $(COQDOC) -q -boot --gallina --body-only --latex --stdout --utf8 \ - -R theories Coq $(THEORIESLIGHTVO:.vo=.v) >> $@ + -R theories Coq $(THEORIESLIGHTVO:.vo=.v) > $@ endif doc/stdlib/Library.dvi: $(DOCCOMMON) doc/stdlib/Library.coqdoc.tex doc/stdlib/Library.tex diff --git a/theories/Logic/ChoiceFacts.v b/theories/Logic/ChoiceFacts.v index ef59a4e69..b2c4a049d 100644 --- a/theories/Logic/ChoiceFacts.v +++ b/theories/Logic/ChoiceFacts.v @@ -50,9 +50,9 @@ description principles We let also -IPL_2 = 2nd-order impredicative minimal predicate logic (with ex. quant.) -IPL^2 = 2nd-order functional minimal predicate logic (with ex. quant.) -IPL_2^2 = 2nd-order impredicative, 2nd-order functional minimal pred. logic (with ex. quant.) +- IPL_2 = 2nd-order impredicative minimal predicate logic (with ex. quant.) +- IPL^2 = 2nd-order functional minimal predicate logic (with ex. quant.) +- IPL_2^2 = 2nd-order impredicative, 2nd-order functional minimal pred. logic (with ex. quant.) with no prerequisite on the non-emptyness of domains @@ -86,7 +86,7 @@ unpublished. [[Bell93]] John L. Bell, Hilbert's Epsilon Operator in Intuitionistic Type Theories, Mathematical Logic Quarterly, volume 39, 1993. -[Carlström05] Jesper Carlström, Interpreting descriptions in +[[Carlström05]] Jesper Carlström, Interpreting descriptions in intentional type theory, Journal of Symbolic Logic 70(2):488-514, 2005. *) diff --git a/theories/Logic/ClassicalUniqueChoice.v b/theories/Logic/ClassicalUniqueChoice.v index 2a32323cb..4a7bd2ccc 100644 --- a/theories/Logic/ClassicalUniqueChoice.v +++ b/theories/Logic/ClassicalUniqueChoice.v @@ -16,11 +16,11 @@ be used to build functions outside the scope of a theorem proof) *) (** Classical logic and unique choice, as shown in - [ChicliPottierSimpson02], implies the double-negation of + [[ChicliPottierSimpson02]], implies the double-negation of excluded-middle in [Set], hence it implies a strongly classical world. Especially it conflicts with the impredicativity of [Set]. - [ChicliPottierSimpson02] Laurent Chicli, Loïc Pottier, Carlos + [[ChicliPottierSimpson02]] Laurent Chicli, Loïc Pottier, Carlos Simpson, Mathematical Quotients and Quotient Types in Coq, Proceedings of TYPES 2002, Lecture Notes in Computer Science 2646, Springer Verlag. *) @@ -44,7 +44,7 @@ intros A B. apply (dependent_unique_choice A (fun _ => B)). Qed. -(** The following proof comes from [ChicliPottierSimpson02] *) +(** The following proof comes from [[ChicliPottierSimpson02]] *) Require Import Setoid. diff --git a/tools/coqdoc/cpretty.mll b/tools/coqdoc/cpretty.mll index 1834a7d33..95ad1c113 100644 --- a/tools/coqdoc/cpretty.mll +++ b/tools/coqdoc/cpretty.mll @@ -942,7 +942,7 @@ and comment = parse else (brackets := 1; Output.start_inline_coq (); escaped_coq lexbuf; Output.end_inline_coq ()); comment lexbuf } - | "[[" { + | "[[" nl { if !Cdglobals.parse_comments then if !Cdglobals.plain_comments then (Output.char '['; Output.char '[') else (formatted := true; diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml index c077fc492..d77257a0b 100644 --- a/toplevel/vernacentries.ml +++ b/toplevel/vernacentries.ml @@ -308,7 +308,8 @@ let start_proof_and_print k l hook = if !pcoq <> None then (Option.get !pcoq).start_proof () let vernac_definition (local,boxed,k) (loc,id as lid) def hook = - Dumpglob.dump_definition lid false "def"; + if local = Local then Dumpglob.dump_definition lid true "var" + else Dumpglob.dump_definition lid false "def"; (match def with | ProveBody (bl,t) -> (* local binders, typ *) let hook _ _ = () in |