Skip to content

Commit

Permalink
chore: bump Std (#10378)
Browse files Browse the repository at this point in the history
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
kim-em and kim-em committed Feb 9, 2024
1 parent 3a4cb1b commit 359fc77
Show file tree
Hide file tree
Showing 16 changed files with 19 additions and 4 deletions.
1 change: 1 addition & 0 deletions Mathlib/Lean/Expr/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,7 @@ Floris van Doorn, E.W.Ayers, Arthur Paulino
-/
import Lean.Meta.Tactic.Rewrite
import Std.Lean.Expr
import Std.Lean.Name
import Std.Data.Rat.Basic
import Std.Data.List.Basic

Expand Down
1 change: 1 addition & 0 deletions Mathlib/Lean/Meta/Simp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ Authors: Scott Morrison, Gabriel Ebner, Floris van Doorn
-/
import Std.Tactic.OpenPrivate
import Std.Lean.Meta.DiscrTree
import Lean.Elab.Tactic.Simp

/-!
# Helper functions for using the simplifier.
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Lean/Name.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ Authors: Scott Morrison
-/
import Std.Data.HashMap.Basic
import Std.Lean.SMap
import Std.Lean.Name

/-!
# Additional functions on `Lean.Name`.
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/Congr!.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,7 @@ Copyright (c) 2023 Kyle Miller. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kyle Miller
-/
import Lean.Elab.Tactic.Config
import Mathlib.Lean.Meta.CongrTheorems
import Mathlib.Tactic.Relation.Rfl
import Std.Logic
Expand Down
2 changes: 2 additions & 0 deletions Mathlib/Tactic/LibrarySearch.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,9 @@ Authors: Gabriel Ebner, Scott Morrison
-/
import Std.Util.Pickle
import Std.Util.Cache
import Std.Lean.Parser
import Std.Tactic.SolveByElim
import Std.Tactic.TryThis
import Std.Data.MLList.Heartbeats
import Mathlib.Lean.Meta
import Mathlib.Lean.Meta.DiscrTree
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/Monotonicity/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ Authors: Simon Hudon
-/
import Mathlib.Tactic.Monotonicity.Attr
import Std.Tactic.SolveByElim
import Std.Lean.Parser

/-! # Monotonicity tactic
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/NormNum/Core.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,6 +7,7 @@ import Std.Lean.Parser
import Std.Lean.Meta.DiscrTree
import Mathlib.Tactic.NormNum.Result
import Mathlib.Util.Qq
import Lean.Elab.Tactic.Location

/-!
## `norm_num` core functionality
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/PushNeg.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,7 @@ import Mathlib.Logic.Basic
import Mathlib.Init.Order.Defs
import Mathlib.Tactic.Conv
import Mathlib.Init.Set
import Lean.Elab.Tactic.Location

set_option autoImplicit true

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Relation/Trans.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Siddhartha Gadgil, Mario Carneiro
-/
import Mathlib.Lean.Meta
import Mathlib.Lean.Elab.Tactic.Basic
import Lean.Elab.Tactic.Location

/-!
# `trans` tactic
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/Rewrites.lean
Original file line number Diff line number Diff line change
Expand Up @@ -13,6 +13,7 @@ import Mathlib.Control.Basic
import Mathlib.Data.MLList.Dedup
import Mathlib.Lean.Expr.Basic
import Mathlib.Lean.Meta.DiscrTree
import Lean.Elab.Tactic.Location

/-!
# The `rewrites` tactic.
Expand Down
2 changes: 2 additions & 0 deletions Mathlib/Tactic/Says.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,8 @@ Authors: Kim Liesinger
-/
import Std.Data.String.Basic
import Std.Tactic.GuardMsgs
import Std.Tactic.TryThis
import Std.Linter.UnreachableTactic
import Qq.Match

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic/Simps/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Floris van Doorn. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Floris van Doorn
-/

import Lean.Elab.Tactic.Simp
import Mathlib.Tactic.Simps.NotationClass
import Std.Classes.Dvd
import Std.Data.String.Basic
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/Widget/Calc.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ Authors: Patrick Massot
-/
import Lean.Elab.Tactic.Calc
import Std.CodeAction
import Std.Data.Json

import Mathlib.Data.String.Defs
import Mathlib.Tactic.Widget.SelectPanelUtils
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/Widget/Conv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,7 @@ Copyright (c) 2023 Robin Böhne. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Robin Böhne, Wojciech Nawrocki, Patrick Massot
-/
import Std.Data.Json
import Mathlib.Tactic.Widget.SelectPanelUtils
import Mathlib.Data.String.Defs

Expand Down
4 changes: 2 additions & 2 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "2a1b7546b2df0f8e65a70d3b228c30d91752acc4",
"rev": "6132dd32b49f17b1d300aba3fb15966e8f489432",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -22,7 +22,7 @@
{"url": "https://github.com/leanprover-community/aesop",
"type": "git",
"subDir": null,
"rev": "4746cab6320a0d87ec951105ccd42e656fb15e89",
"rev": "204c8f47bd79fba6b53d72536826a97fd58c016a",
"name": "aesop",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
Expand Down
2 changes: 2 additions & 0 deletions test/says.lean
Original file line number Diff line number Diff line change
@@ -1,6 +1,8 @@
import Mathlib.Tactic.Says
import Mathlib.Tactic.RunCmd
import Aesop
import Std.Tactic.ShowTerm
import Std.Tactic.SimpTrace

set_option autoImplicit true
/--
Expand Down

0 comments on commit 359fc77

Please sign in to comment.