Skip to content

Commit

Permalink
perf: add instance shortcut to remove heartbeat bump (#6410)
Browse files Browse the repository at this point in the history
This removes a maxHeartbeats bump (the only one in the file).
  • Loading branch information
kbuzzard committed Aug 14, 2023
1 parent c54060b commit c1776a3
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion Mathlib/NumberTheory/NumberField/Units.lean
Expand Up @@ -111,7 +111,9 @@ instance [NumberField K] : Fintype (torsion K) := by
· rw [← h_ua]
exact le_of_eq ((eq_iff_eq _ 1).mp ((mem_torsion K).mp h_tors) φ)

set_option synthInstance.maxHeartbeats 30000 in
-- a shortcut instance to stop the next instance from timing out
instance [NumberField K] : Finite (torsion K) := inferInstance

/-- The torsion subgroup is cylic. -/
instance [NumberField K] : IsCyclic (torsion K) := subgroup_units_cyclic _

Expand Down

0 comments on commit c1776a3

Please sign in to comment.