Skip to content

Commit

Permalink
Improve comments
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata committed Jan 8, 2024
1 parent 0caafcb commit 8278b00
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions src/Lean/Elab/PreDefinition/WF/Fix.lean
Original file line number Diff line number Diff line change
Expand Up @@ -188,8 +188,9 @@ def assignSubsumed (mvars : Array MVarId) : MetaM (Array MVarId) :=
return (true, true)

/--
The subgoals are of the form `rel arg param`, where `param` is the `PackMutual`'ed parameter
of the current function, and thus we can peek at that to know which function is making the call.
The subgoals, created by `mkDecreasingProof`, are of the form `[data _recApp: rel arg param]`, where
`param` is the `PackMutual`'ed parameter of the current function, and thus we can peek at that to
know which function is making the call.
The close coupling with how arguments are packed and termination goals look like is not great,
but it works for now.
-/
Expand Down

0 comments on commit 8278b00

Please sign in to comment.