We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent ba505b0 commit 1029995Copy full SHA for 1029995
src/Algebra/Properties/Semiring/Primality.agda
@@ -22,8 +22,7 @@ open import Algebra.Properties.Semiring.Divisibility R
22
23
private
24
variable
25
- x p : A
26
-
+ x : A
27
28
------------------------------------------------------------------------
29
-- Re-export primality definitions
@@ -43,6 +42,6 @@ Coprime-sym coprime = flip coprime
43
42
44
-- Properties of Irreducible
45
46
-Irreducible⇒≉0 : 0# ≉ 1# → Irreducible p → p ≉ 0#
+Irreducible⇒≉0 : 0# ≉ 1# → ∀ {p} → Irreducible p → p ≉ 0#
47
Irreducible⇒≉0 0≉1 (mkIrred _ chooseInvertible) p≈0 =
48
0∤1 0≉1 (reduce (chooseInvertible (trans p≈0 (sym (zeroˡ 0#)))))
0 commit comments