Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit c3019c7

Browse files
committed
refactor(data/fintype/basic): split file (#17578)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent 7f96363 commit c3019c7

File tree

90 files changed

+2122
-1796
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

90 files changed

+2122
-1796
lines changed

archive/100-theorems-list/73_ascending_descending_sequences.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2020 Bhavik Mehta. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Bhavik Mehta
55
-/
6-
import data.fintype.basic
6+
import data.fintype.powerset
77

88
/-!
99
# Erdős–Szekeres theorem

archive/imo/imo1987_q1.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,9 @@ Copyright (c) 2021 Yury Kudryashov. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yury Kudryashov
55
-/
6-
import data.fintype.card
6+
import data.fintype.big_operators
7+
import data.fintype.perm
8+
import data.fintype.prod
79
import dynamics.fixed_points.basic
810

911
/-!

archive/imo/imo1994_q1.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Antoine Labelle
55
-/
66
import algebra.big_operators.basic
77
import algebra.big_operators.order
8-
import data.fintype.card
8+
import data.fintype.big_operators
99
import data.finset.sort
1010
import data.fin.interval
1111
import tactic.linarith

src/algebra/big_operators/basic.lean

Lines changed: 11 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -7,9 +7,11 @@ Authors: Johannes Hölzl
77
import algebra.group.pi
88
import algebra.hom.equiv.basic
99
import algebra.ring.opposite
10-
import data.finset.fold
11-
import data.fintype.basic
1210
import data.set.pairwise
11+
import data.finset.sum
12+
import data.fintype.basic
13+
import data.finset.sigma
14+
import algebra.group_power.lemmas
1315

1416
/-!
1517
# Big operators
@@ -1414,7 +1416,13 @@ end
14141416
@[simp]
14151417
lemma sum_boole {s : finset α} {p : α → Prop} [non_assoc_semiring β] {hp : decidable_pred p} :
14161418
(∑ x in s, if p x then (1 : β) else (0 : β)) = (s.filter p).card :=
1417-
by simp [sum_ite]
1419+
by simp only [add_zero,
1420+
mul_one,
1421+
finset.sum_const,
1422+
nsmul_eq_mul,
1423+
eq_self_iff_true,
1424+
finset.sum_const_zero,
1425+
finset.sum_ite]
14181426

14191427
lemma _root_.commute.sum_right [non_unital_non_assoc_semiring β] (s : finset α)
14201428
(f : α → β) (b : β) (h : ∀ i ∈ s, commute b (f i)) :

src/algebra/big_operators/fin.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2020 Yury Kudryashov, Anne Baanen. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yury Kudryashov, Anne Baanen
55
-/
6-
import data.fintype.card
6+
import data.fintype.big_operators
77
import data.fintype.fin
88
import logic.equiv.fin
99

src/algebra/big_operators/pi.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,8 @@ Copyright (c) 2018 Simon Hudon. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Simon Hudon, Patrick Massot
55
-/
6+
import data.fintype.card
7+
import algebra.group.prod
68
import algebra.big_operators.basic
79
import algebra.ring.pi
810

src/algebra/char_zero.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,8 @@ Authors: Mario Carneiro
55
-/
66

77
import data.nat.cast.field
8-
import data.fintype.basic
8+
import data.fintype.lattice
9+
import algebra.group_power.lemmas
910

1011
/-!
1112
# Characteristic zero (additional theorems)

src/algebra/group/conj.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -8,6 +8,7 @@ import algebra.group_with_zero.basic
88
import algebra.hom.aut
99
import algebra.hom.group
1010
import data.finite.basic
11+
import data.fintype.units
1112

1213
/-!
1314
# Conjugacy of group elements

src/algebra/order/field/pi.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: Yaël Dillies
55
-/
66
import algebra.order.field.basic
7-
import data.fintype.basic
7+
import data.fintype.lattice
88

99
/-!
1010
# Lemmas about (finite domain) functions into fields.

src/algebra/order/field/power.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2014 Robert Lewis. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Robert Lewis, Leonardo de Moura, Mario Carneiro, Floris van Doorn
55
-/
6+
import algebra.parity
67
import algebra.char_zero
78
import algebra.group_with_zero.power
89
import algebra.order.field.basic

0 commit comments

Comments
 (0)