Skip to content

Commit

Permalink
remove decidability instance
Browse files Browse the repository at this point in the history
  • Loading branch information
MichaelStollBayreuth committed Jun 27, 2022
1 parent a4af8b1 commit 4f34377
Showing 1 changed file with 0 additions and 3 deletions.
3 changes: 0 additions & 3 deletions src/number_theory/legendre_symbol/mul_character.lean
Original file line number Diff line number Diff line change
Expand Up @@ -476,9 +476,6 @@ begin
exact eq_zero_of_mul_eq_self_left hb h₁,
end

-- this can go once #14873 is merged
instance {M} [monoid M] (x : M) [h : decidable (∃ u : Mˣ, ↑u = x)] : decidable (is_unit x) := h

/-- The sum over all values of the trivial multiplicative character on a finite ring is
the cardinality of its unit group. -/
lemma sum_eq_card_units_of_is_trivial [fintype R] [decidable_eq R] :
Expand Down

0 comments on commit 4f34377

Please sign in to comment.