@@ -369,11 +369,11 @@ structure References where
369369 the spans for `foo`, `bar`, and `baz`. Global definitions are always treated as used.
370370 (It would be nice to be able to detect unused global definitions but this requires more
371371 information than the linter framework can provide.) -/
372- constDecls : Std.HashSet String .Range := ∅
372+ constDecls : Std.HashSet Lean.Syntax .Range := ∅
373373 /-- The collection of all local declarations, organized by the span of the declaration.
374374 We collapse all declarations declared at the same position into a single record using
375375 `FVarDefinition.aliases`. -/
376- fvarDefs : Std.HashMap String .Range FVarDefinition := ∅
376+ fvarDefs : Std.HashMap Lean.Syntax .Range FVarDefinition := ∅
377377 /-- The set of `FVarId`s that are used directly. These may or may not be aliases. -/
378378 fvarUses : Std.HashSet FVarId := ∅
379379 /-- A mapping from alias to original FVarId. We don't guarantee that the value is not itself
@@ -386,7 +386,7 @@ structure References where
386386
387387/-- Collect information from the `infoTrees` into `References`.
388388See `References` for more information about the return value. -/
389- partial def collectReferences (infoTrees : Array Elab.InfoTree) (cmdStxRange : String .Range)
389+ partial def collectReferences (infoTrees : Array Elab.InfoTree) (cmdStxRange : Lean.Syntax .Range)
390390 (linterSets : LinterSets) :
391391 StateRefT References IO Unit := ReaderT.run (r := false ) <| go infoTrees none
392392where
0 commit comments