File tree Expand file tree Collapse file tree 1 file changed +4
-16
lines changed Expand file tree Collapse file tree 1 file changed +4
-16
lines changed Original file line number Diff line number Diff line change @@ -17,28 +17,16 @@ open import Data.Product.Base using (proj₂)
17
17
open import Relation.Binary.Reasoning.Setoid setoid
18
18
19
19
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))
24
21
25
22
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))
30
24
31
25
ε\\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))
36
27
37
28
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))
42
30
43
31
identityˡ-unique : ∀ x y → x ∙ y ≈ y → x ≈ ε
44
32
identityˡ-unique x y eq = begin
You can’t perform that action at this time.
0 commit comments