PhysLean/HepLean/Meta/Notes/NoteFile.lean
KUO-TSAN HSU (Gordon) f8f94979ab
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
2025-02-02 03:17:17 +08:00

38 lines
851 B
Text

/-
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
Released under Apache 2.0 license.
Authors: Joseph Tooby-Smith
-/
import HepLean.Meta.Notes.Basic
/-!
# Note file
A note file is a structure which contains the information to go into a note.
-/
namespace HepLean
open Lean
/-- A note consists of a title and a list of Lean files which make up the note. -/
structure NoteFile where
/-- The overall title of the note. -/
title : String
/-- The abstract of the note. -/
abstract : String
/-- A list of authors. -/
authors : List String
/-- The files making up the note in the order in which they should appear. -/
files : List Name
namespace NoteFile
variable (N : NoteFile)
/-- All imports associated to a note. -/
def imports : Array Import := (N.files.map fun f => {module := f}).toArray
end NoteFile
end HepLean