Skip to content

Commit

Permalink
fix no-longer inferred instance
Browse files Browse the repository at this point in the history
  • Loading branch information
pechersky committed Aug 1, 2021
1 parent 1763b43 commit 4d8c0b0
Showing 1 changed file with 4 additions and 1 deletion.
5 changes: 4 additions & 1 deletion src/group_theory/specific_groups/dihedral.lean
Original file line number Diff line number Diff line change
Expand Up @@ -113,7 +113,10 @@ instance : nontrivial (dihedral_group n) := ⟨⟨r 0, sr 0, dec_trivial⟩⟩
If `0 < n`, then `dihedral_group n` has `2n` elements.
-/
lemma card [fact (0 < n)] : fintype.card (dihedral_group n) = 2 * n :=
by rw [← fintype.card_eq.mpr ⟨fintype_helper⟩, fintype.card_sum, zmod.card, two_mul]
begin
rw [← fintype.card_eq.mpr ⟨fintype_helper⟩, fintype.card_sum, zmod.card, two_mul],
apply_instance
end

@[simp] lemma r_one_pow (k : ℕ) : (r 1 : dihedral_group n) ^ k = r k :=
begin
Expand Down

0 comments on commit 4d8c0b0

Please sign in to comment.