Skip to content

Commit

Permalink
refactor: doc comment and remove redundant instance
Browse files Browse the repository at this point in the history
  • Loading branch information
mhuisi committed Jan 19, 2024
1 parent 2f6d2be commit 7946ee3
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 3 deletions.
5 changes: 5 additions & 0 deletions src/Lean/Elab/InfoTree/Types.lean
Original file line number Diff line number Diff line change
Expand Up @@ -44,6 +44,11 @@ node is always contained within a `commandCtx` node.
-/
inductive PartialContextInfo where
| commandCtx (info : CommandContextInfo)
/--
Context for the name of the declaration that surrounds nodes contained within this `context` node.
For example, this makes the name of the surrounding declaration available in `InfoTree` nodes
corresponding to the terms within the declaration.
-/
| parentDeclCtx (parentDecl : Name)
-- TODO: More constructors for the different kinds of scopes `commandCtx` is currently
-- used for (e.g. eliminating `Info.updateContext?` would be nice!).
Expand Down
3 changes: 0 additions & 3 deletions src/Lean/Elab/Tactic/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -51,9 +51,6 @@ instance : Monad TacticM :=
let i := inferInstanceAs (Monad TacticM);
{ pure := i.pure, bind := i.bind }

instance : MonadParentDecl TacticM where
getParentDeclName? := Term.getDeclName?

def getGoals : TacticM (List MVarId) :=
return (← get).goals

Expand Down

0 comments on commit 7946ee3

Please sign in to comment.