We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
Algebra.Properties.Magma.Divisibility
1 parent 10e115d commit e435db2Copy full SHA for e435db2
src/Algebra/Properties/CommutativeMagma/Divisibility.agda
@@ -28,7 +28,7 @@ x∣xy : ∀ x y → x ∣ x ∙ y
28
x∣xy x y = y , comm y x
29
30
xy≈z⇒x∣z : ∀ x y {z} → x ∙ y ≈ z → x ∣ z
31
-xy≈z⇒x∣z x y xy≈z = ∣-respʳ xy≈z (x∣xy x y)
+xy≈z⇒x∣z x y xy≈z = ∣-respʳ-≈ xy≈z (x∣xy x y)
32
33
x|xy∧y|xy : ∀ x y → (x ∣ x ∙ y) × (y ∣ x ∙ y)
34
x|xy∧y|xy x y = x∣xy x y , x∣yx y x
src/Algebra/Properties/Magma/Divisibility.agda
@@ -39,7 +39,7 @@ x∣yx : ∀ x y → x ∣ y ∙ x
39
x∣yx x y = y , refl
40
41
xy≈z⇒y∣z : ∀ x y {z} → x ∙ y ≈ z → y ∣ z
42
-xy≈z⇒y∣z x y xy≈z = ∣-respʳ-≈ xy≈z (x∣yx y x)
+xy≈z⇒y∣z x y xy≈z = x , xy≈z
43
44
------------------------------------------------------------------------
45
-- Properties of non-divisibility
0 commit comments