[ minor ] Make NotBothZero parameter of standard gcd to be erased

This commit is contained in:
Denis Buzdalov 2022-10-28 21:14:47 +03:00 committed by G. Allais
parent 8d7b993cca
commit ff6afb0c59

View File

@ -390,7 +390,7 @@ Integral Nat where
export
covering
gcd : (a: Nat) -> (b: Nat) -> {auto ok: NotBothZero a b} -> Nat
gcd : (a: Nat) -> (b: Nat) -> {auto 0 ok: NotBothZero a b} -> Nat
gcd a Z = a
gcd Z b = b
gcd a (S b) = gcd (S b) (modNatNZ a (S b) SIsNonZero)