Skip to content

Commit

Permalink
tweaks to accomodate agda#2292
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna committed Feb 13, 2024
1 parent 623d854 commit 4076cc5
Showing 1 changed file with 6 additions and 4 deletions.
10 changes: 6 additions & 4 deletions src/Data/Nat/Bounded/Base.agda
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,7 @@ open import Relation.Nullary.Negation.Core using (¬_)

private
variable
m n :
m n o :

------------------------------------------------------------------------
-- Definition
Expand Down Expand Up @@ -87,8 +87,10 @@ record _∼_ {n} (lhs rhs : ℕ) : Set where
lhs/∼≡ : lhs /∼≡ k
rhs/∼≡ : rhs /∼≡ k

≡-Mod : Rel ℕ _
≡-Mod n i j = _∼_ {n} i j
≡-Modℕ : Rel ℕ _
≡-Modℕ n = _∼_ {n}

syntax ≡-Mod n i j = ij mod n
syntax ≡-Modℕ n m o = mo modℕ n

nonZeroModulus : (m ≡ o modℕ n) NonZero n
nonZeroModulus eq = nonZeroIndex k where open _∼_ eq

0 comments on commit 4076cc5

Please sign in to comment.