Skip to content
This repository was archived by the owner on Aug 24, 2024. It is now read-only.

Commit 34df8ff

Browse files
committed
chore: update test capture
1 parent 21dadc6 commit 34df8ff

File tree

4 files changed

+38
-7
lines changed

4 files changed

+38
-7
lines changed

test/playground/infoTree.lean.leanInk.expected

Lines changed: 20 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,24 @@
1818
{"contents":
1919
"\n\ndef f2 : (x y : Nat) → (b : Bool) → Nat :=\n fun x y b =>\n let (z, w) := (x + y, x - y)\n let z1 := z + w\n z + z1\n\ndef f3 (s : Nat × Array (Array Nat)) : Array Nat :=\n s.2[1].push s.1\n\ndef f4 (arg : B) : Nat :=\n arg.pair.fst.val 0\n\ndef f5 (x : Nat) : B := {\n pair := ({ val := id }, { val := id })\n}\n\nopen Nat in\n",
2020
"_type": "text"},
21-
{"contents": "#print", "_type": "text"},
21+
{"messages":
22+
[{"contents": "def Nat.xor : Nat → Nat → Nat :=\nbitwise bne\n",
23+
"_type": "message"}],
24+
"goals": [],
25+
"contents": "#print",
26+
"_type": "sentence"},
2227
{"contents": " xor\ninstance : Inhabited Nat where\n\n", "_type": "text"},
23-
{"contents": "macro", "_type": "text"},
24-
{"contents": "", "_type": "text"}]
28+
{"messages":
29+
[{"contents": "infoTree.lean:39:0: error: expected identifier or term\n",
30+
"_type": "message"}],
31+
"goals": [],
32+
"contents": "macro",
33+
"_type": "sentence"},
34+
{"messages":
35+
[{"contents": "infoTree.lean:39:0: error: expected identifier or term\n",
36+
"_type": "message"},
37+
{"contents": "infoTree.lean:39:5: error: unexpected end of input\n",
38+
"_type": "message"}],
39+
"goals": [],
40+
"contents": "",
41+
"_type": "sentence"}]

test/playground/playground_1.lean.leanInk.expected

Lines changed: 8 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,9 +1,15 @@
11
[{"contents":
22
"/-|\n=======\n Title\n=======\n\nProse. *Emphasis*; **strong emphasis**; ``code``; `coq code`; `link <url>`__.\n|-/\n\n",
33
"_type": "text"},
4-
{"contents": "#check", "_type": "text"},
4+
{"messages": [{"contents": "Bool : Type\n", "_type": "message"}],
5+
"goals": [],
6+
"contents": "#check",
7+
"_type": "sentence"},
58
{"contents": " Bool\n\n", "_type": "text"},
6-
{"contents": "#print", "_type": "text"},
9+
{"messages": [{"contents": "Hello World\n", "_type": "message"}],
10+
"goals": [],
11+
"contents": "#print",
12+
"_type": "sentence"},
713
{"contents":
814
" \"Hello World\"\n\nexample (p q r : Prop) : p ∧ (q ∨ r) ↔ (p ∧ q) ∨ (p ∧ r) := ",
915
"_type": "text"},
Lines changed: 6 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,9 @@
11
[{"contents": "theorem test (p q : Prop) (hp : p) (hq : q) : p ∧ q ∧ p :=\n ",
22
"_type": "text"},
3-
{"contents": "sorry", "_type": "text"},
3+
{"messages":
4+
[{"contents": "001.lean:2:2: warning: declaration uses 'sorry'\n",
5+
"_type": "message"}],
6+
"goals": [],
7+
"contents": "sorry",
8+
"_type": "sentence"},
49
{"contents": "", "_type": "text"}]

test/theorem_proving/005.lean.leanInk.expected

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -49,5 +49,8 @@
4949
"contents": "exact And.intro hq hp",
5050
"_type": "sentence"},
5151
{"contents": "\n\n", "_type": "text"},
52-
{"contents": "#check", "_type": "text"},
52+
{"messages": [{"contents": "And : Prop → Prop → Prop\n", "_type": "message"}],
53+
"goals": [],
54+
"contents": "#check",
55+
"_type": "sentence"},
5356
{"contents": " And", "_type": "text"}]

0 commit comments

Comments
 (0)