Skip to content

Commit

Permalink
refactor(data/finsupp/basic): split data/finsupp/basic into three p…
Browse files Browse the repository at this point in the history
…arts (#15699)

This PR splits the ~2900 lines of `data/finsupp/basic` into more manageable parts:
* the most basic material (~1000 lines) moves to `data/finsupp/defs`
* lemmas about `finsupp.sum` and `finsupp.prod` move to `algebra/big_operators/finsupp`
* the remaining less-used definitions and lemmas remain in `data/finsupp/basic` (~1600 lines)
  • Loading branch information
stuart-presnell committed Aug 19, 2022
1 parent 0fc5496 commit f9c3000
Show file tree
Hide file tree
Showing 17 changed files with 1,629 additions and 1,549 deletions.
3 changes: 1 addition & 2 deletions src/algebra/big_operators/associated.lean
Expand Up @@ -5,8 +5,7 @@ Authors: Johannes Hölzl, Jens Wagemaker, Anne Baanen
-/

import algebra.associated
import algebra.big_operators.basic
import data.finsupp.basic
import algebra.big_operators.finsupp

/-!
# Products of associated, prime, and irreducible elements.
Expand Down
460 changes: 457 additions & 3 deletions src/algebra/big_operators/finsupp.lean

Large diffs are not rendered by default.

1 change: 1 addition & 0 deletions src/data/finset/finsupp.lean
Expand Up @@ -3,6 +3,7 @@ Copyright (c) 2022 Yaël Dillies. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import algebra.big_operators.finsupp
import data.finset.pointwise
import data.finsupp.indicator
import data.fintype.card
Expand Down
1,702 changes: 170 additions & 1,532 deletions src/data/finsupp/basic.lean

Large diffs are not rendered by default.

2 changes: 1 addition & 1 deletion src/data/finsupp/big_operators.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yakov Pechersky
-/

import data.finsupp.basic
import data.finsupp.defs

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/data/finsupp/default.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Chris Hughes. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Chris Hughes
-/
import data.finsupp.basic
import data.finsupp.defs
/-!
# Default finsupp file
This file imports `data.finsupp.basic`
Expand Down

0 comments on commit f9c3000

Please sign in to comment.