Skip to content

Commit 5230db6

Browse files
committed
chore: remove upstreamed tactics 11-21 (#684)
1 parent edcfa8f commit 5230db6

File tree

15 files changed

+27
-540
lines changed

15 files changed

+27
-540
lines changed

Mathlib.lean

Lines changed: 0 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -148,13 +148,11 @@ import Mathlib.Tactic.Clear!
148148
import Mathlib.Tactic.ClearExcept
149149
import Mathlib.Tactic.Clear_
150150
import Mathlib.Tactic.Coe
151-
import Mathlib.Tactic.Congr
152151
import Mathlib.Tactic.Constructor
153152
import Mathlib.Tactic.Contrapose
154153
import Mathlib.Tactic.Conv
155154
import Mathlib.Tactic.Convert
156155
import Mathlib.Tactic.Core
157-
import Mathlib.Tactic.DocCommands
158156
import Mathlib.Tactic.Existsi
159157
import Mathlib.Tactic.Expect
160158
import Mathlib.Tactic.FinCases
@@ -199,11 +197,9 @@ import Mathlib.Tactic.Ring.RingNF
199197
import Mathlib.Tactic.RunCmd
200198
import Mathlib.Tactic.Sat.FromLRAT
201199
import Mathlib.Tactic.ScopedNS
202-
import Mathlib.Tactic.SeqFocus
203200
import Mathlib.Tactic.Set
204201
import Mathlib.Tactic.SimpIntro
205202
import Mathlib.Tactic.SimpRw
206-
import Mathlib.Tactic.SimpTrace
207203
import Mathlib.Tactic.Simps.Basic
208204
import Mathlib.Tactic.Simps.NotationClass
209205
import Mathlib.Tactic.SolveByElim

Mathlib/Data/FunLike/Basic.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -148,9 +148,8 @@ instance (priority := 100) : CoeFun F fun _ ↦ ∀ a : α, β a where coe := Fu
148148
Tactic.NormCast.registerCoercion ``FunLike.coe
149149
(some { numArgs := 5, coercee := 4, type := .coeFun })
150150

151-
@[simp]
152-
theorem coe_eq_coe_fn : (FunLike.coe : F → ∀ a : α, β a) = (fun f ↦ ↑f) :=
153-
rfl
151+
-- @[simp] -- porting note: this loops in lean 4
152+
theorem coe_eq_coe_fn : (FunLike.coe (F := F)) = (fun f => ↑f) := rfl
154153

155154
theorem coe_injective : Function.Injective (fun f : F ↦ (f : ∀ a : α, β a)) :=
156155
FunLike.coe_injective'

Mathlib/Init/Logic.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,6 @@ import Std.Tactic.Lint.Basic
88
import Std.Logic
99
import Mathlib.Tactic.Alias
1010
import Mathlib.Tactic.Basic
11-
import Mathlib.Tactic.SimpTrace
1211
import Mathlib.Tactic.Relation.Symm
1312
import Mathlib.Mathport.Attributes
1413
import Mathlib.Mathport.Rename

Mathlib/Logic/Basic.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,6 @@ import Mathlib.Init.Function
88
import Mathlib.Init.Algebra.Classes
99
import Mathlib.Tactic.Basic
1010
import Mathlib.Tactic.LeftRight
11-
import Mathlib.Tactic.SimpTrace
1211
import Std.Util.LibraryNote
1312
import Std.Tactic.Lint.Basic
1413

Mathlib/Mathport/Syntax.lean

Lines changed: 0 additions & 14 deletions
Original file line numberDiff line numberDiff line change
@@ -21,13 +21,11 @@ import Mathlib.Tactic.Classical
2121
import Mathlib.Tactic.Clear_
2222
import Mathlib.Tactic.Clear!
2323
import Mathlib.Tactic.ClearExcept
24-
import Mathlib.Tactic.Congr
2524
import Mathlib.Tactic.Constructor
2625
import Mathlib.Tactic.Contrapose
2726
import Mathlib.Tactic.Conv
2827
import Mathlib.Tactic.Convert
2928
import Mathlib.Tactic.Core
30-
import Mathlib.Tactic.DocCommands
3129
import Mathlib.Tactic.Existsi
3230
import Mathlib.Tactic.FinCases
3331
import Mathlib.Tactic.Find
@@ -58,12 +56,10 @@ import Mathlib.Tactic.RestateAxiom
5856
import Mathlib.Tactic.Ring
5957
import Mathlib.Tactic.RunCmd
6058
import Mathlib.Tactic.ScopedNS
61-
import Mathlib.Tactic.SeqFocus
6259
import Mathlib.Tactic.Set
6360
import Mathlib.Tactic.SimpIntro
6461
import Mathlib.Tactic.SimpRw
6562
import Mathlib.Tactic.Simps.Basic
66-
import Mathlib.Tactic.SimpTrace
6763
import Mathlib.Tactic.SolveByElim
6864
import Mathlib.Tactic.SplitIfs
6965
import Mathlib.Tactic.Substs
@@ -209,7 +205,6 @@ namespace Tactic
209205

210206
/- S -/ syntax (name := propagateTags) "propagate_tags " tacticSeq : tactic
211207
/- S -/ syntax (name := mapply) "mapply " term : tactic
212-
/- S -/ syntax (name := withCases) "with_cases " tacticSeq : tactic
213208
/- S -/ syntax "destruct " term : tactic
214209
/- N -/ syntax (name := abstract) "abstract" (ppSpace ident)? ppSpace tacticSeq : tactic
215210

@@ -221,15 +216,6 @@ namespace Tactic
221216
/- S -/ syntax (name := compVal) "comp_val" : tactic
222217
/- S -/ syntax (name := async) "async " tacticSeq : tactic
223218

224-
/- E -/ syntax (name := apply') "apply' " term : tactic
225-
/- E -/ syntax (name := fapply') "fapply' " term : tactic
226-
/- E -/ syntax (name := eapply') "eapply' " term : tactic
227-
/- E -/ syntax (name := applyWith') "apply_with' " (config)? term : tactic
228-
/- E -/ syntax (name := mapply') "mapply' " term : tactic
229-
/- E -/ syntax (name := rfl') "rfl'" : tactic
230-
/- E -/ syntax (name := symm') "symm'" (ppSpace location)? : tactic
231-
/- E -/ syntax (name := trans') "trans'" (ppSpace term)? : tactic
232-
233219
/- M -/ syntax (name := injectionsAndClear) "injections_and_clear" : tactic
234220

235221
/- E -/ syntax (name := tryFor) "try_for " term:max tacticSeq : tactic

Mathlib/Tactic/Congr.lean

Lines changed: 0 additions & 82 deletions
This file was deleted.

Mathlib/Tactic/DocCommands.lean

Lines changed: 0 additions & 23 deletions
This file was deleted.

Mathlib/Tactic/SeqFocus.lean

Lines changed: 0 additions & 43 deletions
This file was deleted.

0 commit comments

Comments
 (0)