You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
Copy file name to clipboardExpand all lines: src/Data/Nat/Base.agda
+5-5
Original file line number
Diff line number
Diff line change
@@ -18,7 +18,7 @@ open import Data.Parity.Base using (Parity; 0ℙ; 1ℙ)
18
18
open importLevelusing (0ℓ)
19
19
open importRelation.Binary.Coreusing (Rel)
20
20
open importRelation.Binary.PropositionalEquality.Core
21
-
using (_≡_; _≢_; refl)
21
+
using (_≡_; _≢_; refl; cong)
22
22
open importRelation.Nullary.Negation.Coreusing (¬_; contradiction)
23
23
open importRelation.Unaryusing (Pred)
24
24
@@ -375,7 +375,7 @@ m >″ n = n <″ m
375
375
-- Smart destructor of _<″_
376
376
377
377
s<″s⁻¹ :∀ {m n} → suc m <″ suc n → m <″ n
378
-
s<″s⁻¹ (k , refl) = k , refl
378
+
s<″s⁻¹ (k , eq) = k , cong pred eq
379
379
380
380
-- _≤‴_: this definition is useful for induction with an upper bound.
381
381
@@ -435,10 +435,10 @@ pattern <″-offset k = k , refl
435
435
"Warning: <″-offset was deprecated in v2.1. Please match directly on proofs of ≤″ using pattern (_, refl) from Algebra.Definitions.RawMagma._∣ˡ_ instead. "
436
436
#-}
437
437
438
-
-- Smart destructors of _<″_
438
+
-- Smart destructor of _≤″_
439
439
440
440
s≤″s⁻¹ :∀ {m n} → suc m ≤″ suc n → m ≤″ n
441
-
s≤″s⁻¹ (k , refl) = k , refl
441
+
s≤″s⁻¹ (k , eq) = k , cong pred eq
442
442
{-# WARNING_ON_USAGE s≤″s⁻¹
443
-
"Warning: s≤″s⁻¹ was deprecated in v2.1. Please match directly on proofs of ≤″ using pattern (_, refl) from Algebra.Definitions.RawMagma._∣ˡ_ instead. "
443
+
"Warning: s≤″s⁻¹ was deprecated in v2.1. Please match directly on proofs of ≤″ using constructor Algebra.Definitions.RawMagma._∣ˡ_._,_ instead. "
0 commit comments