|
9 | 9 | public import Lean.Elab.ElabRules |
10 | 10 | public import Lean.Elab.Tactic.Simp |
11 | 11 | public import Lean.Meta.Tactic.TryThis |
12 | | -public import Lean.PremiseSelection.Basic |
| 12 | +public import Lean.LibrarySuggestions.Basic |
13 | 13 |
|
14 | 14 | public section |
15 | 15 |
|
@@ -56,7 +56,7 @@ def mkSimpCallStx (stx : Syntax) (usedSimps : UsedSimps) : MetaM (TSyntax `tacti |
56 | 56 | if let some a := args then a.getElems else #[] |
57 | 57 | if config.suggestions then |
58 | 58 | -- Get premise suggestions from the premise selector |
59 | | - let suggestions ← Lean.PremiseSelection.select (← getMainGoal) |
| 59 | + let suggestions ← Lean.LibrarySuggestions.select (← getMainGoal) |
60 | 60 | -- Convert suggestions to simp argument syntax and add them to the args |
61 | 61 | for sugg in suggestions do |
62 | 62 | let arg ← `(Parser.Tactic.simpLemma| $(mkIdent sugg.name):term) |
@@ -91,7 +91,7 @@ def mkSimpCallStx (stx : Syntax) (usedSimps : UsedSimps) : MetaM (TSyntax `tacti |
91 | 91 | if let some a := args then a.getElems else #[] |
92 | 92 | if config.suggestions then |
93 | 93 | -- Get premise suggestions from the premise selector |
94 | | - let suggestions ← Lean.PremiseSelection.select (← getMainGoal) |
| 94 | + let suggestions ← Lean.LibrarySuggestions.select (← getMainGoal) |
95 | 95 | -- Convert suggestions to simp argument syntax and add them to the args |
96 | 96 | for sugg in suggestions do |
97 | 97 | let arg ← `(Parser.Tactic.simpLemma| $(mkIdent sugg.name):term) |
|
0 commit comments