Skip to content

Commit

Permalink
avoid some unused variables
Browse files Browse the repository at this point in the history
  • Loading branch information
tobiasgrosser committed Oct 19, 2024
1 parent 514d0da commit a3c333d
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
4 changes: 2 additions & 2 deletions src/Init/Data/Int/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -24,9 +24,9 @@ theorem subNatNat_of_sub_eq_succ {m n k : Nat} (h : n - m = succ k) : subNatNat
theorem subNatNat_of_sub {m n : Nat} (h : n ≤ m) : subNatNat m n = ↑(m - n) := by
rw [subNatNat, ofNat_eq_coe]
split
case h_1 x h' =>
case h_1 _ _ =>
simp
case h_2 x h' =>
case h_2 _ h' =>
rw [Nat.sub_eq_zero_of_le h] at h'
simp at h'

Expand Down
2 changes: 1 addition & 1 deletion src/Init/Omega/Int.lean
Original file line number Diff line number Diff line change
Expand Up @@ -94,7 +94,7 @@ 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 t := Int.ofNat_sub h
have := Int.ofNat_sub h
simp [h]
· right
have t := Nat.not_le.mp h
Expand Down

0 comments on commit a3c333d

Please sign in to comment.