File tree Expand file tree Collapse file tree 2 files changed +4
-16
lines changed Expand file tree Collapse file tree 2 files changed +4
-16
lines changed Original file line number Diff line number Diff line change @@ -15,12 +15,8 @@ set_option pp.rawOnError true
15
15
set_option guard_msgs.diff true
16
16
17
17
18
- def Inline.errorExplanationLink (errorName : Name) : Manual.Inline where
19
- name := `Manual.Inline.errorExplanationLink
18
+ inline_extension Inline.errorExplanationLink (errorName : Name) where
20
19
data := toJson errorName
21
-
22
- @[inline_extension Inline.errorExplanationLink]
23
- def Inline.errorExplanationLink.descr : InlineDescr where
24
20
traverse := fun _ _ _ => pure none
25
21
toTeX := none
26
22
toHtml := some fun go _ data content =>
Original file line number Diff line number Diff line change @@ -62,16 +62,12 @@ def explanationMWE : CodeBlockExpander
62
62
(Block.lean $(quote hls) (some $(quote (← getFileName))) none)
63
63
#[Block.code $str])]
64
64
65
- /--
65
+ /-
66
66
A tabbed container for MWEs in an error explanation example. Must satisfy the
67
67
invariant that `titles.size` is equal to the number of children of this block.
68
68
-/
69
- def Block.tabbedMWEs (titles : Array String) : Block where
70
- name := `Manual.Block.tabbedMWEs
69
+ block_extension Block.tabbedMWEs (titles : Array String) where
71
70
data := toJson titles
72
-
73
- @[block_extension Block.tabbedMWEs]
74
- def Block.tabbedMWEs.descr : BlockDescr where
75
71
traverse id data _blocks := do
76
72
let name :=
77
73
match FromJson.fromJson? (α := Option String) data with
@@ -550,12 +546,8 @@ def addExplanationBodyBlocks : ExplanElabM Unit := do
550
546
551
547
deriving instance Quote for ErrorExplanation.Metadata
552
548
553
- def Block.errorExplanationMetadata (metadata : ErrorExplanation.Metadata) : Block where
554
- name := `Manual.Block.errorExplanationMetadata
549
+ block_extension Block.errorExplanationMetadata (metadata : ErrorExplanation.Metadata) where
555
550
data := toJson metadata
556
-
557
- @[block_extension Block.errorExplanationMetadata]
558
- def Block.errorExplanationMetadata.descr : BlockDescr where
559
551
traverse _ _ _ := pure none
560
552
toTeX := none
561
553
extraCss := ["
You can’t perform that action at this time.
0 commit comments