mathlib icon indicating copy to clipboard operation
mathlib copied to clipboard

apply' can close the goal with metavariables

Open fpvandoorn opened this issue 3 years ago • 0 comments

Example

import tactic.apply
import data.set.basic
example {α : Type*} (a b : set α) : a ⊆ b :=
by refl' -- closes the goal
-- by apply' set.subset.refl -- same behavior

Note, the following script shows that refl' (or apply') really makes no progress, and therefore should fail instead.

by { refl', recover, change a ⊆ b, }

fpvandoorn avatar Jun 27 '22 09:06 fpvandoorn