Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 6eedc0e

Browse files
committed
feat(tactic/norm_num): rewrite norm_num to use simp instead of reflection
1 parent 0663945 commit 6eedc0e

File tree

3 files changed

+195
-577
lines changed

3 files changed

+195
-577
lines changed

tactic/interactive.lean

Lines changed: 11 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -82,5 +82,16 @@ do max ← i_to_expr_strict max >>= tactic.eval_expr nat,
8282
meta def substs (l : parse ident*) : tactic unit :=
8383
l.mmap' (λ h, get_local h >>= tactic.subst)
8484

85+
meta def unfold_coes (loc : parse location) : tactic unit :=
86+
unfold [`coe,`lift_t,`has_lift_t.lift,`coe_t,`has_coe_t.coe,`coe_b,`has_coe.coe] loc
87+
88+
meta def recover : tactic unit :=
89+
do r ← tactic.result,
90+
tactic.set_goals $ r.fold [] $ λ e _ l,
91+
match e with
92+
| expr.mvar _ _ _ := insert e l
93+
| _ := l
94+
end
95+
8596
end interactive
8697
end tactic

0 commit comments

Comments
 (0)