File tree Expand file tree Collapse file tree 1 file changed +5
-2
lines changed Expand file tree Collapse file tree 1 file changed +5
-2
lines changed Original file line number Diff line number Diff line change @@ -88,14 +88,14 @@ lemma stabilizerMulEquiv_apply (g : (stabilizer (Perm α)ᵈᵐᵃ f)ᵐᵒᵖ)
88
88
89
89
section Fintype
90
90
91
- variable [Fintype α] [DecidableEq α] [DecidableEq ι]
91
+ variable [Fintype α]
92
92
93
93
open Nat
94
94
95
95
variable (f)
96
96
97
97
/-- The cardinality of the type of permutations preserving a function -/
98
- theorem stabilizer_card [Fintype ι] :
98
+ theorem stabilizer_card [DecidableEq α] [DecidableEq ι] [ Fintype ι] :
99
99
Fintype.card {g : Perm α // f ∘ g = f} = ∏ i, (Fintype.card {a // f a = i})! := by
100
100
-- rewriting via Nat.card because Fintype instance is not found
101
101
rw [← Nat.card_eq_fintype_card,
@@ -108,9 +108,12 @@ theorem stabilizer_card [Fintype ι] :
108
108
/-- The cardinality of the set of permutations preserving a function -/
109
109
theorem stabilizer_ncard [Fintype ι] :
110
110
Set.ncard {g : Perm α | f ∘ g = f} = ∏ i, (Set.ncard {a | f a = i})! := by
111
+ classical
111
112
simp only [← Set.Nat.card_coe_set_eq, Set.coe_setOf, card_eq_fintype_card]
112
113
exact stabilizer_card f
113
114
115
+ variable [DecidableEq α] [DecidableEq ι]
116
+
114
117
/-- The cardinality of the type of permutations preserving a function
115
118
(without the finiteness assumption on target)-/
116
119
theorem stabilizer_card' :
You can’t perform that action at this time.
0 commit comments