Skip to content

Commit

Permalink
simplify things
Browse files Browse the repository at this point in the history
  • Loading branch information
tobiasgrosser committed Oct 19, 2024
1 parent a3c333d commit 08a460b
Showing 1 changed file with 1 addition and 4 deletions.
5 changes: 1 addition & 4 deletions src/Init/Omega/Int.lean
Original file line number Diff line number Diff line change
Expand Up @@ -94,12 +94,9 @@ theorem ofNat_sub_dichotomy {a b : Nat} :
b ≤ a ∧ ((a - b : Nat) : Int) = a - b ∨ a < b ∧ ((a - b : Nat) : Int) = 0 := by
by_cases h : b ≤ a
· left
have := Int.ofNat_sub h
simp [h]
· right
have t := Nat.not_le.mp h
simp [Int.ofNat_sub_eq_zero h]
exact t
simp [Int.ofNat_sub_eq_zero, Nat.not_le.mp, h]

theorem ofNat_congr {a b : Nat} (h : a = b) : (a : Int) = (b : Int) := congrArg _ h

Expand Down

0 comments on commit 08a460b

Please sign in to comment.