Skip to content

Conversation

@alok
Copy link

@alok alok commented Jan 2, 2026

Summary

Upgrade plain backticks to Verso's semantic markup ({name}, {keywordOf}, {tactic}, {lean}) across core documentation files for improved semantic consistency and clickability in the generated docs.

Changes

BasicTypes/Nat.lean:

  • \Nat`{name}`Nat`` (2 occurrences)
  • Fixed typo: "an natural" → "a natural"

BasicTypes/Int.lean:

  • \Int`namespace →{name}`Int``

BasicTypes/List/Predicates.lean:

  • \List`namespace →{name}`List`` (2 occurrences)

BasicTypes/Maps.lean:

  • \Std`namespace →{name}`Std``

BasicTypes/BitVec.lean:

  • \BitVec`namespace →{name}`BitVec`` (2 occurrences)

Types.lean:

  • \let`{keywordOf Lean.Parser.Term.let}`let``
  • \variable`{keywordOf Lean.Parser.Command.variable}`variable``
  • \universe`{keywordOf Lean.Parser.Command.universe}`universe``

Terms.lean:

  • \Function`namespace →{name}`Function``

Namespaces.lean:

  • \namespace`{keywordOf Lean.Parser.Command.namespace}`namespace``
  • \in`{keywordOf Lean.Parser.Command.in}`in``
  • \variable`{keywordOf Lean.Parser.Command.variable}`variable``
  • \Greetings`namespace →{name}`Greetings``
  • More namespace upgrades: HotDrink, ColdDrink, Forest, _root_

Tactics.lean:

  • \cases`{tactic}`cases``
  • \match`{keywordOf Lean.Parser.Tactic.match}`match``

Simp.lean:

  • \simp`{tactic}`simp``

Tactics/Custom.lean:

  • \trivial`{tactic}`trivial``

Classes/BasicClasses.lean:

  • \Ord`, `Max`, `Min`, `LT`, `LE`, `Classical`{name}` versions

Classes/InstanceSynth.lean:

  • \let`{keywordOf Lean.Parser.Term.let}`let``

Language/Functions.lean:

  • \Function`namespace →{name}`Function``

Language/Namespaces.lean:

  • \Forest`, `root`{name}` versions

Language/InductiveTypes.lean:

  • \Prop`{name}`Prop``

Language/InductiveTypes/LogicalModel.lean:

  • \fun`{keywordOf Lean.Parser.Term.fun}`fun``

RecursiveDefs/PartialFixpoint/Theory.lean:

  • \Lean.Order`namespace →{name}`Lean.Order``

Grind/Algebra.lean, Grind/Linarith.lean:

  • Solver names → {name} markup

Grind/ExtendedExamples/IfElseNorm.lean:

  • \IfExpr`namespace →{name}`IfExpr``

ErrorExplanations/InferBinderTypeFailed.lean:

  • \example`, `def`, `theorem`, `opaque`{keywordOf}` versions

ErrorExplanations/InductionWithNoAlts.lean:

  • \induction`, `induction'`{tactic}` versions
  • \import`{keywordOf}` version

ErrorExplanations/InferDefTypeFailed.lean:

  • \List`{name}`List``
  • \theorem`{keywordOf}` version (2 occurrences)

ErrorExplanations/DependsOnNoncomputable.lean:

  • \Inhabited`, `Nonempty`{name}` versions

ErrorExplanations/UnknownIdentifier.lean:

  • \Color`namespace/type →{name}` versions
  • \Color.rgb`{lean}` version

Test plan

  • Build reference-manual successfully with lake build (pre-existing Verso package issues, not from changes)

🤖 Generated with Claude Code

alok and others added 8 commits January 1, 2026 17:43
This PR upgrades plain backticks to Verso's semantic markup where appropriate:

- `{name}` for declared identifiers (Nat)
- `{keywordOf Parser.Path}` for keywords (namespace, in, variable, let, match)
- `{tactic}` for tactic references (cases)

Also fixes a minor typo: "an natural" → "a natural" in Nat.lean.

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Additional upgrades:
- Simp.lean: `simp` → {tactic}`simp`
- Tactics/Custom.lean: `trivial` → {tactic}`trivial`
- ErrorExplanations/InferBinderTypeFailed.lean: `example`, `def`, `theorem`, `opaque` → {keywordOf}
- ErrorExplanations/InductionWithNoAlts.lean: `induction`, `induction'` → {tactic}, `import` → {keywordOf}

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Classes/BasicClasses.lean:
- `Ord`, `Max`, `Min`, `LT`, `LE`, `Classical` → {name}

Classes/InstanceSynth.lean:
- `let` → {keywordOf}

Grind/Algebra.lean, Grind/Linarith.lean:
- `ring`, `linarith` solver names → {name}

Language/Functions.lean:
- `Function` namespace → {name}

RecursiveDefs/PartialFixpoint/Theory.lean:
- `Lean.Order` namespace → {name}

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Language/Namespaces.lean:
- `_root_`, `HotDrink`, `ColdDrink` namespace names → {name}

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Use {keywordOf} for `fun` keyword and {name} for `Prop`.

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Use {name} for namespace references: Int, List, Std, BitVec, Function,
Greetings, Forest, Color, IfExpr.

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Use {name} for List, Inhabited, Nonempty type references.

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Use {keywordOf} for theorem keyword references.

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
@alok alok marked this pull request as draft January 2, 2026 02:12
alok and others added 8 commits January 1, 2026 23:14
- Classes.lean: Ord instance
- DependsOnNoncomputable.lean: Classical, Decidable, fromImage, noncomputable
- UnknownIdentifier.lean: Color, Color.rgb
- Algebra.lean: ring, Lean.Grind, CommSemiring, CommRing, AddRightCancel, Nat, NoNatZeroDivisors
- Linarith.lean: NatModule, ring, linarith
- DerivingHandlers.lean: Bool
- Syntax.lean: for (keywordOf), ForIn.forIn, ForM.forM
- Maps.lean: Std.Data.HashMap.RawLemmas, Std.HashMap.Raw, Std.HashMap.RawLemmas,
  Std.DHashMap.Raw, Std.DHashMap.RawLemmas, Std.HashSet.Raw, Std.HashSet.RawLemmas,
  Std.DTreeMap.Raw
- Maps/TreeMap.lean: Std.TreeMap.Raw
- Maps/TreeSet.lean: Std.TreeSet.Raw
- Nat.lean: Nat.succ_lt_succ
- String.lean: List.Lex
- Sum.lean: PSum
- Nats.iter, Finite, Iter.toArray
- Finite (Triple Char) Id as {lean}
- VCGen/Tutorial.lean: Std.Do → {namespace}
- InductiveParamMissing.lean: RoseTree.All, List.All → {name}

🤖 Generated with [Claude Code](https://claude.com/claude-code)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

None yet

Projects

None yet

Development

Successfully merging this pull request may close these issues.

1 participant