Skip to content

Commit

Permalink
chore: bump Lean toolchain
Browse files Browse the repository at this point in the history
  • Loading branch information
david-christiansen committed Jan 3, 2024
1 parent 4e70b19 commit 0ff2297
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:nightly-2023-12-04
leanprover/lean4:nightly-2023-12-31
4 changes: 2 additions & 2 deletions src/leandoc/LeanDoc/Doc/Concrete.lean
Original file line number Diff line number Diff line change
Expand Up @@ -59,10 +59,10 @@ elab "inlines!" s:inlineStr : term => open Lean Elab Term in
set_option pp.rawOnError true

/--
info: #[Inline.text "Hello, ", Inline.emph #[Inline.bold #[Inline.text "emph"]]] : Array (Inline ?m.11031)
info: #[Inline.text "Hello, ", Inline.emph #[Inline.bold #[Inline.text "emph"]]] : Array (Inline Genre.none)
-/
#guard_msgs in
#check inlines!"Hello, _*emph*_"
#check (inlines!"Hello, _*emph*_" : Array (Inline .none))

def document : Parser where
fn := rawFn <| atomicFn <| LeanDoc.Parser.document (blockContext := {maxDirective := some 6})
Expand Down

0 comments on commit 0ff2297

Please sign in to comment.