Skip to content

Commit 3ce877a

Browse files
committed
chore(DomMulAct): remove decidability assumptions (#17510)
Found by the linter in #10235.
1 parent 4c46b67 commit 3ce877a

File tree

1 file changed

+5
-2
lines changed

1 file changed

+5
-2
lines changed

Mathlib/GroupTheory/Perm/DomMulAct.lean

Lines changed: 5 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -88,14 +88,14 @@ lemma stabilizerMulEquiv_apply (g : (stabilizer (Perm α)ᵈᵐᵃ f)ᵐᵒᵖ)
8888

8989
section Fintype
9090

91-
variable [Fintype α] [DecidableEq α] [DecidableEq ι]
91+
variable [Fintype α]
9292

9393
open Nat
9494

9595
variable (f)
9696

9797
/-- The cardinality of the type of permutations preserving a function -/
98-
theorem stabilizer_card [Fintype ι] :
98+
theorem stabilizer_card [DecidableEq α] [DecidableEq ι] [Fintype ι] :
9999
Fintype.card {g : Perm α // f ∘ g = f} = ∏ i, (Fintype.card {a // f a = i})! := by
100100
-- rewriting via Nat.card because Fintype instance is not found
101101
rw [← Nat.card_eq_fintype_card,
@@ -108,9 +108,12 @@ theorem stabilizer_card [Fintype ι] :
108108
/-- The cardinality of the set of permutations preserving a function -/
109109
theorem stabilizer_ncard [Fintype ι] :
110110
Set.ncard {g : Perm α | f ∘ g = f} = ∏ i, (Set.ncard {a | f a = i})! := by
111+
classical
111112
simp only [← Set.Nat.card_coe_set_eq, Set.coe_setOf, card_eq_fintype_card]
112113
exact stabilizer_card f
113114

115+
variable [DecidableEq α] [DecidableEq ι]
116+
114117
/-- The cardinality of the type of permutations preserving a function
115118
(without the finiteness assumption on target)-/
116119
theorem stabilizer_card':

0 commit comments

Comments
 (0)