Skip to content

Commit

Permalink
feat: SubVerso support for using a name as an example
Browse files Browse the repository at this point in the history
This makes it easier to just refer to a name in the text.
  • Loading branch information
david-christiansen committed May 15, 2024
1 parent c4622e3 commit ef41c92
Show file tree
Hide file tree
Showing 2 changed files with 32 additions and 1 deletion.
2 changes: 2 additions & 0 deletions demo/Demo.lean
Original file line number Diff line number Diff line change
Expand Up @@ -28,3 +28,5 @@ theorem test (n : Nat) : n * 1 = n := by
def test2 [ToString α] (x : α) : Decidable (toString x = "") := by
constructor; sorry
%end

%show_name Nat.rec
31 changes: 30 additions & 1 deletion src/examples/SubVerso/Examples.lean
Original file line number Diff line number Diff line change
Expand Up @@ -13,7 +13,6 @@ scoped syntax "%ex" "{" ident (" : " term)? "}" "{" term "}" : term
scoped syntax "%ex" "{" ident "}" "{" tactic "}" : tactic
scoped syntax "%ex" "{" ident "}" "{" doElem "}" : doElem


class MonadMessageState (m : TypeType v) where
getMessages : m MessageLog
setMessages : MessageLog → m Unit
Expand Down Expand Up @@ -148,6 +147,34 @@ elab_rules : command
else
throwErrorAt name "No highlighting found for '{name}'"

namespace Internals
scoped syntax "%show_name" ident : term
elab_rules : term
| `(%show_name $x) => do
let _ ← Compat.realizeNameNoOverloads x
elabTerm (← `((() : Unit))) none

end Internals

scoped syntax "%show_name" ident ("as" ident)? : command

macro_rules
| `(%show_name $x) => `(%show_name $x as $x)

open Internals in
elab_rules : command
| `(%show_name $x as $name) => do
_ ← elabCommand <| ← `(def helper := %show_name $x)
let trees ← getInfoTrees
let mod ← getMainModule
let text ← getFileMap
let .original leading startPos trailing stopPos := x.raw.getHeadInfo
| throwErrorAt x "Failed to get source position"
let str := text.source.extract leading.startPos trailing.stopPos
let hl ← liftTermElabM <| highlight x #[] trees
modifyEnv fun ρ =>
highlighted.addEntry ρ (mod, name.getId, {highlighted := #[hl], original := str, start := text.toPosition startPos, stop := text.toPosition stopPos, messages := []})

open System in
partial def loadExamples
(leanProject : FilePath)
Expand Down Expand Up @@ -233,3 +260,5 @@ def wxyz (n : Nat) := 1 + 3 + n
#check wxyz
def xyz (n : Nat) := 1 + %ex{test2}{3 + n}
%end

%show_name Nat.rec

0 comments on commit ef41c92

Please sign in to comment.