Skip to content

Commit

Permalink
move(data/pi/*): Group pi files (#13826)
Browse files Browse the repository at this point in the history
Move `data.pi` to `data.pi.algebra` and `order.pilex` to `data.pi.lex`.
  • Loading branch information
YaelDillies committed May 3, 2022
1 parent 8a5b4a7 commit 4cea0a8
Show file tree
Hide file tree
Showing 6 changed files with 5 additions and 4 deletions.
2 changes: 1 addition & 1 deletion src/algebra/group/pi.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon, Patrick Massot
-/
import algebra.hom.group_instances
import data.pi
import data.pi.algebra
import data.set.function
import data.set.pairwise
import tactic.pi_instances
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/hom/equiv.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov
-/
import algebra.group.type_tags
import algebra.group_with_zero.basic
import data.pi
import data.pi.algebra

/-!
# Multiplicative and additive equivs
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/ring/basic.lean
Expand Up @@ -6,7 +6,7 @@ Neil Strickland
-/
import algebra.divisibility
import algebra.regular.basic
import data.pi
import data.pi.algebra

/-!
# Properties and homomorphisms of semirings and rings
Expand Down
3 changes: 2 additions & 1 deletion src/data/fin/tuple/basic.lean
Expand Up @@ -4,7 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Floris van Doorn, Yury Kudryashov, Sébastien Gouëzel, Chris Hughes
-/
import data.fin.basic
import order.pilex
import data.pi.lex

/-!
# Operation on tuples
Expand Down
File renamed without changes.
File renamed without changes.

0 comments on commit 4cea0a8

Please sign in to comment.