Skip to content

Commit

Permalink
chore(data/equiv): split and move to logic/equiv (#12929)
Browse files Browse the repository at this point in the history
Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Rearranging.20files.20in.20.60data.2F.60

This PR rearranges files in `data/equiv/` by 1) moving bundled isomorphisms to a relevant subfolder of `algebra/`; 2) moving `denumerable` and `encodable` to `logic/`; 3) moving the remainder of `data/equiv/` to `logic/equiv/`. The commits of this PR correspond to those steps.

In particular, the following files were moved:

 * `data/equiv/module.lean` → `algebra/module/equiv.lean`
 * `data/equiv/mul_add.lean` → `algebra/hom/equiv.lean`
 * `data/equiv/mul_add_aut.lean` → `algebra/hom/aut.lean`
 * `data/equiv/ring.lean` → `algebra/ring/equiv.lean`
 * `data/equiv/ring_aut.lean` → `algebra/ring/aut.lean`
 * `data/equiv/denumerable.lean` → `logic/denumerable.lean`
 * `data/equiv/encodable/*.lean` → `logic/encodable/basic.lean logic/encodable/lattice.lean logic/encodable/small.lean`
 * `data/equiv/*.lean` to: `logic/equiv/basic.lean logic/equiv/fin.lean logic/equiv/functor.lean logic/equiv/local_equiv.lean logic/equiv/option.lean logic/equiv/transfer_instance.lean logic/equiv/embedding.lean logic/equiv/fintype.lean logic/equiv/list.lean logic/equiv/nat.lean logic/equiv/set.lean`
  • Loading branch information
Vierkantor committed Mar 26, 2022
1 parent 434a938 commit cc8c90d
Show file tree
Hide file tree
Showing 118 changed files with 148 additions and 148 deletions.
2 changes: 1 addition & 1 deletion src/algebra/algebra/basic.lean
Expand Up @@ -4,9 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau, Yury Kudryashov
-/
import algebra.module.basic
import algebra.ring.aut
import linear_algebra.span
import tactic.abel
import data.equiv.ring_aut

/-!
# Algebras over commutative semirings
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/big_operators/basic.lean
Expand Up @@ -5,8 +5,8 @@ Authors: Johannes Hölzl
-/

import algebra.group.pi
import algebra.hom.equiv
import algebra.ring.opposite
import data.equiv.mul_add
import data.finset.fold
import data.fintype.basic
import data.set.pairwise
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/category/CommRing/basic.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Scott Morrison, Johannes Hölzl, Yury Kudryashov
-/
import algebra.category.Group.basic
import category_theory.concrete_category.reflects_isomorphisms
import data.equiv.ring
import algebra.ring.equiv

/-!
# Category instances for semiring, ring, comm_semiring, and comm_ring.
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/field_power.lean
Expand Up @@ -4,8 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Robert Y. Lewis
-/
import algebra.group_with_zero.power
import algebra.ring.equiv
import tactic.linarith
import data.equiv.ring

/-!
# Integer power operation on fields and division rings
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/free.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Kenny Lau
import algebra.hom.group
import control.applicative
import control.traversable.basic
import data.equiv.basic
import logic.equiv.basic

/-!
# Free constructions
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/group/conj.lean
Expand Up @@ -5,8 +5,8 @@ Authors: Patrick Massot, Chris Hughes, Michael Howes
-/
import algebra.group.semiconj
import algebra.group_with_zero.basic
import algebra.hom.aut
import algebra.hom.group
import data.equiv.mul_add_aut
import data.fintype.basic

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/group/opposite.lean
Expand Up @@ -5,8 +5,8 @@ Authors: Kenny Lau
-/
import algebra.group.inj_surj
import algebra.group.commute
import algebra.hom.equiv
import algebra.opposites
import data.equiv.mul_add

/-!
# Group structures on the multiplicative and additive opposites
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/group/type_tags.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/
import algebra.hom.group
import data.equiv.basic
import logic.equiv.basic
/-!
# Type tags that turn additive structures into multiplicative, and vice versa
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/group/ulift.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import data.equiv.mul_add
import algebra.hom.equiv

