Skip to content

Commit f0587c5

Browse files
committed
chore(Logic/Function/Defs): move file out of Init (#14754)
1 parent 60750e1 commit f0587c5

File tree

21 files changed

+58
-45
lines changed

21 files changed

+58
-45
lines changed

Mathlib.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2742,7 +2742,6 @@ import Mathlib.Init.Data.Quot
27422742
import Mathlib.Init.Data.Rat.Basic
27432743
import Mathlib.Init.Data.Sigma.Basic
27442744
import Mathlib.Init.Data.Sigma.Lex
2745-
import Mathlib.Init.Function
27462745
import Mathlib.Init.Logic
27472746
import Mathlib.Init.Meta.WellFoundedTactics
27482747
import Mathlib.Init.Order.Defs
@@ -2995,9 +2994,11 @@ import Mathlib.Logic.Equiv.TransferInstance
29952994
import Mathlib.Logic.Function.Basic
29962995
import Mathlib.Logic.Function.CompTypeclasses
29972996
import Mathlib.Logic.Function.Conjugate
2997+
import Mathlib.Logic.Function.Defs
29982998
import Mathlib.Logic.Function.FromTypes
29992999
import Mathlib.Logic.Function.Iterate
30003000
import Mathlib.Logic.Function.OfArity
3001+
import Mathlib.Logic.Function.ULift
30013002
import Mathlib.Logic.Godel.GodelBetaFunction
30023003
import Mathlib.Logic.Hydra
30033004
import Mathlib.Logic.IsEmpty

Mathlib/CategoryTheory/Yoneda.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -6,6 +6,7 @@ Authors: Scott Morrison
66
import Mathlib.CategoryTheory.Functor.Hom
77
import Mathlib.CategoryTheory.Products.Basic
88
import Mathlib.Data.ULift
9+
import Mathlib.Logic.Function.ULift
910

1011
#align_import category_theory.yoneda from "leanprover-community/mathlib"@"369525b73f229ccd76a6ec0e0e0bf2be57599768"
1112

Mathlib/Control/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl
55
-/
66
import Mathlib.Control.Combinators
7-
import Mathlib.Init.Function
7+
import Mathlib.Logic.Function.Defs
88
import Mathlib.Tactic.CasesM
99
import Mathlib.Tactic.Attr.Core
1010

Mathlib/Control/Traversable/Basic.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -5,6 +5,7 @@ Authors: Simon Hudon
55
-/
66
import Mathlib.Data.Option.Defs
77
import Mathlib.Control.Functor
8+
import Batteries.Data.List.Basic
89

910
#align_import control.traversable.basic from "leanprover-community/mathlib"@"1fc36cc9c8264e6e81253f88be7fb2cb6c92d76a"
1011

Mathlib/Data/Bool/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2014 Microsoft Corporation. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Leonardo de Moura, Jeremy Avigad
55
-/
6-
import Mathlib.Init.Function
6+
import Mathlib.Logic.Function.Defs
77
import Mathlib.Init.Order.Defs
88

99
#align_import data.bool.basic from "leanprover-community/mathlib"@"c4658a649d216f57e99621708b09dcb3dcccbd23"

Mathlib/Data/List/Defs.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -8,6 +8,7 @@ import Mathlib.Control.Functor
88
import Mathlib.Data.SProd
99
import Mathlib.Util.CompileInductive
1010
import Batteries.Tactic.Lint.Basic
11+
import Batteries.Data.List.Lemmas
1112

1213
#align_import data.list.defs from "leanprover-community/mathlib"@"d2d8742b0c21426362a9dacebc6005db895ca963"
1314

Mathlib/Data/Option/NAry.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2022 Yaël Dillies. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yaël Dillies
55
-/
6-
import Mathlib.Init.Function
6+
import Mathlib.Logic.Function.Defs
77

88
#align_import data.option.n_ary from "leanprover-community/mathlib"@"995b47e555f1b6297c7cf16855f1023e355219fb"
99

Mathlib/Data/Prod/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2017 Johannes Hölzl. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl
55
-/
6-
import Mathlib.Init.Function
6+
import Mathlib.Logic.Function.Defs
77
import Mathlib.Logic.Function.Iterate
88
import Mathlib.Tactic.Inhabit
99

Mathlib/Data/Prod/PProd.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2020 Eric Wieser. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Eric Wieser
55
-/
6-
import Mathlib.Init.Function
6+
import Mathlib.Logic.Function.Defs
77

88
#align_import data.prod.pprod from "leanprover-community/mathlib"@"c4658a649d216f57e99621708b09dcb3dcccbd23"
99

Mathlib/Data/Sigma/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2017 Johannes Hölzl. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl
55
-/
6-
import Mathlib.Init.Function
6+
import Mathlib.Logic.Function.Defs
77
import Mathlib.Logic.Function.Basic
88

99
#align_import data.sigma.basic from "leanprover-community/mathlib"@"a148d797a1094ab554ad4183a4ad6f130358ef64"

0 commit comments

Comments
 (0)