Skip to content
Merged
Changes from 1 commit
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
2 changes: 1 addition & 1 deletion src/Algebra/Morphism/Construct/DirectProduct.agda
Original file line number Diff line number Diff line change
Expand Up @@ -133,7 +133,7 @@ module Monoid-Export {M : RawMonoid a ℓ₁} {N : RawMonoid b ℓ₂} where
module N = RawMonoid N

module _ {refl : Reflexive M._≈_} where
proj₁ = Proj₁.isMonoidHomomorphism M M refl
proj₁ = Proj₁.isMonoidHomomorphism M N refl

module _ {refl : Reflexive N._≈_} where
proj₂ = Proj₂.isMonoidHomomorphism M N refl
Expand Down