Skip to content

Commit f891093

Browse files
committed
refactor: another attempt to resolve merge of agda#2576
1 parent 31b51a6 commit f891093

File tree

3 files changed

+13
-25
lines changed

3 files changed

+13
-25
lines changed

Diff for: CHANGELOG.md

+6
Original file line numberDiff line numberDiff line change
@@ -42,6 +42,12 @@ Deprecated modules
4242
Deprecated names
4343
----------------
4444

45+
* In `Algebra.Apartness.Properties.HeytingCommutativeRing`:
46+
```agda
47+
x-0≈x ↦ Algebra.Properties.Ring.x-0#≈x
48+
#-sym ↦ Algebra.Apartness.Structures.IsHeytingCommutativeRing.#-sym
49+
```
50+
4551
* In `Algebra.Definitions.RawMagma`:
4652
```agda
4753
_∣∣_ ↦ _∥_

Diff for: src/Algebra/Apartness/Properties/HeytingCommutativeRing.agda

+7-1
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ module Algebra.Apartness.Properties.HeytingCommutativeRing
1313

1414
open import Algebra.Bundles using (CommutativeRing)
1515

16-
open HeytingCommutativeRing HCR
16+
open HeytingCommutativeRing HCR using (commutativeRing)
1717
open CommutativeRing commutativeRing using (ring)
1818
open import Algebra.Properties.Ring ring using (x-0#≈x)
1919

@@ -31,3 +31,9 @@ x-0≈x = x-0#≈x
3131
"Warning: x-0≈x was deprecated in v2.3.
3232
Please use Algebra.Properties.Ring.x-0#≈x instead."
3333
#-}
34+
35+
open HeytingCommutativeRing HCR public using (#-sym)
36+
{-# WARNING_ON_USAGE #-sym
37+
"Warning: #-sym was deprecated in v2.3.
38+
Please use Algebra.Apartness.Structures.IsHeytingCommutativeRing.#-sym instead."
39+
#-}

Diff for: src/Algebra/Apartness/Properties/HeytingField.agda

-24
Original file line numberDiff line numberDiff line change
@@ -66,30 +66,6 @@ x#0y#0→xy#0 {x} {y} x#0 y#0 = helper (#⇒invertible x#0) (#⇒invertible y#0)
6666
y⁻¹ * (y - 0#) ≈⟨ y⁻¹*y≈1 ⟩
6767
1# ∎
6868

69-
#-sym : Symmetric _#_
70-
#-sym {x} {y} x#y = invertibleˡ⇒# (- x-y⁻¹ , x-y⁻¹*y-x≈1)
71-
where
72-
open ≈-Reasoning setoid
73-
InvX-Y : Invertible 1# _*_ (x - y)
74-
InvX-Y = #⇒invertible x#y
75-
76-
x-y⁻¹ = InvX-Y .proj₁
77-
78-
y-x≈-[x-y] : y - x ≈ - (x - y)
79-
y-x≈-[x-y] = begin
80-
y - x ≈⟨ +-congʳ (-‿involutive y) ⟨
81-
- - y - x ≈⟨ -‿anti-homo-+ x (- y) ⟨
82-
- (x - y) ∎
83-
84-
x-y⁻¹*y-x≈1 : (- x-y⁻¹) * (y - x) ≈ 1#
85-
x-y⁻¹*y-x≈1 = begin
86-
(- x-y⁻¹) * (y - x) ≈⟨ -‿distribˡ-* x-y⁻¹ (y - x) ⟨
87-
- (x-y⁻¹ * (y - x)) ≈⟨ -‿cong (*-congˡ y-x≈-[x-y]) ⟩
88-
- (x-y⁻¹ * - (x - y)) ≈⟨ -‿cong (-‿distribʳ-* x-y⁻¹ (x - y)) ⟨
89-
- - (x-y⁻¹ * (x - y)) ≈⟨ -‿involutive (x-y⁻¹ * (x - y)) ⟩
90-
x-y⁻¹ * (x - y) ≈⟨ InvX-Y .proj₂ .proj₁ ⟩
91-
1# ∎
92-
9369
#-congʳ : x ≈ y x # z y # z
9470
#-congʳ {x} {y} {z} x≈y = helper ∘ #⇒invertible
9571
where

0 commit comments

Comments
 (0)