File tree 3 files changed +0
-41
lines changed
3 files changed +0
-41
lines changed Original file line number Diff line number Diff line change @@ -199,7 +199,6 @@ New modules
199
199
Algebra.Properties.Semiring.Divisibility
200
200
Algebra.Properties.Semiring.Exp
201
201
Algebra.Properties.Semiring.Exp.TCOptimised
202
- Algebra.Properties.Semiring.GCD
203
202
Algebra.Properties.Semiring.Mult
204
203
Algebra.Properties.Semiring.Mult.TCOptimised
205
204
Original file line number Diff line number Diff line change @@ -72,13 +72,3 @@ record Prime (p : A) : Set (a ⊔ ℓ) where
72
72
p≉0 : p ≉ 0#
73
73
split-∣ : ∀ {x y} → p ∣ x * y → p ∣ x ⊎ p ∣ y
74
74
75
- ------------------------------------------------------------------------
76
- -- Greatest common divisor
77
-
78
- record IsGCD (x y gcd : A) : Set (a ⊔ ℓ) where
79
- constructor gcdᶜ
80
- field
81
- divides₁ : gcd ∣ x
82
- divides₂ : gcd ∣ y
83
- greatest : ∀ {z} → z ∣ x → z ∣ y → z ∣ gcd
84
-
Load Diff This file was deleted.
You can’t perform that action at this time.
0 commit comments