Skip to content
This repository has been archived by the owner on Oct 14, 2023. It is now read-only.

Commit

Permalink
fix(init/meta/interactive): mk_simp_set: also remove equational lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
Kha committed Mar 24, 2017
1 parent 028c0e6 commit a11ee6b
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion library/init/meta/interactive.lean
Original file line number Diff line number Diff line change
Expand Up @@ -507,7 +507,9 @@ private meta def simp_lemmas.append_pexprs : simp_lemmas → list pexpr → tact
private meta def mk_simp_set (attr_names : list name) (hs : list pexpr) (ex : list name) : tactic simp_lemmas :=
do s₀ ← join_user_simp_lemmas attr_names,
s₁ ← simp_lemmas.append_pexprs s₀ hs,
return $ simp_lemmas.erase s₁ ex
-- add equational lemmas, if any
ex ← ex^.mfor (λ n, list.cons n <$> get_eqn_lemmas_for tt n),
return $ simp_lemmas.erase s₁ $ ex^.join

private meta def simp_goal (cfg : simp_config) : simp_lemmas → tactic unit
| s := do
Expand Down

0 comments on commit a11ee6b

Please sign in to comment.