lean2/tests/lean/run/blast_ematch_heq2.lean

11 lines
155 B
Text
Raw Permalink Normal View History

import algebra.group
variable {A : Type}
variable [s : group A]
include s
set_option blast.cc.heq true
example (a : A) : a * 1⁻¹ = a :=
by inst_simp