Skip to content

Commit

Permalink
chore: bump for std4#241 (#6975)
Browse files Browse the repository at this point in the history
- [x] depends on: leanprover-community/batteries#241



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Nov 28, 2023
1 parent aa204e9 commit 2577ef7
Show file tree
Hide file tree
Showing 16 changed files with 6 additions and 134 deletions.
1 change: 0 additions & 1 deletion Mathlib.lean
Expand Up @@ -3275,7 +3275,6 @@ import Mathlib.Tactic.NthRewrite
import Mathlib.Tactic.Observe
import Mathlib.Tactic.PPWithUniv
import Mathlib.Tactic.Peel
import Mathlib.Tactic.PermuteGoals
import Mathlib.Tactic.Polyrith
import Mathlib.Tactic.Positivity
import Mathlib.Tactic.Positivity.Basic
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Control/Traversable/Basic.lean
Expand Up @@ -277,10 +277,10 @@ section
variable {F : Type u → Type v} [Applicative F]

instance : Traversable Option :=
@Option.traverse⟩
⟨Option.traverse⟩

instance : Traversable List :=
@List.traverse⟩
⟨List.traverse⟩

end

Expand Down
8 changes: 0 additions & 8 deletions Mathlib/Data/List/Defs.lean
Expand Up @@ -446,15 +446,7 @@ def mapDiagM' {m} [Monad m] {α} (f : α → α → m Unit) : List α → m Unit
-- | h :: t => (f h h >> t.mapM' (f h)) >> t.mapDiagM'
#align list.mmap'_diag List.mapDiagM'

/-- Map each element of a `List` to an action, evaluate these actions in order,
and collect the results.
-/
protected def traverse {F : Type u → Type v} [Applicative F]
{α : Type*} {β : Type u} (f : α → F β) : List α → F (List β)
| [] => pure []
| x :: xs => List.cons <$> f x <*> List.traverse f xs
#align list.traverse List.traverse

#align list.get_rest List.getRest
#align list.slice List.dropSlice

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Init/Data/Nat/Bitwise.lean
Expand Up @@ -9,7 +9,6 @@ import Mathlib.Data.Bool.Basic
import Mathlib.Init.Data.Bool.Lemmas
import Mathlib.Init.ZeroOne
import Mathlib.Tactic.Cases
import Mathlib.Tactic.PermuteGoals

#align_import init.data.nat.bitwise from "leanprover-community/lean"@"53e8520d8964c7632989880372d91ba0cecbaf00"

Expand Down
8 changes: 0 additions & 8 deletions Mathlib/Lean/Expr/Basic.lean
Expand Up @@ -182,18 +182,10 @@ namespace Expr

/-! ### Declarations about `Expr` -/

/-- If the expression is a constant, return that name. Otherwise return `Name.anonymous`. -/
def constName (e : Expr) : Name :=
e.constName?.getD Name.anonymous

def bvarIdx? : Expr → Option Nat
| bvar idx => some idx
| _ => none

/-- Return the function (name) and arguments of an application. -/
def getAppFnArgs (e : Expr) : Name × Array Expr :=
withApp e λ e a => (e.constName, a)

/-- Invariant: `i : ℕ` should be less than the size of `as : Array Expr`. -/
private def getAppAppsAux : Expr → Array Expr → Nat → Array Expr
| .app f a, as, i => getAppAppsAux f (as.set! i (.app f a)) (i-1)
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Mathport/Syntax.lean
Expand Up @@ -64,7 +64,6 @@ import Mathlib.Tactic.Monotonicity
import Mathlib.Tactic.Nontriviality
import Mathlib.Tactic.NormNum
import Mathlib.Tactic.NthRewrite
import Mathlib.Tactic.PermuteGoals
import Mathlib.Tactic.Polyrith
import Mathlib.Tactic.Positivity
import Mathlib.Tactic.PushNeg
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic.lean
Expand Up @@ -114,7 +114,6 @@ import Mathlib.Tactic.NthRewrite
import Mathlib.Tactic.Observe
import Mathlib.Tactic.PPWithUniv
import Mathlib.Tactic.Peel
import Mathlib.Tactic.PermuteGoals
import Mathlib.Tactic.Polyrith
import Mathlib.Tactic.Positivity
import Mathlib.Tactic.Positivity.Basic
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Common.lean
Expand Up @@ -57,7 +57,6 @@ import Mathlib.Tactic.MkIffOfInductiveProp
-- import Mathlib.Tactic.NormNum.Basic
import Mathlib.Tactic.NthRewrite
import Mathlib.Tactic.Observe
import Mathlib.Tactic.PermuteGoals
import Mathlib.Tactic.ProjectionNotation
import Mathlib.Tactic.Propose
import Mathlib.Tactic.PushNeg
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Lift.lean
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Floris van Doorn
-/
import Mathlib.Tactic.Cases
import Mathlib.Tactic.PermuteGoals
import Mathlib.Init.Data.Int.Order

/-!
Expand Down
61 changes: 0 additions & 61 deletions Mathlib/Tactic/PermuteGoals.lean

This file was deleted.

2 changes: 1 addition & 1 deletion lake-manifest.json
Expand Up @@ -4,7 +4,7 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "a652e09bd81bcb43ea132d64ecc16580b0c7fa50",
"rev": "d2d9ea14f353d177d4ac9d781b78191b206daa24",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand Down
1 change: 0 additions & 1 deletion scripts/style-exceptions.txt
Expand Up @@ -112,7 +112,6 @@ Mathlib/Tactic/Expect.lean : line 9 : ERR_MOD : Module docstring missing, or too
Mathlib/Tactic/Have.lean : line 10 : ERR_MOD : Module docstring missing, or too late
Mathlib/Tactic/LeftRight.lean : line 9 : ERR_MOD : Module docstring missing, or too late
Mathlib/Tactic/NormCast/Tactic.lean : line 13 : ERR_MOD : Module docstring missing, or too late
Mathlib/Tactic/PermuteGoals.lean : line 11 : ERR_MOD : Module docstring missing, or too late
Mathlib/Tactic/PrintPrefix.lean : line 9 : ERR_MOD : Module docstring missing, or too late
Mathlib/Tactic/PushNeg.lean : line 13 : ERR_MOD : Module docstring missing, or too late
Mathlib/Tactic/Recover.lean : line 10 : ERR_MOD : Module docstring missing, or too late
Expand Down
44 changes: 0 additions & 44 deletions test/PermuteGoals.lean

This file was deleted.

2 changes: 1 addition & 1 deletion test/classical.lean
@@ -1,5 +1,5 @@
import Mathlib.Tactic.Classical
import Mathlib.Tactic.PermuteGoals
import Std.Tactic.PermuteGoals
import Std.Tactic.GuardExpr

noncomputable def foo : Bool := by
Expand Down
2 changes: 1 addition & 1 deletion test/lift.lean
@@ -1,5 +1,5 @@
import Mathlib.Tactic.Lift
import Mathlib.Tactic.PermuteGoals
import Std.Tactic.PermuteGoals
import Mathlib.Tactic.Coe
import Mathlib.Init.Set
import Mathlib.Order.Basic
Expand Down
2 changes: 1 addition & 1 deletion test/solve_by_elim/basic.lean
Expand Up @@ -7,7 +7,7 @@ import Mathlib.Init.Data.Nat.Basic
import Mathlib.Init.Logic
import Std.Tactic.RCases
import Mathlib.Tactic.Constructor
import Mathlib.Tactic.PermuteGoals
import Std.Tactic.PermuteGoals
import Mathlib.Tactic.SolveByElim
import Std.Test.Internal.DummyLabelAttr

Expand Down

0 comments on commit 2577ef7

Please sign in to comment.