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

Commit

Permalink
feat(library/init/meta/tactic): add applyc tactic
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura committed Feb 25, 2017
1 parent 7ec0505 commit 04e27eb
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions library/init/meta/tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -769,6 +769,10 @@ do env ← get_env,
ls ← mk_num_meta_univs num,
return (expr.const c ls)

/-- Apply the constant `c` -/
meta def applyc (c : name) : tactic unit :=
mk_const c >>= apply

meta def save_const_type_info (n : name) (ref : expr) : tactic unit :=
try (do c ← mk_const n, save_type_info c ref)

Expand Down

0 comments on commit 04e27eb

Please sign in to comment.