File tree Expand file tree Collapse file tree 3 files changed +15
-11
lines changed
Expand file tree Collapse file tree 3 files changed +15
-11
lines changed Original file line number Diff line number Diff line change @@ -11,6 +11,10 @@ Bug-fixes
1111
1212* Fix a type error in ` README.Data.Fin.Relation.Unary.Top ` within the definition of ` >-weakInduction ` .
1313
14+ * Remove spurious definition of ` Algebra.Consequences.Propositional.sel⇒idem ` ,
15+ which duplicated lemma from ` Algebra.Consequences.Base ` , instead of importing
16+ from ` Algebra.Consequences.Setoid ` .
17+
1418* Fix a typo in ` Algebra.Morphism.Construct.DirectProduct ` .
1519
1620* Fix a typo in ` Function.Construct.Constant ` .
@@ -122,6 +126,7 @@ Additions to existing modules
122126
123127* In ` Algebra.Consequences.Setoid ` :
124128 ``` agda
129+ sel⇒idem : Selective _∙_ → Idempotent _∙_
125130 binomial-expansion : Congruent₂ _∙_ → Associative _∙_ → _◦_ DistributesOver _∙_ →
126131 ∀ w x y z → ((w ∙ x) ◦ (y ∙ z)) ≈ ((((w ◦ y) ∙ (w ◦ z)) ∙ (x ◦ y)) ∙ (x ◦ z))
127132 ```
Original file line number Diff line number Diff line change @@ -41,7 +41,6 @@ open Base public
4141 ; comm⇒sym[distribˡ]
4242 ; subst∧comm⇒sym
4343 ; wlog
44- ; sel⇒idem
4544 ; binomial-expansion
4645-- plus all the deprecated versions of the above
4746 ; comm+assoc⇒middleFour
@@ -55,7 +54,7 @@ open Base public
5554 ; comm+distrʳ⇒distrˡ
5655 ; subst+comm⇒sym
5756 )
58-
57+ test = {!sel⇒idem!}
5958------------------------------------------------------------------------
6059-- Group-like structures
6160
@@ -111,14 +110,6 @@ module _ {_∙_ _◦_ : Op₂ A}
111110 ((w ∙ x) ◦ (y ∙ z)) ≡ ((((w ◦ y) ∙ (w ◦ z)) ∙ (x ◦ y)) ∙ (x ◦ z))
112111 binomial-expansion = Base.binomial-expansion {_∙_} {_◦_} (cong₂ _) ∙-assoc distrib
113112
114- ------------------------------------------------------------------------
115- -- Selectivity
116-
117- module _ {_∙_ : Op₂ A} where
118-
119- sel⇒idem : Selective _∙_ → Idempotent _∙_
120- sel⇒idem = Base.sel⇒idem _≡_
121-
122113------------------------------------------------------------------------
123114-- Middle-Four Exchange
124115
Original file line number Diff line number Diff line change @@ -33,14 +33,22 @@ open import Relation.Binary.Reasoning.Setoid S
3333-- Export base lemmas that don't require the setoid
3434
3535open Base public
36- hiding (module Congruence )
36+ hiding (module Congruence ; sel⇒idem )
3737
3838-- Export congruence lemmas using reflexivity
3939
4040module Congruence {_∙_ : Op₂ A} (cong : Congruent₂ _∙_) where
4141
4242 open Base.Congruence _≈_ cong refl public
4343
44+ ------------------------------------------------------------------------
45+ -- Selectivity
46+
47+ module _ {_∙_ : Op₂ A} where
48+
49+ sel⇒idem : Selective _∙_ → Idempotent _∙_
50+ sel⇒idem = Base.sel⇒idem _≈_
51+
4452------------------------------------------------------------------------
4553-- MiddleFourExchange
4654
You can’t perform that action at this time.
0 commit comments