Skip to content

Commit

Permalink
chore: bump to 2023-01-04 (#1335)
Browse files Browse the repository at this point in the history
  • Loading branch information
gebner committed Jan 4, 2023
1 parent 047e52a commit 7e2613a
Show file tree
Hide file tree
Showing 36 changed files with 6 additions and 92 deletions.
1 change: 0 additions & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -593,7 +593,6 @@ import Mathlib.Testing.SlimCheck.Sampleable
import Mathlib.Testing.SlimCheck.Testable
import Mathlib.Util.Export
import Mathlib.Util.IncludeStr
import Mathlib.Util.MapsTo
import Mathlib.Util.MemoFix
import Mathlib.Util.Simp
import Mathlib.Util.Syntax
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Control/Functor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,6 +10,7 @@ Authors: Simon Hudon
-/
import Mathlib.Control.Basic
import Mathlib.Init.Set
import Std.Tactic.Lint

/-!
# Functors
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Data/KVMap.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Alex J. Best
-/
import Lean.Data.KVMap
import Mathlib.Util.MapsTo

/-!
# Additional functionality for `KVMap`
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Init/Data/Fin/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Leonardo de Moura
-/
import Mathlib.Init.Data.Nat.Notation
import Mathlib.Util.MapsTo

/-!
# Theorems about equality in `Fin`.
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Init/Set.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Leonardo de Moura
-/
import Lean.Parser.Term
import Mathlib.Util.MapsTo
import Std.Classes.SetNotation
import Mathlib.Mathport.Rename

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Lean/Expr/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Mario Carneiro, Simon Hudon, Scott Morrison, Keeley Hoek, Robert Y. Lew
Floris van Doorn, E.W.Ayers, Arthur Paulino
-/
import Lean
import Mathlib.Util.MapsTo
import Std.Lean.Expr
import Std.Data.List.Basic

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Lean/Meta.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ Authors: Mario Carneiro
import Lean.Elab
import Lean.Meta.Tactic.Assert
import Lean.Meta.Tactic.Clear
import Mathlib.Util.MapsTo

/-! ## Additional utilities in `Lean.MVarId` -/

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Mathport/Rename.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Daniel Selsam
-/
import Lean
import Mathlib.Util.MapsTo

namespace Mathlib.Prelude.Rename

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/Antichain.lean
Original file line number Diff line number Diff line change
Expand Up @@ -338,7 +338,7 @@ variable {ι : Type _} {α : ι → Type _} [∀ i, Preorder (α i)] {s t : Set

-- Porting note: local notation given a name because of https://github.com/leanprover/lean4/issues/2000
@[inherit_doc]
local infixl:50 (name := «OrderAntichainLocal≺») " ≺ " => StrongLT
local infixl:50 " ≺ " => StrongLT

/-- A weak antichain in `Π i, α i` is a set such that no two distinct elements are strongly less
than each other. -/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/Chain.lean
Original file line number Diff line number Diff line change
Expand Up @@ -45,7 +45,7 @@ variable (r : α → α → Prop)

/-- In this file, we use `≺` as a local notation for any relation `r`. -/
-- Porting note: local notation given a name because of https://github.com/leanprover/lean4/issues/2000
local infixl:50 (name := «OrderChainLocal≺») " ≺ " => r
local infixl:50 " ≺ " => r

/-- A chain is a set `s` satisfying `x ≺ y ∨ x = y ∨ y ≺ x` for all `x y ∈ s`. -/
def IsChain (s : Set α) : Prop :=
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/Zorn.lean
Original file line number Diff line number Diff line change
Expand Up @@ -72,7 +72,7 @@ variable {α β : Type _} {r : α → α → Prop} {c : Set α}

/-- Local notation for the relation being considered. -/
-- Porting note: local notation given a name because of https://github.com/leanprover/lean4/issues/2000
local infixl:50 (name := «OrderZornLocal≺») " ≺ " => r
local infixl:50 " ≺ " => r

/-- **Zorn's lemma**
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Alias.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, David Renshaw
-/
import Lean
import Mathlib.Util.MapsTo

/-!
# The `alias` command
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/ApplyRules.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ Authors: Scott Morrison
import Lean
import Std.Util.TermUnsafe
import Std.Lean.Meta.Basic
import Mathlib.Util.MapsTo

/-!
# The `apply_rules` tactic
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ Authors: Mario Carneiro
import Lean
import Std
import Mathlib.Tactic.Cases
import Mathlib.Util.MapsTo

namespace Mathlib.Tactic
open Lean Parser.Tactic Elab Command Elab.Tactic Meta
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/CasesM.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/
import Lean
import Mathlib.Util.MapsTo

/-!
# `casesm`, `cases_type`, `constructorm` tactics
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Clear!.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joshua Clune
-/
import Lean
import Mathlib.Util.MapsTo

/-! # `clear!` tactic -/

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/ClearExcept.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joshua Clune
-/
import Lean
import Mathlib.Util.MapsTo

open Lean.Meta

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Clear_.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joshua Clune
-/
import Lean
import Mathlib.Util.MapsTo

/-! # `clear_` tactic -/

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Coe.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner
-/
import Lean
import Mathlib.Util.MapsTo

open Lean Elab Term Meta

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Convert.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import Lean
import Mathlib.Util.MapsTo

/-!
# The `convert` tactic.
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Have.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Arthur Paulino, Edward Ayers, Mario Carneiro
-/
import Lean
import Mathlib.Data.Array.Defs
import Mathlib.Util.MapsTo

/--
Uses `checkColGt` to prevent
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/IrreducibleDef.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner
-/
import Lean
import Mathlib.Util.MapsTo

/-!
# Irreducible definitions
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/LeftRight.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Siddhartha Gadgil
-/
import Lean
import Mathlib.Util.MapsTo

namespace Mathlib.Tactic.LeftRight
open Lean Meta Elab Tactic
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/PrintPrefix.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Shing Tak Lam, Daniel Selsam, Mario Carneiro
-/
import Lean.Elab.Command
import Mathlib.Util.MapsTo

open Lean Meta Elab Command

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Relation/Rfl.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Newell Jensen
-/
import Lean
import Mathlib.Util.MapsTo

/-!
# `rfl` tactic extension for reflexive relations
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Rename.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner
-/
import Lean
import Mathlib.Util.MapsTo

namespace Mathlib.Tactic

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/RunCmd.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sebastian Ullrich, Mario Carneiro
-/
import Lean.Elab.Eval
import Mathlib.Util.MapsTo
import Std.Util.TermUnsafe

/-!
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/Set.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Ian Benway.
-/
import Lean
import Mathlib.Util.MapsTo

namespace Mathlib.Tactic
open Lean Elab Elab.Tactic Meta
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/SimpIntro.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Mario Carneiro
-/
import Lean
import Std.Lean.Parser
import Mathlib.Util.MapsTo

/-! # `simp_intro` tactic -/

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic/SudoSetOption.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Gabriel Ebner
-/

import Lean
import Mathlib.Util.MapsTo

/-!
# Defines the `sudo set_option` command.
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Tactic/ToAdditive.lean
Original file line number Diff line number Diff line change
Expand Up @@ -16,6 +16,7 @@ import Mathlib.Tactic.Relation.Rfl -- just to copy the attribute
import Mathlib.Tactic.Relation.Symm -- just to copy the attribute
import Mathlib.Tactic.Relation.Trans -- just to copy the attribute
import Mathlib.Tactic.RunCmd -- not necessary, but useful for debugging
import Std.Tactic.Lint.Simp -- for DiscrTree.elements

/-!
# The `@[to_additive]` attribute.
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Util/Export.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/
import Lean
import Mathlib.Util.MapsTo

/-!
A rudimentary export format, adapted from
Expand Down
59 changes: 0 additions & 59 deletions Mathlib/Util/MapsTo.lean

This file was deleted.

1 change: 0 additions & 1 deletion Mathlib/Util/Simp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ Authors: Gabriel Ebner

import Lean
import Std.Tactic.OpenPrivate
import Mathlib.Util.MapsTo

/-!
# Helper functions for the `norm_cast` tactic.
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Util/WithWeakNamespace.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Mario Carneiro, Daniel Selsam, Gabriel Ebner
-/

import Lean
import Mathlib.Util.MapsTo

/-!
# Defines `with_weak_namespace` command.
Expand Down
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:nightly-2022-12-23
leanprover/lean4:nightly-2023-01-04

0 comments on commit 7e2613a

Please sign in to comment.