@@ -11,7 +11,7 @@ module Data.Char.Properties where
1111open import Data.Bool.Base using (Bool)
1212open import Data.Char.Base
1313import Data.Nat.Base as ℕ
14- import Data.Nat.Properties as ℕₚ
14+ import Data.Nat.Properties as ℕ
1515open import Data.Product.Base using (_,_)
1616
1717open import Function.Base
@@ -56,7 +56,7 @@ open import Agda.Builtin.Char.Properties
5656
5757infix 4 _≟_
5858_≟_ : Decidable {A = Char} _≡_
59- x ≟ y = map′ ≈⇒≡ ≈-reflexive (toℕ x ℕₚ .≟ toℕ y)
59+ x ≟ y = map′ ≈⇒≡ ≈-reflexive (toℕ x ℕ .≟ toℕ y)
6060
6161setoid : Setoid _ _
6262setoid = PropEq.setoid Char
@@ -95,22 +95,22 @@ private
9595
9696infix 4 _<?_
9797_<?_ : Decidable _<_
98- _<?_ = On.decidable toℕ ℕ._<_ ℕₚ ._<?_
98+ _<?_ = On.decidable toℕ ℕ._<_ ℕ ._<?_
9999
100100<-cmp : Trichotomous _≡_ _<_
101- <-cmp c d with ℕₚ .<-cmp (toℕ c) (toℕ d)
101+ <-cmp c d with ℕ .<-cmp (toℕ c) (toℕ d)
102102... | tri< lt ¬eq ¬gt = tri< lt (≉⇒≢ ¬eq) ¬gt
103103... | tri≈ ¬lt eq ¬gt = tri≈ ¬lt (≈⇒≡ eq) ¬gt
104104... | tri> ¬lt ¬eq gt = tri> ¬lt (≉⇒≢ ¬eq) gt
105105
106106<-irrefl : Irreflexive _≡_ _<_
107- <-irrefl = ℕₚ .<-irrefl ∘′ cong toℕ
107+ <-irrefl = ℕ .<-irrefl ∘′ cong toℕ
108108
109109<-trans : Transitive _<_
110- <-trans {c} {d} {e} = On.transitive toℕ ℕ._<_ ℕₚ .<-trans {c} {d} {e}
110+ <-trans {c} {d} {e} = On.transitive toℕ ℕ._<_ ℕ .<-trans {c} {d} {e}
111111
112112<-asym : Asymmetric _<_
113- <-asym {c} {d} = On.asymmetric toℕ ℕ._<_ ℕₚ .<-asym {c} {d}
113+ <-asym {c} {d} = On.asymmetric toℕ ℕ._<_ ℕ .<-asym {c} {d}
114114
115115<-isStrictPartialOrder : IsStrictPartialOrder _≡_ _<_
116116<-isStrictPartialOrder = record
@@ -151,7 +151,7 @@ _≤?_ = Reflₚ.decidable <-cmp
151151≤-trans = Reflₚ.trans (λ {a} {b} {c} → <-trans {a} {b} {c})
152152
153153≤-antisym : Antisymmetric _≡_ _≤_
154- ≤-antisym = Reflₚ.antisym _≡_ refl ℕₚ .<-asym
154+ ≤-antisym = Reflₚ.antisym _≡_ refl ℕ .<-asym
155155
156156≤-isPreorder : IsPreorder _≡_ _≤_
157157≤-isPreorder = record
@@ -220,7 +220,7 @@ Please use Propositional Equality's subst instead."
220220
221221infix 4 _≈?_
222222_≈?_ : Decidable _≈_
223- x ≈? y = toℕ x ℕₚ .≟ toℕ y
223+ x ≈? y = toℕ x ℕ .≟ toℕ y
224224
225225≈-isEquivalence : IsEquivalence _≈_
226226≈-isEquivalence = record
@@ -277,28 +277,28 @@ Please use decSetoid instead."
277277#-}
278278
279279<-isStrictPartialOrder-≈ : IsStrictPartialOrder _≈_ _<_
280- <-isStrictPartialOrder-≈ = On.isStrictPartialOrder toℕ ℕₚ .<-isStrictPartialOrder
280+ <-isStrictPartialOrder-≈ = On.isStrictPartialOrder toℕ ℕ .<-isStrictPartialOrder
281281{-# WARNING_ON_USAGE <-isStrictPartialOrder-≈
282282"Warning: <-isStrictPartialOrder-≈ was deprecated in v1.5.
283283Please use <-isStrictPartialOrder instead."
284284#-}
285285
286286<-isStrictTotalOrder-≈ : IsStrictTotalOrder _≈_ _<_
287- <-isStrictTotalOrder-≈ = On.isStrictTotalOrder toℕ ℕₚ .<-isStrictTotalOrder
287+ <-isStrictTotalOrder-≈ = On.isStrictTotalOrder toℕ ℕ .<-isStrictTotalOrder
288288{-# WARNING_ON_USAGE <-isStrictTotalOrder-≈
289289"Warning: <-isStrictTotalOrder-≈ was deprecated in v1.5.
290290Please use <-isStrictTotalOrder instead."
291291#-}
292292
293293<-strictPartialOrder-≈ : StrictPartialOrder _ _ _
294- <-strictPartialOrder-≈ = On.strictPartialOrder ℕₚ .<-strictPartialOrder toℕ
294+ <-strictPartialOrder-≈ = On.strictPartialOrder ℕ .<-strictPartialOrder toℕ
295295{-# WARNING_ON_USAGE <-strictPartialOrder-≈
296296"Warning: <-strictPartialOrder-≈ was deprecated in v1.5.
297297Please use <-strictPartialOrder instead."
298298#-}
299299
300300<-strictTotalOrder-≈ : StrictTotalOrder _ _ _
301- <-strictTotalOrder-≈ = On.strictTotalOrder ℕₚ .<-strictTotalOrder toℕ
301+ <-strictTotalOrder-≈ = On.strictTotalOrder ℕ .<-strictTotalOrder toℕ
302302{-# WARNING_ON_USAGE <-strictTotalOrder-≈
303303"Warning: <-strictTotalOrder-≈ was deprecated in v1.5.
304304Please use <-strictTotalOrder instead."
0 commit comments