/-!
# `ulift` instances for groups and monoids
Expand Down
6 changes: 3 additions & 3 deletions src/algebra/group/with_one.lean
Expand Up @@ -3,10 +3,10 @@ Copyright (c) 2018 Mario Carneiro. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Johan Commelin
-/
import algebra.hom.equiv
import algebra.ring.basic
import data.equiv.basic
import data.equiv.mul_add
import data.equiv.option
import logic.equiv.basic
import logic.equiv.option

/-!
# Adjoining a zero/one to semigroups and related algebraic structures
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/group_ring_action.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau
-/

import data.equiv.ring
import algebra.ring.equiv
import group_theory.group_action.group
import ring_theory.subring.basic

Expand Down
File renamed without changes.
File renamed without changes.
4 changes: 2 additions & 2 deletions src/algebra/lie/basic.lean
Expand Up @@ -3,10 +3,10 @@ Copyright (c) 2019 Oliver Nash. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Oliver Nash
-/
import tactic.noncomm_ring
import data.equiv.module
import algebra.module.equiv
import data.bracket
import linear_algebra.basic
import tactic.noncomm_ring

/-!
# Lie algebras
Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion src/algebra/module/opposites.lean
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2020 Eric Wieser. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import algebra.module.equiv
import group_theory.group_action.opposite
import data.equiv.module

/-!
# Module operations on `Mᵐᵒᵖ`
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/module/submodule.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nathaniel Thomas, Jeremy Avigad, Johannes Hölzl, Mario Carneiro
-/
import algebra.module.linear_map
import data.equiv.module
import algebra.module.equiv
import group_theory.group_action.sub_mul_action
/-!
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/module/ulift.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import algebra.ring.ulift
import data.equiv.module
import algebra.module.equiv

/-!
# `ulift` instances for module and multiplicative actions
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/opposites.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau
-/
import algebra.group.defs
import data.equiv.basic
import logic.equiv.basic
import logic.nontrivial

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/order/hom/ring.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Alex J. Best, Yaël Dillies
-/
import algebra.order.hom.monoid
import algebra.order.ring
import data.equiv.ring
import algebra.ring.equiv

/-!
# Ordered ring homomorphisms
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/order/monoid.lean
Expand Up @@ -6,8 +6,8 @@ Authors: Jeremy Avigad, Leonardo de Moura, Mario Carneiro, Johannes Hölzl
import algebra.group.with_one
import algebra.group.type_tags
import algebra.group.prod
import algebra.hom.equiv
import algebra.order.monoid_lemmas
import data.equiv.mul_add
import order.bounded_order
import order.min_max
import order.hom.basic
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/quandle.lean
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2020 Kyle Miller. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kyle Miller
-/
import algebra.hom.equiv
import data.zmod.basic
import data.equiv.mul_add
import tactic.group

/-!
Expand Down
4 changes: 2 additions & 2 deletions src/algebra/quaternion.lean
Expand Up @@ -3,10 +3,10 @@ Copyright (c) 2020 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import tactic.ring_exp
import algebra.algebra.basic
import algebra.ring.equiv
import algebra.ring.opposite
import data.equiv.ring
import tactic.ring_exp

/-!
# Quaternions
Expand Down
4 changes: 2 additions & 2 deletions src/data/equiv/ring_aut.lean → src/algebra/ring/aut.lean
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2018 Johannes Hölzl. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov
-/
import data.equiv.mul_add_aut
import data.equiv.ring
import algebra.hom.aut
import algebra.ring.equiv

/-!
# Ring automorphisms
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/ring/comp_typeclasses.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Frédéric Dupuis, Heather Macbeth
-/

import algebra.ring.basic
import data.equiv.ring
import algebra.ring.equiv

/-!
# Propositional typeclasses on several ring homs
Expand Down
4 changes: 2 additions & 2 deletions src/data/equiv/ring.lean → src/algebra/ring/equiv.lean
Expand Up @@ -3,10 +3,10 @@ Copyright (c) 2018 Johannes Hölzl. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov
-/
import data.equiv.mul_add
import algebra.big_operators.basic
import algebra.field.basic
import algebra.hom.equiv
import algebra.ring.opposite
import algebra.big_operators.basic

/-!
# (Semi)ring equivs
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/ring/prod.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl, Chris Hughes, Mario Carneiro, Yury Kudryashov
-/
import algebra.group.prod
import algebra.ring.basic
import data.equiv.ring
import algebra.ring.equiv

