Zulip Chat Archive
Stream: triage
Topic: issue #1535: have `library_search` call `symmetry` before...
Random Issue Bot (Nov 07 2020 at 14:16):
Today I chose issue 1535 for discussion!
have library_search
call symmetry
before giving up
Created by @Scott Morrison (@semorrison) on 2019-10-09
Labels: feature-request, meta
Is this issue still relevant? Any recent updates? Anyone making progress?
Random Issue Bot (Dec 14 2020 at 14:25):
Today I chose issue 1535 for discussion!
have library_search
call symmetry
before giving up
Created by @Scott Morrison (@semorrison) on 2019-10-09
Labels: feature-request, meta
Is this issue still relevant? Any recent updates? Anyone making progress?
Rob Lewis (Dec 14 2020 at 15:52):
I think this is implemented already, right?
import tactic.suggest
constants P Q : Prop
axiom pq : P ↔ Q
example : Q ↔ P := by library_search
constants a b : ℕ
axiom ab : a = b
example : b = a := by library_search
Rob Lewis (Dec 14 2020 at 15:53):
Yes, #2415
Last updated: Dec 20 2023 at 11:08 UTC