Skip to content

Commit

Permalink
refactor(data/ordmap/ordset): simpler proof of not_le_delta (#6119)
Browse files Browse the repository at this point in the history
Co-authors: `lean-gptf`, Stanislas Polu

This was found by `formal-lean-wm-to-tt-m1-m2-v4-c4` when we evaluated it on theorems added to `mathlib` after we last extracted training data.
  • Loading branch information
Jesse Michael Han committed Feb 9, 2021
1 parent 7e5ff2f commit ec8f2ac
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/data/ordmap/ordset.lean
Expand Up @@ -70,7 +70,7 @@ namespace ordnode
/-! ### delta and ratio -/

theorem not_le_delta {s} (H : 1 ≤ s) : ¬ s ≤ delta * 0 :=
λ h, by rw mul_zero at h; exact not_lt_of_le h H
not_le_of_gt H

theorem delta_lt_false {a b : ℕ}
(h₁ : delta * a < b) (h₂ : delta * b < a) : false :=
Expand Down

0 comments on commit ec8f2ac

Please sign in to comment.