bookshelf-doc/DocGen4/IncludeStr.lean

27 lines
693 B
Plaintext
Raw Normal View History

2021-12-12 12:28:52 +00:00
/-
Copyright (c) 2021 Henrik Böving. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Henrik Böving
-/
import Lean
namespace DocGen4
open Lean System IO Lean.Elab.Term
syntax (name := includeStr) "include_str" str : term
@[termElab includeStr] def includeStrImpl : TermElab := λ stx expectedType? => do
let str := stx[1].isStrLit?.get!
let path := FilePath.mk str
if ←path.pathExists then
if ←path.isDir then
throwError s!"{str} is a directory"
else
let content ← FS.readFile path
2022-02-12 14:09:13 +00:00
pure $ mkStrLit content
else
throwError s!"\"{str}\" does not exist as a file"
end DocGen4