/-!
# Semiring, ring etc structures on `R × S`
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/ring/ulift.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import algebra.group.ulift
import data.equiv.ring
import algebra.ring.equiv

/-!
# `ulift` instances for ring
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/star/basic.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Scott Morrison
import tactic.apply_fun
import algebra.field.opposite
import algebra.field_power
import data.equiv.ring_aut
import algebra.ring.aut
import group_theory.group_action.units
import group_theory.group_action.opposite
import algebra.ring.comp_typeclasses
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/star/module.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser, Frédéric Dupuis
-/
import algebra.star.self_adjoint
import data.equiv.module
import algebra.module.equiv
import linear_algebra.prod

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/algebraic_geometry/Spec.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Scott Morrison, Justus Springer
-/
import algebraic_geometry.locally_ringed_space
import algebraic_geometry.structure_sheaf
import data.equiv.transfer_instance
import logic.equiv.transfer_instance
import ring_theory.localization.localization_localization
import topology.sheaves.sheaf_condition.sites
import topology.sheaves.functors
Expand Down
2 changes: 1 addition & 1 deletion src/algebraic_geometry/locally_ringed_space.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Johan Commelin

import algebraic_geometry.ringed_space
import algebraic_geometry.stalks
import data.equiv.transfer_instance
import logic.equiv.transfer_instance

/-!
# The category of locally ringed spaces
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/analytic/basic.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Sébastien Gouëzel, Yury Kudryashov
-/
import analysis.calculus.formal_multilinear_series
import analysis.specific_limits.normed
import data.equiv.fin
import logic.equiv.fin

/-!
# Analytic functions
Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/endomorphism.lean
Expand Up @@ -3,9 +3,9 @@ Copyright (c) 2019 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov, Scott Morrison, Simon Hudon
-/
import algebra.hom.equiv
import category_theory.groupoid
import category_theory.opposites
import data.equiv.mul_add
import group_theory.group_action.defs

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/functor/fully_faithful.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import category_theory.natural_isomorphism
import data.equiv.basic
import logic.equiv.basic

/-!
# Full and faithful functors
Expand Down
Expand Up @@ -8,7 +8,7 @@ import category_theory.limits.preserves.shapes.products
import category_theory.limits.shapes.binary_products
import category_theory.limits.shapes.finite_products
import category_theory.pempty
import data.equiv.fin
import logic.equiv.fin

/-!
# Constructing finite products from binary products and terminal.
Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/preadditive/opposite.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Scott Morrison, Adam Topaz
-/
import category_theory.preadditive
import category_theory.preadditive.additive_functor
import data.equiv.transfer_instance
import logic.equiv.transfer_instance

/-!
# If `C` is preadditive, `Cᵒᵖ` has a natural preadditive structure.
Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/types.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Stephen Morgan, Scott Morrison, Johannes Hölzl
-/
import category_theory.epi_mono
import category_theory.functor.fully_faithful
import data.equiv.basic
import logic.equiv.basic

/-!
# The category `Type`.
Expand Down
4 changes: 2 additions & 2 deletions src/combinatorics/derangements/basic.lean
Expand Up @@ -3,10 +3,10 @@ Copyright (c) 2021 Henry Swanson. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Henry Swanson
-/
import data.equiv.basic
import data.equiv.option
import dynamics.fixed_points.basic
import group_theory.perm.option
import logic.equiv.basic
import logic.equiv.option

/-!
# Derangements on types
Expand Down
2 changes: 1 addition & 1 deletion src/computability/primrec.lean
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2018 Mario Carneiro. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/
import data.equiv.list
import data.list.join
import logic.equiv.list
import logic.function.iterate

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/control/equiv_functor.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import data.equiv.basic
import logic.equiv.basic

/-!
# Functions functorial with respect to equivalences
Expand Down
2 changes: 1 addition & 1 deletion src/control/monad/basic.lean
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2019 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon
-/
import logic.equiv.basic
import tactic.basic
import data.equiv.basic

/-!
# Monad
Expand Down
2 changes: 1 addition & 1 deletion src/control/monad/writer.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Simon Hudon
The writer monad transformer for passing immutable state.
-/
import algebra.group.defs
import data.equiv.basic
import logic.equiv.basic

universes u v w u₀ u₁ v₀ v₁

Expand Down

0 comments on commit cc8c90d

Please sign in to comment.