Skip to content

Commit

Permalink
chore(ring_theory/adjoin_root): remove some unused decidable_eq (#1530)
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 authored and mergify[bot] committed Oct 9, 2019
1 parent a17a9a6 commit 7d792ec
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/ring_theory/adjoin_root.lean
Original file line number Diff line number Diff line change
Expand Up @@ -16,13 +16,13 @@ variables {α : Type u} {β : Type v} {γ : Type w}

open polynomial ideal

def adjoin_root [comm_ring α] [decidable_eq α] (f : polynomial α) : Type u :=
def adjoin_root [comm_ring α] (f : polynomial α) : Type u :=
ideal.quotient (span {f} : ideal (polynomial α))

namespace adjoin_root

section comm_ring
variables [comm_ring α] [decidable_eq α] (f : polynomial α)
variables [comm_ring α] (f : polynomial α)

instance : comm_ring (adjoin_root f) := ideal.quotient.comm_ring _

Expand Down

0 comments on commit 7d792ec

Please sign in to comment.