Skip to content

Commit

Permalink
Update doc/tools/docgram/common.edit_mlg
Browse files Browse the repository at this point in the history
Co-authored-by: Jim Fehrle <[email protected]>
  • Loading branch information
Villetaneuse and jfehrle committed May 16, 2024
1 parent 8dbbcd6 commit 7a7efb8
Show file tree
Hide file tree
Showing 3 changed files with 6 additions and 6 deletions.
4 changes: 2 additions & 2 deletions doc/sphinx/proof-engine/vernacular-commands.rst
Original file line number Diff line number Diff line change
Expand Up @@ -190,8 +190,8 @@ described elsewhere
.. prodn::
logical_kind ::= {| @thm_token | @assumption_token }
| {| Definition | Example | Context | Primitive | Symbol }
| {| Coercion | Instance | Scheme | Canonical | SubClass | Fixpoint | CoFixpoint }
| {| Field | Method }
| {| Coercion | Instance | Scheme | Canonical | SubClass }
| {| Fixpoint | CoFixpoint | Field | Method }
Filters objects by the keyword that was used to define them
(`Theorem`, `Lemma`, `Axiom`, `Variable`, `Context`,
Expand Down
4 changes: 2 additions & 2 deletions doc/tools/docgram/common.edit_mlg
Original file line number Diff line number Diff line change
Expand Up @@ -1971,12 +1971,12 @@ logical_kind: [
| DELETE "Instance"
| DELETE "Scheme"
| DELETE "Canonical"
| [ "Coercion" | "Instance" | "Scheme" | "Canonical" | "SubClass" ]
| DELETE "Fixpoint"
| DELETE "CoFixpoint"
| [ "Coercion" | "Instance" | "Scheme" | "Canonical" | "SubClass" | "Fixpoint" | "CoFixpoint" ]
| DELETE "Field"
| DELETE "Method"
| [ "Field" | "Method" ]
| [ "Fixpoint" | "CoFixpoint" | "Field" | "Method" ]
]

(* ltac2 *)
Expand Down
4 changes: 2 additions & 2 deletions doc/tools/docgram/orderedGrammar
Original file line number Diff line number Diff line change
Expand Up @@ -1055,8 +1055,8 @@ search_item: [
logical_kind: [
| [ thm_token | assumption_token ]
| [ "Definition" | "Example" | "Context" | "Primitive" | "Symbol" ]
| [ "Coercion" | "Instance" | "Scheme" | "Canonical" | "SubClass" | "Fixpoint" | "CoFixpoint" ]
| [ "Field" | "Method" ]
| [ "Coercion" | "Instance" | "Scheme" | "Canonical" | "SubClass" ]
| [ "Fixpoint" | "CoFixpoint" | "Field" | "Method" ]
]

univ_name_list: [
Expand Down

0 comments on commit 7a7efb8

Please sign in to comment.