File tree Expand file tree Collapse file tree 2 files changed +15
-0
lines changed Expand file tree Collapse file tree 2 files changed +15
-0
lines changed Original file line number Diff line number Diff line change @@ -39,6 +39,7 @@ import Mathlib.Mathport.Syntax
39
39
import Mathlib.Tactic.Basic
40
40
import Mathlib.Tactic.Cache
41
41
import Mathlib.Tactic.Coe
42
+ import Mathlib.Tactic.CommandQuote
42
43
import Mathlib.Tactic.Core
43
44
import Mathlib.Tactic.Ext
44
45
import Mathlib.Tactic.Find
Original file line number Diff line number Diff line change
1
+ /-
2
+ Copyright (c) 2021 Microsoft Corporation. All rights reserved.
3
+ Released under Apache 2.0 license as described in the file LICENSE.
4
+ Authors: Mario Carneiro
5
+ -/
6
+ import Lean
7
+
8
+ namespace Lean
9
+
10
+ @[termParser default+1] def Parser.Term.Command.quot : Parser :=
11
+ leading_parser "`(command|" >> incQuotDepth commandParser >> ")"
12
+
13
+ @[termElab Command.quot] def Elab.Term.elabCommandQuot : TermElab :=
14
+ adaptExpander Quotation.stxQuot.expand
You can’t perform that action at this time.
0 commit comments