feat: make informal_definition and informal_lemma commands (#300)
* make informal_definition and informal_lemma commands * drop the fields "math", "physics", and "proof" from InformalDefinition/InformalLemma and use docstrings instead * render informal docstring in dependency graph
This commit is contained in:
parent
6aab0ba3cd
commit
f8f94979ab
33 changed files with 666 additions and 1089 deletions
|
@ -3,12 +3,6 @@ Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
|
|||
Released under Apache 2.0 license.
|
||||
Authors: Joseph Tooby-Smith
|
||||
-/
|
||||
import Batteries.Lean.HashSet
|
||||
import Lean
|
||||
import Mathlib.Lean.Expr.Basic
|
||||
import Mathlib.Lean.CoreM
|
||||
import HepLean.Meta.Informal.Post
|
||||
import ImportGraph.RequiredModules
|
||||
|
||||
def main (_: List String) : IO UInt32 := do
|
||||
println! "Style lint ... "
|
||||
|
@ -20,9 +14,6 @@ def main (_: List String) : IO UInt32 := do
|
|||
println! "File imports ... "
|
||||
let importCheck ← IO.Process.output {cmd := "lake", args := #["exe", "check_file_imports"]}
|
||||
println! importCheck.stdout
|
||||
println! "Doc check ..."
|
||||
let docCheck ← IO.Process.output {cmd := "lake", args := #["exe", "no_docs"]}
|
||||
println! docCheck.stdout
|
||||
println! "Lean linter ..."
|
||||
let leanCheck ← IO.Process.output {cmd := "lake", args := #["exe", "runLinter", "HepLean"]}
|
||||
println! leanCheck.stdout
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue