Skip to content

Commit

Permalink
fix: long lines
Browse files Browse the repository at this point in the history
  • Loading branch information
fgdorais committed Jun 21, 2024
1 parent 738f4b7 commit ce7bd25
Showing 1 changed file with 10 additions and 5 deletions.
15 changes: 10 additions & 5 deletions Batteries/Data/UInt.lean
Original file line number Diff line number Diff line change
Expand Up @@ -65,7 +65,8 @@ theorem UInt8.le_iff_toNat_le_toNat {x y : UInt8} : x ≤ y ↔ x.toNat ≤ y.to

theorem UInt8.lt_iff_toNat_lt_toNat {x y : UInt8} : x < y ↔ x.toNat < y.toNat := .rfl

theorem UInt8.compare_eq_toNat_compare_toNat (x y : UInt8) : compare x y = compare x.toNat y.toNat := by
theorem UInt8.compare_eq_toNat_compare_toNat (x y : UInt8) :
compare x y = compare x.toNat y.toNat := by
simp only [compare, compareOfLessAndEq, lt_iff_toNat_lt_toNat, ext_iff]

theorem UInt8.max_def (x y : UInt8) : max x y = if x ≤ y then y else x := rfl
Expand Down Expand Up @@ -152,7 +153,8 @@ theorem UInt16.le_iff_toNat_le_toNat {x y : UInt16} : x ≤ y ↔ x.toNat ≤ y.

theorem UInt16.lt_iff_toNat_lt_toNat {x y : UInt16} : x < y ↔ x.toNat < y.toNat := .rfl

theorem UInt16.compare_eq_toNat_compare_toNat (x y : UInt16) : compare x y = compare x.toNat y.toNat := by
theorem UInt16.compare_eq_toNat_compare_toNat (x y : UInt16) :
compare x y = compare x.toNat y.toNat := by
simp only [compare, compareOfLessAndEq, lt_iff_toNat_lt_toNat, ext_iff]

theorem UInt16.max_def (x y : UInt16) : max x y = if x ≤ y then y else x := rfl
Expand Down Expand Up @@ -239,7 +241,8 @@ theorem UInt32.le_iff_toNat_le_toNat {x y : UInt32} : x ≤ y ↔ x.toNat ≤ y.

theorem UInt32.lt_iff_toNat_lt_toNat {x y : UInt32} : x < y ↔ x.toNat < y.toNat := .rfl

theorem UInt32.compare_eq_toNat_compare_toNat (x y : UInt32) : compare x y = compare x.toNat y.toNat := by
theorem UInt32.compare_eq_toNat_compare_toNat (x y : UInt32) :
compare x y = compare x.toNat y.toNat := by
simp only [compare, compareOfLessAndEq, lt_iff_toNat_lt_toNat, ext_iff]

theorem UInt32.max_def (x y : UInt32) : max x y = if x ≤ y then y else x := rfl
Expand Down Expand Up @@ -327,7 +330,8 @@ theorem UInt64.le_iff_toNat_le_toNat {x y : UInt64} : x ≤ y ↔ x.toNat ≤ y.

theorem UInt64.lt_iff_toNat_lt_toNat {x y : UInt64} : x < y ↔ x.toNat < y.toNat := .rfl

theorem UInt64.compare_eq_toNat_compare_toNat (x y : UInt64) : compare x y = compare x.toNat y.toNat := by
theorem UInt64.compare_eq_toNat_compare_toNat (x y : UInt64) :
compare x y = compare x.toNat y.toNat := by
simp only [compare, compareOfLessAndEq, lt_iff_toNat_lt_toNat, ext_iff]

theorem UInt64.max_def (x y : UInt64) : max x y = if x ≤ y then y else x := rfl
Expand Down Expand Up @@ -427,7 +431,8 @@ theorem USize.le_iff_toNat_le_toNat {x y : USize} : x ≤ y ↔ x.toNat ≤ y.to

theorem USize.lt_iff_toNat_lt_toNat {x y : USize} : x < y ↔ x.toNat < y.toNat := .rfl

theorem USize.compare_eq_toNat_compare_toNat (x y : USize) : compare x y = compare x.toNat y.toNat := by
theorem USize.compare_eq_toNat_compare_toNat (x y : USize) :
compare x y = compare x.toNat y.toNat := by
simp only [compare, compareOfLessAndEq, lt_iff_toNat_lt_toNat, ext_iff]

theorem USize.max_def (x y : USize) : max x y = if x ≤ y then y else x := rfl
Expand Down

0 comments on commit ce7bd25

Please sign in to comment.