Skip to content

Commit 2a0af34

Browse files
committed
restore test
1 parent d0935fc commit 2a0af34

File tree

1 file changed

+73
-1
lines changed

1 file changed

+73
-1
lines changed

tests/lean/run/info_trees.lean

Lines changed: 73 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2,6 +2,78 @@
22
-- If it proves too fragile to test the result using `#guard_msgs`,
33
-- it is fine to simply remove the `#guard_msgs` and expected output.
44

5-
#guard_msgs (drop info) in
5+
/--
6+
info: • [Command] @ ⟨79, 0⟩-⟨79, 40⟩ @ Lean.Elab.Command.elabDeclaration
7+
[Term] Nat : Type @ ⟨79, 15⟩-⟨79, 18⟩ @ Lean.Elab.Term.elabIdent
8+
[Completion-Id] Nat : some Sort.{?_uniq.1} @ ⟨79, 15⟩-⟨79, 18⟩
9+
[Term] Nat : Type @ ⟨79, 15⟩-⟨79, 18⟩
10+
[Term] n (isBinder := true) : Nat @ ⟨79, 11⟩-⟨79, 12⟩
11+
[Term] 0 ≤ n : Prop @ ⟨79, 22⟩-⟨79, 27⟩ @ «_aux_Init_Notation___macroRules_term_≤__2»
12+
[MacroExpansion]
13+
0 ≤ n
14+
===>
15+
binrel% LE.le✝ 0 n
16+
[Term] 0 ≤ n : Prop @ ⟨79, 22⟩†-⟨79, 27⟩† @ Lean.Elab.Term.Op.elabBinRel
17+
[Term] 0 ≤ n : Prop @ ⟨79, 22⟩†-⟨79, 27⟩†
18+
[Completion-Id] LE.le✝ : none @ ⟨79, 22⟩†-⟨79, 27⟩†
19+
[Term] 0 : Nat @ ⟨79, 22⟩-⟨79, 23⟩ @ Lean.Elab.Term.elabNumLit
20+
[Term] n : Nat @ ⟨79, 26⟩-⟨79, 27⟩ @ Lean.Elab.Term.elabIdent
21+
[Completion-Id] n : none @ ⟨79, 26⟩-⟨79, 27⟩
22+
[Term] n : Nat @ ⟨79, 26⟩-⟨79, 27⟩
23+
[CustomInfo(Lean.Elab.Term.AsyncBodyInfo)]
24+
[Term] n (isBinder := true) : Nat @ ⟨79, 11⟩-⟨79, 12⟩
25+
[CustomInfo(Lean.Elab.Term.BodyInfo)]
26+
[Tactic] @ ⟨79, 31⟩-⟨79, 40⟩
27+
(Term.byTactic
28+
"by"
29+
(Tactic.tacticSeq (Tactic.tacticSeq1Indented [(Tactic.exact? "exact?" (Tactic.optConfig []) [])])))
30+
before ⏎
31+
n : Nat
32+
⊢ 0 ≤ n
33+
after no goals
34+
[Tactic] @ ⟨79, 31⟩-⟨79, 33⟩
35+
"by"
36+
before ⏎
37+
n : Nat
38+
⊢ 0 ≤ n
39+
after no goals
40+
[Tactic] @ ⟨79, 34⟩-⟨79, 40⟩ @ Lean.Elab.Tactic.evalTacticSeq
41+
(Tactic.tacticSeq (Tactic.tacticSeq1Indented [(Tactic.exact? "exact?" (Tactic.optConfig []) [])]))
42+
before ⏎
43+
n : Nat
44+
⊢ 0 ≤ n
45+
after no goals
46+
[Tactic] @ ⟨79, 34⟩-⟨79, 40⟩ @ Lean.Elab.Tactic.evalTacticSeq1Indented
47+
(Tactic.tacticSeq1Indented [(Tactic.exact? "exact?" (Tactic.optConfig []) [])])
48+
before ⏎
49+
n : Nat
50+
⊢ 0 ≤ n
51+
after no goals
52+
[Tactic] @ ⟨79, 34⟩-⟨79, 40⟩ @ Lean.Elab.LibrarySearch.evalExact
53+
(Tactic.exact? "exact?" (Tactic.optConfig []) [])
54+
before ⏎
55+
n : Nat
56+
⊢ 0 ≤ n
57+
after no goals
58+
[Tactic] @ ⟨79, 34⟩†-⟨79, 40⟩† @ Lean.Elab.Tactic.evalExact
59+
(Tactic.exact "exact" (Term.app `Nat.zero_le [`n]))
60+
before ⏎
61+
n : Nat
62+
⊢ 0 ≤ n
63+
after no goals
64+
[Term] Nat.zero_le n : 0 ≤ n @ ⟨1, 1⟩†-⟨1, 1⟩† @ Lean.Elab.Term.elabApp
65+
[Completion-Id] Nat.zero_le : some LE.le.{0} Nat instLENat (OfNat.ofNat.{0} Nat 0 (instOfNatNat 0)) _uniq.37 @ ⟨1, 0⟩†-⟨1, 0⟩†
66+
[Term] Nat.zero_le : ∀ (n : Nat), 0 ≤ n @ ⟨1, 0⟩†-⟨1, 0⟩†
67+
[Term] n : Nat @ ⟨1, 5⟩†-⟨1, 5⟩† @ Lean.Elab.Term.elabIdent
68+
[Completion-Id] n : some Nat @ ⟨1, 5⟩†-⟨1, 5⟩†
69+
[Term] n : Nat @ ⟨1, 5⟩†-⟨1, 5⟩†
70+
[CustomInfo(Lean.Meta.Tactic.TryThis.TryThisInfo)]
71+
[Term] t (isBinder := true) : ∀ (n : Nat), 0 ≤ n @ ⟨79, 8⟩-⟨79, 9⟩
72+
[Term] t (isBinder := true) : ∀ (n : Nat), 0 ≤ n @ ⟨79, 8⟩-⟨79, 9⟩
73+
---
74+
info: Try this:
75+
[apply] exact Nat.zero_le n
76+
-/
77+
#guard_msgs in
678
#info_trees in
779
theorem t (n : Nat) : 0 ≤ n := by exact?

0 commit comments

Comments
 (0)