aboutsummaryrefslogtreecommitdiffhomepage
path: root/tools/coqdoc/output.ml
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-02-11 03:18:39 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-02-11 03:18:39 +0000
commitc922e479053477789bd4d455ba0630e6ad71c3d5 (patch)
treeef0d7f713c1866c84eeb4b3ffed61ffbe53fc0b2 /tools/coqdoc/output.ml
parented54c8c767c6a3dfe9ce453c57bd849c20df7951 (diff)
Add keywords that were missing, notably for terms.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9638 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tools/coqdoc/output.ml')
-rw-r--r--tools/coqdoc/output.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/tools/coqdoc/output.ml b/tools/coqdoc/output.ml
index 737cd4d75..123faa62e 100644
--- a/tools/coqdoc/output.ml
+++ b/tools/coqdoc/output.ml
@@ -40,18 +40,18 @@ let is_keyword =
"Module"; "Module Type"; "Declare Module";
"Mutual"; "Parameter"; "Parameters"; "Print"; "Proof"; "Qed";
"Record"; "Recursive"; "Remark"; "Require"; "Save"; "Scheme";
- "Section"; "Show"; "Syntactic"; "Syntax"; "Tactic"; "Theorem";
+ "Section"; "Show"; "Structure"; "Syntactic"; "Syntax"; "Tactic"; "Theorem";
"Unset"; "Variable"; "Variables";
"Notation";
(* Program *)
"Program Definition"; "Program Fixpoint"; "Program Lemma";
- "Obligation"; "Obligations"; "Solve";
+ "Obligation"; "Obligations"; "Solve"; "Next Obligation"; "Next";
(*i (* correctness *)
"array"; "assert"; "begin"; "do"; "done"; "else"; "end"; "if";
"in"; "invariant"; "let"; "of"; "ref"; "state"; "then"; "variant";
"while"; i*)
(*i (* coq terms *) *)
- "match"; "with"; "end"; "if"; "then"; "else"; "Prop"; "Set"; "Type"; ":="
+ "match"; "in"; "return"; "with"; "end"; "let"; "dest"; "fun"; "if"; "then"; "else"; "Prop"; "Set"; "Type"; ":="
]
(*s Current Coq module *)