Skip to content

Commit b6d01e2

Browse files
Add test example
1 parent f91fcd0 commit b6d01e2

File tree

2 files changed

+71
-0
lines changed

2 files changed

+71
-0
lines changed
Lines changed: 68 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,68 @@
1+
{"tactics":
2+
[{"usedConstants":
3+
["Nat.gcd",
4+
"HMul.hMul",
5+
"Mathlib.Meta.NormNum.isNat_eq_true",
6+
"instMulNat",
7+
"instOfNatNat",
8+
"Mathlib.Meta.NormNum.isNat_ofNat",
9+
"Tactic.NormNum.nat_gcd_helper_2",
10+
"Nat.instAddMonoidWithOne",
11+
"Nat",
12+
"Eq.refl",
13+
"Mathlib.Meta.NormNum.instAddMonoidWithOneNat",
14+
"Tactic.NormNum.isNat_gcd",
15+
"OfNat.ofNat",
16+
"instHMul"],
17+
"tactic": "norm_num",
18+
"proofState": 0,
19+
"pos": {"line": 2, "column": 60},
20+
"goals": "⊢ Nat.gcd 180 168 = 12",
21+
"endPos": {"line": 2, "column": 68}},
22+
{"usedConstants": ["Eq.refl"],
23+
"tactic": "rfl",
24+
"proofState": 1,
25+
"pos": {"line": 10, "column": 2},
26+
"goals": "α✝ : Sort u_1\nn : α✝\n⊢ n = n",
27+
"endPos": {"line": 10, "column": 5}}],
28+
"messages":
29+
[{"severity": "info",
30+
"pos": {"line": 8, "column": 0},
31+
"endPos": {"line": 8, "column": 5},
32+
"data": "9227465"}],
33+
"env": 0}
34+
35+
{"tactics":
36+
[{"usedConstants":
37+
["Nat.gcd",
38+
"HMul.hMul",
39+
"Mathlib.Meta.NormNum.isNat_eq_true",
40+
"instMulNat",
41+
"instOfNatNat",
42+
"Mathlib.Meta.NormNum.isNat_ofNat",
43+
"Tactic.NormNum.nat_gcd_helper_2",
44+
"Nat.instAddMonoidWithOne",
45+
"Nat",
46+
"Eq.refl",
47+
"Mathlib.Meta.NormNum.instAddMonoidWithOneNat",
48+
"Tactic.NormNum.isNat_gcd",
49+
"OfNat.ofNat",
50+
"instHMul"],
51+
"tactic": "norm_num",
52+
"proofState": 2,
53+
"pos": {"line": 2, "column": 60},
54+
"goals": "⊢ Nat.gcd 180 168 = 12",
55+
"endPos": {"line": 2, "column": 68}},
56+
{"usedConstants": ["Nat", "Eq.refl"],
57+
"tactic": "rfl",
58+
"proofState": 3,
59+
"pos": {"line": 10, "column": 2},
60+
"goals": "n : ℕ\n⊢ n = n + 0",
61+
"endPos": {"line": 10, "column": 5}}],
62+
"messages":
63+
[{"severity": "info",
64+
"pos": {"line": 8, "column": 0},
65+
"endPos": {"line": 8, "column": 5},
66+
"data": "9227465"}],
67+
"env": 1}
68+
Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,3 @@
1+
{"cmd": "import Mathlib\ntheorem mathd_numbertheory_188 : Nat.gcd 180 168 = 12 := by norm_num\ndef fib : Nat → Nat\n | 0 => 0\n | 1 => 1\n | n + 2 => fib (n + 1) + fib n\n\n#eval fib 35\ntheorem foo : n = n := by\n rfl", "allTactics": true}
2+
3+
{"cmd": "import Mathlib\ntheorem mathd_numbertheory_188 : Nat.gcd 180 168 = 12 := by norm_num\ndef fib : Nat → Nat\n | 0 => 0\n | 1 => 1\n | n + 2 => fib (n + 1) + fib n\n\n#eval fib 35\ntheorem foo2 : n = n+0 := by\n rfl", "allTactics": true}

0 commit comments

Comments
 (0)