Skip to content

Commit 274edf8

Browse files
committed
chore: add deprecations for {Extract,Lift}Lets.lean (#24871)
Automatically created by #24861. These files were removed in the toolchain bump in ##24561.
1 parent 753ef7e commit 274edf8

File tree

4 files changed

+26
-0
lines changed

4 files changed

+26
-0
lines changed

Mathlib.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -5588,6 +5588,7 @@ import Mathlib.Tactic.Explode.Datatypes
55885588
import Mathlib.Tactic.Explode.Pretty
55895589
import Mathlib.Tactic.ExtendDoc
55905590
import Mathlib.Tactic.ExtractGoal
5591+
import Mathlib.Tactic.ExtractLets
55915592
import Mathlib.Tactic.FBinop
55925593
import Mathlib.Tactic.FailIfNoProgress
55935594
import Mathlib.Tactic.FastInstance
@@ -5630,6 +5631,7 @@ import Mathlib.Tactic.IntervalCases
56305631
import Mathlib.Tactic.IrreducibleDef
56315632
import Mathlib.Tactic.Lemma
56325633
import Mathlib.Tactic.Lift
5634+
import Mathlib.Tactic.LiftLets
56335635
import Mathlib.Tactic.Linarith
56345636
import Mathlib.Tactic.Linarith.Datatypes
56355637
import Mathlib.Tactic.Linarith.Frontend

Mathlib/Tactic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -81,6 +81,7 @@ import Mathlib.Tactic.Explode.Datatypes
8181
import Mathlib.Tactic.Explode.Pretty
8282
import Mathlib.Tactic.ExtendDoc
8383
import Mathlib.Tactic.ExtractGoal
84+
import Mathlib.Tactic.ExtractLets
8485
import Mathlib.Tactic.FBinop
8586
import Mathlib.Tactic.FailIfNoProgress
8687
import Mathlib.Tactic.FastInstance
@@ -123,6 +124,7 @@ import Mathlib.Tactic.IntervalCases
123124
import Mathlib.Tactic.IrreducibleDef
124125
import Mathlib.Tactic.Lemma
125126
import Mathlib.Tactic.Lift
127+
import Mathlib.Tactic.LiftLets
126128
import Mathlib.Tactic.Linarith
127129
import Mathlib.Tactic.Linarith.Datatypes
128130
import Mathlib.Tactic.Linarith.Frontend

Mathlib/Tactic/ExtractLets.lean

Lines changed: 12 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,12 @@
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")

Mathlib/Tactic/LiftLets.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,10 @@
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")

0 commit comments

Comments
 (0)