Skip to content

Commit

Permalink
chore(logic/equiv/basic): split into two files (#17038)
Browse files Browse the repository at this point in the history
A fairly easy split of `logic.equiv.basic` into `logic.equiv.defs` (containing the stuff with very little prerequisites, and which suffices for many other files), and `logic.equiv.basic` (the stuff that requires other imports from around `logic.*`).

`logic.equiv.basic` is still a ~1500 line file, so I'd like to split it further shortly.



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Oct 18, 2022
1 parent 8c9b005 commit 9407b03
Show file tree
Hide file tree
Showing 29 changed files with 853 additions and 820 deletions.
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 logic.equiv.basic
import logic.equiv.defs

/-!
# Free constructions
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 logic.equiv.basic
import logic.equiv.defs
import data.finite.defs
/-!
# Type tags that turn additive structures into multiplicative, and vice versa
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/group/with_one.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Mario Carneiro, Johan Commelin
-/
import algebra.hom.equiv
import algebra.ring.basic
import logic.equiv.basic
import logic.equiv.defs
import logic.equiv.option

/-!
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 logic.equiv.basic
import logic.equiv.defs
import logic.nontrivial

/-!
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 logic.equiv.basic
import logic.equiv.defs

/-!
# Full and faithful functors
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 logic.equiv.basic
import logic.equiv.defs

/-!
# The category `Type`.
Expand Down
2 changes: 1 addition & 1 deletion src/combinatorics/derangements/basic.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Henry Swanson
-/
import dynamics.fixed_points.basic
import group_theory.perm.option
import logic.equiv.basic
import logic.equiv.defs
import logic.equiv.option

/-!
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 logic.equiv.basic
import logic.equiv.defs

/-!
# Functions functorial with respect to equivalences
Expand Down
2 changes: 1 addition & 1 deletion src/control/monad/basic.lean
Expand Up @@ -3,7 +3,7 @@ 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 logic.equiv.defs
import tactic.basic

/-!
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 logic.equiv.basic
import logic.equiv.defs

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

Expand Down
2 changes: 1 addition & 1 deletion src/control/traversable/equiv.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon
-/
import control.traversable.lemmas
import logic.equiv.basic
import logic.equiv.defs

/-!
# Transferring `traversable` instances along isomorphisms
Expand Down
2 changes: 1 addition & 1 deletion src/data/erased.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Mario Carneiro. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/
import logic.equiv.basic
import logic.equiv.defs

/-!
# A type for VM-erased data
Expand Down
2 changes: 1 addition & 1 deletion src/data/opposite.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison, Reid Barton, Simon Hudon, Kenny Lau
-/
import logic.equiv.basic
import logic.equiv.defs

/-!
# Opposites
Expand Down
2 changes: 1 addition & 1 deletion src/data/part.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Jeremy Avigad, Simon Hudon
-/
import data.set.basic
import logic.equiv.basic
import logic.equiv.defs

/-!
# Partial values of a type
Expand Down
2 changes: 1 addition & 1 deletion src/logic/embedding.lean
Expand Up @@ -7,7 +7,7 @@ import data.fun_like.embedding
import data.prod.pprod
import data.set.basic
import data.sigma.basic
import logic.equiv.basic
import logic.equiv.defs

/-!
# Injective functions
Expand Down

0 comments on commit 9407b03

Please sign in to comment.