-
Notifications
You must be signed in to change notification settings - Fork 14
/
lakefile.lean
84 lines (68 loc) · 2.36 KB
/
lakefile.lean
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
import Lake
open Lake DSL
require subverso from git "https://github.com/leanprover/subverso.git"@"main"
require MD4Lean from git "https://github.com/david-christiansen/md4lean"@"parser"
package verso where
precompileModules := true
-- add package configuration options here
@[default_target]
lean_lib Verso where
srcDir := "src/verso"
roots := #[`Verso]
@[default_target]
lean_lib VersoBlog where
srcDir := "src/verso-blog"
roots := #[`VersoBlog]
@[default_target]
lean_lib VersoManual where
srcDir := "src/verso-manual"
roots := #[`VersoManual]
@[default_target]
lean_exe «verso» where
root := `Main
-- Enables the use of the Lean interpreter by the executable (e.g.,
-- `runFrontend`) at the expense of increased binary size on Linux.
-- Remove this line if you do not need such functionality.
supportInterpreter := true
lean_lib UsersGuide where
srcDir := "doc"
@[default_target]
lean_exe usersguide where
root := `UsersGuideMain
-- Enables the use of the Lean interpreter by the executable (e.g.,
-- `runFrontend`) at the expense of increased binary size on Linux.
-- Remove this line if you do not need such functionality.
supportInterpreter := true
-- A demo site that shows how to generate websites with Verso
lean_lib DemoSite where
srcDir := "examples/website"
roots := #[`DemoSite]
@[default_target]
lean_exe demosite where
srcDir := "examples/website"
root := `DemoSiteMain
-- Enables the use of the Lean interpreter by the executable (e.g.,
-- `runFrontend`) at the expense of increased binary size on Linux.
-- Remove this line if you do not need such functionality.
supportInterpreter := true
-- An example of a textbook project built in Verso
lean_lib DemoTextbook where
srcDir := "examples/textbook"
roots := #[`DemoTextbook]
@[default_target]
lean_exe demotextbook where
srcDir := "examples/textbook"
root := `DemoTextbookMain
-- Enables the use of the Lean interpreter by the executable (e.g.,
-- `runFrontend`) at the expense of increased binary size on Linux.
-- Remove this line if you do not need such functionality.
supportInterpreter := true
-- An example of a minimal nontrivial custom genre
@[default_target]
lean_lib SimplePage where
srcDir := "examples/custom-genre"
roots := #[`SimplePage]
@[default_target]
lean_exe simplepage where
srcDir := "examples/custom-genre"
root := `SimplePageMain