mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-10 22:28:40 +00:00
14 lines
429 B
Agda
14 lines
429 B
Agda
{-# OPTIONS --safe --warning=error --without-K #-}
|
|
|
|
open import LogicalFormulae
|
|
open import Functions
|
|
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
|
|
|
|
module Monoids.Definition where
|
|
|
|
record Monoid {a : _} {A : Set a} (Zero : A) (_+_ : A → A → A) : Set a where
|
|
field
|
|
associative : (a b c : A) → a + (b + c) ≡ (a + b) + c
|
|
idLeft : (a : A) → Zero + a ≡ a
|
|
idRight : (a : A) → a + Zero ≡ a
|