Skip to content

Commit

Permalink
chore(data/equiv/ring): make ring_aut reducible (leanprover-community…
Browse files Browse the repository at this point in the history
…#2563)

This makes the coercion to fun work. This is the same approach as we used for `perm` and it worked okay for `perm`.

Related Zulip thread: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/ring_aut.20coerce.20to.20function
  • Loading branch information
ChrisHughes24 authored and cipher1024 committed Mar 15, 2022
1 parent 6f38dd8 commit a9aa583
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/data/equiv/ring.lean
Original file line number Diff line number Diff line change
Expand Up @@ -221,7 +221,7 @@ protected def integral_domain {A : Type*} (B : Type*) [ring A] [integral_domain
end ring_equiv

/-- The group of ring automorphisms. -/
def ring_aut (R : Type*) [has_mul R] [has_add R] := ring_equiv R R
@[reducible] def ring_aut (R : Type*) [has_mul R] [has_add R] := ring_equiv R R

namespace ring_aut

Expand Down

0 comments on commit a9aa583

Please sign in to comment.