Skip to content

Commit

Permalink
Fix syntax (nitpick)
Browse files Browse the repository at this point in the history
  • Loading branch information
rtetley committed Jul 12, 2024
1 parent a3e8b67 commit dd01440
Showing 1 changed file with 8 additions and 10 deletions.
18 changes: 8 additions & 10 deletions language-server/dm/document.ml
Original file line number Diff line number Diff line change
Expand Up @@ -117,19 +117,18 @@ let record_outline document id (ast : Synterp.vernac_control_entry) classif (out
match classif with
| VtStartProof (_, names) ->
let vernac_gen_expr = ast.v.expr in
let type_ =
begin match vernac_gen_expr with
let type_ = match vernac_gen_expr with
| VernacSynterp _ -> None
| VernacSynPure pure ->
match pure with
| Vernacexpr.VernacStartTheoremProof (kind, _) -> Some (TheoremKind kind)
| Vernacexpr.VernacDefinition ((_, def), _, _) -> Some (DefinitionType def)
| _ -> None
end in
let name = begin match names with
in
let name = match names with
|[] -> "default"
| n :: _ -> Names.Id.to_string n
end in
in
let statement = "" in
begin match type_ with
| None -> outline
Expand All @@ -140,19 +139,18 @@ let record_outline document id (ast : Synterp.vernac_control_entry) classif (out
end
| VtSideff (names, _) ->
let vernac_gen_expr = ast.v.expr in
let type_ =
begin match vernac_gen_expr with
let type_ = match vernac_gen_expr with
| VernacSynterp _ -> None
| VernacSynPure pure ->
match pure with
| Vernacexpr.VernacStartTheoremProof (kind, _) -> Some (TheoremKind kind)
| Vernacexpr.VernacDefinition ((_, def), _, _) -> Some (DefinitionType def)
| _ -> None
end in
let name = begin match names with
in
let name = match names with
|[] -> "default"
| n :: _ -> Names.Id.to_string n
end in
in
let statement = "" in
begin match type_ with
| None -> outline
Expand Down

0 comments on commit dd01440

Please sign in to comment.