Skip to content

Commit 91db1af

Browse files
committed
refactor: also Loop properties
1 parent ecd82b0 commit 91db1af

File tree

1 file changed

+4
-16
lines changed

1 file changed

+4
-16
lines changed

src/Algebra/Properties/Loop.agda

Lines changed: 4 additions & 16 deletions
Original file line numberDiff line numberDiff line change
@@ -17,28 +17,16 @@ open import Data.Product.Base using (proj₂)
1717
open import Relation.Binary.Reasoning.Setoid setoid
1818

1919
x//x≈ε : x x // x ≈ ε
20-
x//x≈ε x = begin
21-
x // x ≈⟨ //-congʳ (identityˡ x) ⟨
22-
(ε ∙ x) // x ≈⟨ rightDividesʳ x ε ⟩
23-
ε ∎
20+
x//x≈ε x = sym (x≈z//y _ _ _ (identityˡ x))
2421

2522
x\\x≈ε : x x \\ x ≈ ε
26-
x\\x≈ε x = begin
27-
x \\ x ≈⟨ \\-congˡ (identityʳ x ) ⟨
28-
x \\ (x ∙ ε) ≈⟨ leftDividesʳ x ε ⟩
29-
ε ∎
23+
x\\x≈ε x = sym (y≈x\\z _ _ _ (identityʳ x))
3024

3125
ε\\x≈x : x ε \\ x ≈ x
32-
ε\\x≈x x = begin
33-
ε \\ x ≈⟨ identityˡ (ε \\ x) ⟨
34-
ε ∙ (ε \\ x) ≈⟨ leftDividesˡ ε x ⟩
35-
x ∎
26+
ε\\x≈x x = sym (y≈x\\z _ _ _ (identityˡ x))
3627

3728
x//ε≈x : x x // ε ≈ x
38-
x//ε≈x x = begin
39-
x // ε ≈⟨ identityʳ (x // ε) ⟨
40-
(x // ε) ∙ ε ≈⟨ rightDividesˡ ε x ⟩
41-
x ∎
29+
x//ε≈x x = sym (x≈z//y _ _ _ (identityʳ x))
4230

4331
identityˡ-unique : x y x ∙ y ≈ y x ≈ ε
4432
identityˡ-unique x y eq = begin

0 commit comments

Comments
 (0)