Skip to content

Commit cc6a8e7

Browse files
committed
fixes agda#2408
1 parent 606bea8 commit cc6a8e7

File tree

1 file changed

+38
-0
lines changed

1 file changed

+38
-0
lines changed
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,38 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- Some derivable properties
5+
------------------------------------------------------------------------
6+
7+
{-# OPTIONS --cubical-compatible --safe #-}
8+
9+
open import Algebra.Bundles using (IdempotentCommutativeMonoid)
10+
11+
module Algebra.Properties.IdempotentCommutativeMonoid
12+
{c ℓ} (M : IdempotentCommutativeMonoid c ℓ) where
13+
14+
open IdempotentCommutativeMonoid M
15+
16+
open import Algebra.Consequences.Setoid setoid
17+
using (comm∧distrˡ⇒distrʳ; comm∧distrˡ⇒distr)
18+
open import Algebra.Definitions _≈_
19+
using (_DistributesOverˡ_; _DistributesOverʳ_; _DistributesOver_)
20+
open import Algebra.Properties.CommutativeSemigroup commutativeSemigroup
21+
using (interchange)
22+
open import Relation.Binary.Reasoning.Setoid setoid
23+
24+
25+
------------------------------------------------------------------------
26+
-- Distributivity
27+
28+
distrˡ : _∙_ DistributesOverˡ _∙_
29+
distrˡ a b c = begin
30+
a ∙ (b ∙ c) ≈⟨ ∙-congʳ (idem a) ⟨
31+
(a ∙ a) ∙ (b ∙ c) ≈⟨ interchange _ _ _ _ ⟩
32+
(a ∙ b) ∙ (a ∙ c) ∎
33+
34+
distrʳ : _∙_ DistributesOverʳ _∙_
35+
distrʳ = comm∧distrˡ⇒distrʳ ∙-cong comm distrˡ
36+
37+
distr : _∙_ DistributesOver _∙_
38+
distr = comm∧distrˡ⇒distr ∙-cong comm distrˡ

0 commit comments

Comments
 (0)