Skip to content

Commit 7ea7acc

Browse files
authored
chore: lower monad of addSuggestion(s) to CoreM (#10526)
1 parent 161a1c0 commit 7ea7acc

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/Lean/Meta/Tactic/TryThis.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -103,7 +103,7 @@ The parameters are:
103103
-/
104104
def addSuggestion (ref : Syntax) (s : Suggestion) (origSpan? : Option Syntax := none)
105105
(header : String := "Try this:") (codeActionPrefix? : Option String := none)
106-
(diffGranularity : Hint.DiffGranularity := .none) : MetaM Unit := do
106+
(diffGranularity : Hint.DiffGranularity := .none) : CoreM Unit := do
107107
let hintSuggestion := {
108108
span? := origSpan?
109109
diffGranularity
@@ -146,7 +146,7 @@ def addSuggestions (ref : Syntax) (suggestions : Array Suggestion)
146146
(origSpan? : Option Syntax := none) (header : String := "Try these:")
147147
(style? : Option SuggestionStyle := none)
148148
(codeActionPrefix? : Option String := none)
149-
(diffGranularity : Hint.DiffGranularity := .none) : MetaM Unit := do
149+
(diffGranularity : Hint.DiffGranularity := .none) : CoreM Unit := do
150150
if suggestions.isEmpty then throwErrorAt ref "No suggestions available"
151151
let hintSuggestions := suggestions.map fun s => {
152152
span? := origSpan?

0 commit comments

Comments
 (0)