feat: Improved todo list
This commit is contained in:
parent
1b2cc5338f
commit
ca044d3786
37 changed files with 180 additions and 42 deletions
|
@ -4,6 +4,7 @@ Released under Apache 2.0 license.
|
|||
Authors: Joseph Tooby-Smith
|
||||
-/
|
||||
import Lean
|
||||
import HepLean.Meta.TODO.Basic
|
||||
/-!
|
||||
|
||||
## Informal definitions and lemmas
|
||||
|
@ -16,7 +17,7 @@ Everything else about informal definitions and lemmas are in the `Informal.Post`
|
|||
-/
|
||||
open Lean Elab System
|
||||
|
||||
/-! TODO: Can likely make this a bona-fide command. -/
|
||||
TODO "Can likely make this a bona-fide command."
|
||||
|
||||
/-- The structure representing an informal definition. -/
|
||||
structure InformalDefinition where
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue