Skip to content

Commit

Permalink
chore: remove unnecessary classical! (#12255)
Browse files Browse the repository at this point in the history
`classical!` appears to never actually be necessary, and is just being used out of habit, and we can get rid of it to reduce the number of ways to say the same thing.

Co-authored-by: Scott Morrison <[email protected]>
  • Loading branch information
kim-em and kim-em committed Apr 19, 2024
1 parent 9e7997a commit 1d4a722
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Data/Set/Pointwise/Finite.lean
Original file line number Diff line number Diff line change
Expand Up @@ -194,7 +194,7 @@ theorem card_pow_eq_card_pow_card_univ [∀ k : ℕ, DecidablePred (· ∈ S ^ k
fun n h ↦ le_antisymm (mono (n + 1).le_succ) (key a⁻¹ (S ^ (n + 2)) (S ^ (n + 1)) _)
replace h₂ : S ^ n * {a} = S ^ (n + 1) := by
have : Fintype (S ^ n * Set.singleton a) := by
classical!
classical
apply fintypeMul
refine' Set.eq_of_subset_of_card_le _ (le_trans (ge_of_eq h) _)
· exact mul_subset_mul Set.Subset.rfl (Set.singleton_subset_iff.mpr ha)
Expand Down

0 comments on commit 1d4a722

Please sign in to comment.