Skip to content

Commit

Permalink
Render as plain text
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata committed Jan 17, 2025
1 parent ccdb638 commit 898660a
Show file tree
Hide file tree
Showing 2 changed files with 12 additions and 14 deletions.
15 changes: 7 additions & 8 deletions Manual/Language/RecursiveDefs/PartialFixpoint.lean
Original file line number Diff line number Diff line change
Expand Up @@ -327,14 +327,6 @@ The tactic solves goals of the form `monotone (fun x => …)` using the followin
* Zeta-reducing a {keywordOf Lean.Parser.Term.let}`let` expression when value and type do depend on `x`.
* Applying lemmas annotated with {attr}`partial_fixpoint_monotone`

:::example "List of Monotonicity Lemmas"

::::TODO
Not really an example, but probably better to have this collapsible?
::::

The following monotonicity lemmas are registered, and should allow recursive calls in the indicated argument of the higher-order function:

::::TODO

What I’d like to see here is
Expand All @@ -345,6 +337,13 @@ where I use `·` and `_` to distinguish the monotone arguments from others.

::::

:::example "List of Monotonicity Lemmas"

{TODO}[Not really an example, but probably better to have this collapsible?]

The following monotonicity lemmas are registered, and should allow recursive calls in the indicated argument of the higher-order function:


{monotonicityLemmas}

:::
11 changes: 5 additions & 6 deletions Manual/Meta/Monotonicity.lean
Original file line number Diff line number Diff line change
Expand Up @@ -55,12 +55,11 @@ def monotonicityLemmas : BlockRoleExpander
let f := concl.appArg!
unless f.isLambda do
throwError "Unexpecte conclusion of {name}"
lambdaBoundedTelescope f 1 fun _ _call => do
-- Could not get this to work:
-- let _stx ← Lean.PrettyPrinter.delab call
-- `(Inline.code $(quote stx))
`(Inline.text "TODO")
-- pure (some stx)
lambdaBoundedTelescope f 1 fun _ call => do
let stx ← Lean.PrettyPrinter.delab call
let format := Syntax.prettyPrint stx
let str := format.pretty'
`(Inline.code $(quote str))

let hl : Highlighted ← constTok name name.toString
let nameStx ← `(Inline.other {Inline.name with data := ToJson.toJson $(quote hl)} #[Inline.code $(quote name.getString!)])
Expand Down

0 comments on commit 898660a

Please sign in to comment.