Zulip Chat Archive

Stream: new members

Topic: Example of adding clauses to get_elem_tactic_trivial


Mark Fischer (Feb 02 2024 at 19:42):

I'd like to be able to upgrade the get_elem_tactic tactic so that when I'm working with lists/sets/etc of equal length, I can grab elements a bit more smoothly. For example:

theorem foo {s t : List } (h : s.length = t.length) (i : ) : i < t.length  i < s.length := ...

def bar (a b : List ) (i : Fin a.length) (h : a.length = b.length) :  ×  := 
  a[i],
  b[i]'(by simp [foo h i])

I'm not really sure where to start looking though.


Last updated: May 02 2025 at 03:31 UTC