aboutsummaryrefslogtreecommitdiffhomepage
path: root/tools/coqdoc
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-04-23 15:53:44 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-04-23 15:53:44 +0000
commitcef6f54810c50659cc4b6567d23f55d6806263f1 (patch)
treef6473115e817760ec72c4a73bd3b83973ac1bb12 /tools/coqdoc
parent4adb34c2ea8a602f36230b6b10cfeacc3f6be3f4 (diff)
Correction du bug #1496 (ajout de Program Definition et Program Fixpoint aux commandes vernac considérées par Coqdoc)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9790 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tools/coqdoc')
-rw-r--r--tools/coqdoc/pretty.mll2
1 files changed, 2 insertions, 0 deletions
diff --git a/tools/coqdoc/pretty.mll b/tools/coqdoc/pretty.mll
index 80cdb321b..c34a779e3 100644
--- a/tools/coqdoc/pretty.mll
+++ b/tools/coqdoc/pretty.mll
@@ -212,6 +212,8 @@ let def_token =
| "Scheme"
| "Inductive"
| "CoInductive"
+ | "Program" space+ "Definition"
+ | "Program" space+ "Fixpoint"
let decl_token =
"Hypothesis"