blob: fd95291e0fa4f01122f7c8a97761a64a7efc53ad (
plain)
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
85
86
87
88
89
90
91
92
93
94
95
96
97
98
99
100
101
102
103
104
105
106
107
108
109
110
111
112
113
114
115
116
117
118
119
120
121
122
|
import Lean
namespace Diverge
open Lean Elab Term Meta
initialize registerTraceClass `Diverge.elab
initialize registerTraceClass `Diverge.def
initialize registerTraceClass `Diverge.def.sigmas
initialize registerTraceClass `Diverge.def.genBody
initialize registerTraceClass `Diverge.def.valid
initialize registerTraceClass `Diverge.def.unfold
-- TODO: move
-- TODO: small helper
def explore_term (incr : String) (e : Expr) : MetaM Unit :=
match e with
| .bvar _ => do logInfo m!"{incr}bvar: {e}"; return ()
| .fvar _ => do logInfo m!"{incr}fvar: {e}"; return ()
| .mvar _ => do logInfo m!"{incr}mvar: {e}"; return ()
| .sort _ => do logInfo m!"{incr}sort: {e}"; return ()
| .const _ _ => do logInfo m!"{incr}const: {e}"; return ()
| .app fn arg => do
logInfo m!"{incr}app: {e}"
explore_term (incr ++ " ") fn
explore_term (incr ++ " ") arg
| .lam _bName bTy body _binfo => do
logInfo m!"{incr}lam: {e}"
explore_term (incr ++ " ") bTy
explore_term (incr ++ " ") body
| .forallE _bName bTy body _bInfo => do
logInfo m!"{incr}forallE: {e}"
explore_term (incr ++ " ") bTy
explore_term (incr ++ " ") body
| .letE _dName ty val body _nonDep => do
logInfo m!"{incr}letE: {e}"
explore_term (incr ++ " ") ty
explore_term (incr ++ " ") val
explore_term (incr ++ " ") body
| .lit _ => do logInfo m!"{incr}lit: {e}"; return ()
| .mdata _ e => do
logInfo m!"{incr}mdata: {e}"
explore_term (incr ++ " ") e
| .proj _ _ struct => do
logInfo m!"{incr}proj: {e}"
explore_term (incr ++ " ") struct
def explore_decl (n : Name) : TermElabM Unit := do
logInfo m!"Name: {n}"
let env ← getEnv
let decl := env.constants.find! n
match decl with
| .defnInfo val =>
logInfo m!"About to explore defn: {decl.name}"
logInfo m!"# Type:"
explore_term "" val.type
logInfo m!"# Value:"
explore_term "" val.value
| .axiomInfo _ => throwError m!"axiom: {n}"
| .thmInfo _ => throwError m!"thm: {n}"
| .opaqueInfo _ => throwError m!"opaque: {n}"
| .quotInfo _ => throwError m!"quot: {n}"
| .inductInfo _ => throwError m!"induct: {n}"
| .ctorInfo _ => throwError m!"ctor: {n}"
| .recInfo _ => throwError m!"rec: {n}"
syntax (name := printDecl) "print_decl " ident : command
open Lean.Elab.Command
@[command_elab printDecl] def elabPrintDecl : CommandElab := fun stx => do
liftTermElabM do
let id := stx[1]
addCompletionInfo <| CompletionInfo.id id id.getId (danglingDot := false) {} none
let cs ← resolveGlobalConstWithInfos id
explore_decl cs[0]!
private def test1 : Nat := 0
private def test2 (x : Nat) : Nat := x
print_decl test1
print_decl test2
-- We adapted this from AbstractNestedProofs.visit
-- A map visitor function for expressions
partial def mapVisit (k : Expr → MetaM Expr) (e : Expr) : MetaM Expr := do
let mapVisitBinders (xs : Array Expr) (k2 : MetaM Expr) : MetaM Expr := do
let localInstances ← getLocalInstances
let mut lctx ← getLCtx
for x in xs do
let xFVarId := x.fvarId!
let localDecl ← xFVarId.getDecl
let type ← mapVisit k localDecl.type
let localDecl := localDecl.setType type
let localDecl ← match localDecl.value? with
| some value => let value ← mapVisit k value; pure <| localDecl.setValue value
| none => pure localDecl
lctx :=lctx.modifyLocalDecl xFVarId fun _ => localDecl
withLCtx lctx localInstances k2
-- TODO: use a cache? (Lean.checkCache)
-- Explore
let e ← k e
match e with
| .bvar _
| .fvar _
| .mvar _
| .sort _
| .lit _
| .const _ _ => pure e
| .app .. => do e.withApp fun f args => return mkAppN f (← args.mapM (mapVisit k))
| .lam .. =>
lambdaLetTelescope e fun xs b =>
mapVisitBinders xs do mkLambdaFVars xs (← mapVisit k b) (usedLetOnly := false)
| .forallE .. => do
forallTelescope e fun xs b => mapVisitBinders xs do mkForallFVars xs (← mapVisit k b)
| .letE .. => do
lambdaLetTelescope e fun xs b => mapVisitBinders xs do
mkLambdaFVars xs (← mapVisit k b) (usedLetOnly := false)
| .mdata _ b => return e.updateMData! (← mapVisit k b)
| .proj _ _ b => return e.updateProj! (← mapVisit k b)
end Diverge
|