Zulip Chat Archive
Stream: metaprogramming / tactics
Topic: push_neg user command
Heather Macbeth (Oct 06 2022 at 17:06):
I have written (#16775) a user command for push_neg
, so that one can type
#push_neg ¬(∃ x : ℝ, ∀ y, x < y → x = 3)
and see output in the infoview
∀ (x : ℝ), ∃ (y : ℝ), x < y ∧ x ≠ 3
I expect to use this for teaching, and maybe others will too.
Heather Macbeth (Oct 06 2022 at 17:07):
The code is copied blindly from #simp and #norm_num so it could use a careful review.
Kyle Miller (Oct 06 2022 at 17:11):
I made #norm_num
by copying blindly from #simp
, so I'll take a look :smile:
Last updated: Dec 20 2023 at 11:08 UTC