File tree Expand file tree Collapse file tree 2 files changed +12
-0
lines changed
Expand file tree Collapse file tree 2 files changed +12
-0
lines changed Original file line number Diff line number Diff line change @@ -151,6 +151,12 @@ Additions to existing modules
151151 ⊕-∧-booleanRing : BooleanRing _ _
152152 ```
153153
154+ * In ` Algebra.Morphism.Structures.IsMagmaHomomorphism ` :
155+ ``` agda
156+ ⟦_⟧∙_ : A → B → B
157+ _∙⟦_⟧ : B → A → B
158+ ```
159+
154160* In ` Algebra.Properties.RingWithoutOne ` :
155161 ``` agda
156162 [-x][-y]≈xy : ∀ x y → - x * - y ≈ x * y
Original file line number Diff line number Diff line change @@ -89,6 +89,12 @@ module MagmaMorphisms (M₁ : RawMagma a ℓ₁) (M₂ : RawMagma b ℓ₂) wher
8989 open IsRelHomomorphism isRelHomomorphism public
9090 renaming (cong to ⟦⟧-cong)
9191
92+ ⟦_⟧∙_ : A → B → B
93+ ⟦ x ⟧∙ y = ⟦ x ⟧ ◦ y
94+
95+ _∙⟦_⟧ : B → A → B
96+ y ∙⟦ x ⟧ = y ◦ ⟦ x ⟧
97+
9298
9399 record IsMagmaMonomorphism (⟦_⟧ : A → B) : Set (a ⊔ ℓ₁ ⊔ ℓ₂) where
94100 field
You can’t perform that action at this time.
0 commit comments