Skip to content

Commit

Permalink
feat(algebra/free_algebra): Add a nontrivial instance (#5033)
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Nov 18, 2020
1 parent 0e09ada commit 38d2b53
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/algebra/free_algebra.lean
Expand Up @@ -6,6 +6,7 @@ Author: Scott Morrison, Adam Topaz.
import algebra.algebra.subalgebra
import algebra.monoid_algebra
import linear_algebra
import data.equiv.transfer_instance

/-!
# Free Algebras
Expand Down Expand Up @@ -314,6 +315,9 @@ begin
end
(by { ext, simp, })

instance [nontrivial R] : nontrivial (free_algebra R X) :=
equiv_monoid_algebra_free_monoid.to_equiv.nontrivial

end free_algebra

-- There is something weird in the above namespace that breaks the typeclass resolution of `has_coe_to_sort` below.
Expand Down

0 comments on commit 38d2b53

Please sign in to comment.