File tree Expand file tree Collapse file tree 4 files changed +26
-0
lines changed
Expand file tree Collapse file tree 4 files changed +26
-0
lines changed Original file line number Diff line number Diff line change @@ -5588,6 +5588,7 @@ import Mathlib.Tactic.Explode.Datatypes
55885588import Mathlib.Tactic.Explode.Pretty
55895589import Mathlib.Tactic.ExtendDoc
55905590import Mathlib.Tactic.ExtractGoal
5591+ import Mathlib.Tactic.ExtractLets
55915592import Mathlib.Tactic.FBinop
55925593import Mathlib.Tactic.FailIfNoProgress
55935594import Mathlib.Tactic.FastInstance
@@ -5630,6 +5631,7 @@ import Mathlib.Tactic.IntervalCases
56305631import Mathlib.Tactic.IrreducibleDef
56315632import Mathlib.Tactic.Lemma
56325633import Mathlib.Tactic.Lift
5634+ import Mathlib.Tactic.LiftLets
56335635import Mathlib.Tactic.Linarith
56345636import Mathlib.Tactic.Linarith.Datatypes
56355637import Mathlib.Tactic.Linarith.Frontend
Original file line number Diff line number Diff line change @@ -81,6 +81,7 @@ import Mathlib.Tactic.Explode.Datatypes
8181import Mathlib.Tactic.Explode.Pretty
8282import Mathlib.Tactic.ExtendDoc
8383import Mathlib.Tactic.ExtractGoal
84+ import Mathlib.Tactic.ExtractLets
8485import Mathlib.Tactic.FBinop
8586import Mathlib.Tactic.FailIfNoProgress
8687import Mathlib.Tactic.FastInstance
@@ -123,6 +124,7 @@ import Mathlib.Tactic.IntervalCases
123124import Mathlib.Tactic.IrreducibleDef
124125import Mathlib.Tactic.Lemma
125126import Mathlib.Tactic.Lift
127+ import Mathlib.Tactic.LiftLets
126128import Mathlib.Tactic.Linarith
127129import Mathlib.Tactic.Linarith.Datatypes
128130import Mathlib.Tactic.Linarith.Frontend
Original file line number Diff line number Diff line change 1+ /-
2+ Copyright (c) 2023 Kyle Miller. All rights reserved.
3+ Released under Apache 2.0 license as described in the file LICENSE.
4+ Authors: Kyle Miller
5+ -/
6+ import Mathlib.Lean.Expr.Basic
7+ import Mathlib.Tactic.Basic
8+ import Batteries.Tactic.Lint.Misc
9+ import Mathlib.Tactic.Linter.DeprecatedModule
10+
11+ deprecated_module "The extract_let tactic was moved to Lean core; \
12+ you can probably just remove this import" (since := "2025-05-02" )
Original file line number Diff line number Diff line change 1+ /-
2+ Copyright (c) 2023 Kyle Miller. All rights reserved.
3+ Released under Apache 2.0 license as described in the file LICENSE.
4+ Authors: Kyle Miller
5+ -/
6+ import Mathlib.Tactic.Basic
7+ import Mathlib.Tactic.Linter.DeprecatedModule
8+
9+ deprecated_module "The lift_lets tactic was moved to Lean core; \
10+ you can probably just remove this import" (since := "2025-05-02" )
You can’t perform that action at this time.
0 commit comments