Skip to content

Commit 3786f55

Browse files
committed
fix: CHANGELOG plus tidying up
1 parent 55a7384 commit 3786f55

File tree

4 files changed

+30
-7
lines changed

4 files changed

+30
-7
lines changed

CHANGELOG.md

+23-1
Original file line numberDiff line numberDiff line change
@@ -20,6 +20,14 @@ Non-backwards compatible changes
2020
* The definitions of `Algebra.Structures.IsHeyting*` and
2121
`Algebra.Structures.IsHeyting*` have been refactored, together
2222
with that of `Relation.Binary.Definitions.Tight` on which they depend.
23+
Specifically:
24+
- `Tight _≈_ _#_` has been redefined to drop the redundant
25+
second conjunct, because it is equivalent to `Irreflexive _≈_ _#_`.
26+
- new definitions: `(Is)TightApartnessRelation` structure/bundle
27+
- the definition of `HeytingCommutativeRing` now drops the properties of
28+
invertibility, in favour of moving them to `HeytingField`.
29+
- both `Heyting*` algebraic structure/bundles have been redefined to base
30+
off an underlying `TightApartnessRelation`.
2331

2432
Minor improvements
2533
------------------
@@ -144,9 +152,23 @@ Additions to existing modules
144152
commutativeRing : CommutativeRing c ℓ → CommutativeRing (a ⊔ c) (a ⊔ ℓ)
145153
```
146154

155+
* In `Algebra.Properties.AbelianGroup`:
156+
```agda
157+
x-ε≈x : RightIdentity ε _-_
158+
```
159+
160+
* In `Algebra.Properties.RingWithoutOne`:
161+
```agda
162+
x-0#≈x : RightIdentity 0# _-_
163+
```
164+
147165
* In `Relation.Binary.Properties.DecSetoid`:
148166
```agda
149167
≉-isTightApartnessRelation : IsTightApartnessRelation _≈_ _#_
150168
≉-tightApartnessRelation : TightApartnessRelation _ _ _
151169
```
152-
170+
Additionally,
171+
```agda
172+
≉-tight : Tight _≈_ _≉_
173+
```
174+
has been redefined to reflect the change in the definition of `Tight`.

src/Algebra/Apartness/Properties/HeytingCommutativeRing.agda

+1
Original file line numberDiff line numberDiff line change
@@ -17,6 +17,7 @@ open HeytingCommutativeRing HCR
1717
open CommutativeRing commutativeRing using (ring)
1818
open import Algebra.Properties.Ring ring using (x-0#≈x)
1919

20+
2021
------------------------------------------------------------------------
2122
-- DEPRECATED NAMES
2223
------------------------------------------------------------------------

src/Algebra/Apartness/Properties/HeytingField.agda

+4-3
Original file line numberDiff line numberDiff line change
@@ -27,8 +27,9 @@ open import Algebra.Properties.Ring ring
2727
open import Relation.Binary.Definitions using (Symmetric)
2828
import Relation.Binary.Reasoning.Setoid as ≈-Reasoning
2929

30-
private variable
31-
x y z : Carrier
30+
private
31+
variable
32+
x y z : Carrier
3233

3334

3435
invertibleˡ⇒# : LeftInvertible 1# _*_ (x - y) x # y
@@ -85,7 +86,7 @@ x#0y#0→xy#0 {x} {y} x#0 y#0 = helper (#⇒invertible x#0) (#⇒invertible y#0)
8586
(- x-y⁻¹) * (y - x) ≈⟨ -‿distribˡ-* x-y⁻¹ (y - x) ⟨
8687
- (x-y⁻¹ * (y - x)) ≈⟨ -‿cong (*-congˡ y-x≈-[x-y]) ⟩
8788
- (x-y⁻¹ * - (x - y)) ≈⟨ -‿cong (-‿distribʳ-* x-y⁻¹ (x - y)) ⟨
88-
- - (x-y⁻¹ * (x - y)) ≈⟨ -‿involutive (x-y⁻¹ * ((x - y))) ⟩
89+
- - (x-y⁻¹ * (x - y)) ≈⟨ -‿involutive (x-y⁻¹ * (x - y)) ⟩
8990
x-y⁻¹ * (x - y) ≈⟨ InvX-Y .proj₂ .proj₁ ⟩
9091
1# ∎
9192

src/Relation/Binary/Properties/DecSetoid.agda

+2-3
Original file line numberDiff line numberDiff line change
@@ -11,18 +11,17 @@ open import Relation.Binary.Bundles
1111

1212
module Relation.Binary.Properties.DecSetoid {c ℓ} (S : DecSetoid c ℓ) where
1313

14-
open import Data.Product using (_,_)
1514
open import Data.Sum using (inj₁; inj₂)
1615
open import Relation.Binary.Definitions
1716
using (Cotransitive; Tight)
1817
import Relation.Binary.Properties.Setoid as SetoidProperties
1918
open import Relation.Binary.Structures
20-
using (IsApartnessRelation; IsTightApartnessRelation; IsDecEquivalence)
19+
using (IsApartnessRelation; IsTightApartnessRelation)
2120
open import Relation.Nullary.Decidable.Core
2221
using (yes; no; decidable-stable)
2322

2423
open DecSetoid S using (_≈_; _≉_; _≟_; setoid; trans)
25-
open SetoidProperties setoid
24+
open SetoidProperties setoid using (≉-sym; ≉-irrefl)
2625

2726
≉-cotrans : Cotransitive _≉_
2827
≉-cotrans {x} {y} x≉y z with x ≟ z | z ≟ y

0 commit comments

Comments
 (0)