Skip to content

Commit

Permalink
fix(library/init/meta/tactic.lean): turn comment into docstring (#646)
Browse files Browse the repository at this point in the history
This seems to be a slip, rather than a deliberate decision to not make the comment above `subst_core` into its docstring. It's very rare that I try to read meta code, but today I was trying to understand how `subst` worked and ran into the fact that `subst_core` had no docstring.
  • Loading branch information
kbuzzard committed Nov 7, 2021
1 parent 63dc257 commit ace6534
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion library/init/meta/tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -516,7 +516,7 @@ meta constant mk_eq_trans : expr → expr → tactic expr
meta constant mk_eq_mp : expr → expr → tactic expr
/-- (mk_eq_mpr h₁ h₂) is a more efficient version of (mk_app `eq.mpr [h₁, h₂]) -/
meta constant mk_eq_mpr : expr → expr → tactic expr
/- Given a local constant t, if t has type (lhs = rhs) apply substitution.
/-- Given a local constant t, if t has type (lhs = rhs) apply substitution.
Otherwise, try to find a local constant that has type of the form (t = t') or (t' = t).
The tactic fails if the given expression is not a local constant. -/
meta constant subst_core : expr → tactic unit
Expand Down

0 comments on commit ace6534

Please sign in to comment.