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

Commit 1e61dc9

Browse files
committed
chore: update expected test files
1 parent d9510d6 commit 1e61dc9

File tree

7 files changed

+8
-8
lines changed

7 files changed

+8
-8
lines changed

test/dep/Dep.lean.leanInk.expected

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
11
[{"contents":
2-
"import Mathlib.Tactic.Basic\n\nexample : ∀ a b : Nat, a = b → b = a := by\n ",
2+
"import Mathlib.Tactic.Basic\n\nset_option trace.Elab.info true\n\nexample : ∀ a b : Nat, a = b → b = a := by\n ",
33
"_type": "text"},
44
{"messages": [],
55
"goals":

test/dep/lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2021-12-26
1+
leanprover/lean4:nightly-2022-01-06

test/playground/Function.lean.leanInk.expected

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -62,5 +62,5 @@
6262
"_type": "sentence"},
6363
{"messages": [], "goals": [], "contents": "]", "_type": "sentence"},
6464
{"contents":
65-
"\n\ntheorem injective_id : injective (@id α) := id\n\ntheorem surjective_id : surjective (@id α) := λ a => ⟨a, rfl⟩\n\ntheorem bijective_id : bijective (@id α) := ⟨injective_id, surjective_id⟩\n\nend Function\n\nnamespace Function\n\nvariable {α : Type u₁} {β : Type u₂} {φ : Type u₃}\n\n/-- Interpret a function on `α × β` as a function with two arguments. -/\n@[inline] def curry : (α × β → φ) → α → β → φ :=\nλ f a b => f (a, b)\n\n/-- Interpret a function with two arguments as a function on `α × β` -/\n@[inline] def",
65+
"\n\ntheorem injective_id : injective (@id α) := id\n\ntheorem surjective_id : surjective (@id α) := λ a => ⟨a, rfl⟩\n\ntheorem bijective_id : bijective (@id α) := ⟨injective_id, surjective_id⟩\n\nend Function\n\nnamespace Function\n\nvariable {α : Type u₁} {β : Type u₂} {φ : Type u₃}\n\n/-- Interpret a function on `α × β` as a function with two arguments. -/\n@[inline] def curry : (α × β → φ) → α → β → φ :=\nλ f a b => f (a, b)\n\n/-- Interpret a function with two arguments as a function on `α × β` -/\n@[inline] def uncurry : (α → β → φ) → α × β → φ :=\nλ f a => f a.1 a.2\n\n@[simp] theorem curry_uncurry (f : α → β → φ) : curry (uncurry f) = f :=\nrfl\n\n@[simp] theorem uncurry_curry (f : α × β → φ) : uncurry (curry f) = f :=\nfunext (λ ⟨a, b⟩ => rfl)\n\nprotected theorem left_inverse.id {g : β → α} {f : α → β} (h : left_inverse g f) : g ∘ f = id :=\nfunext h\n\nprotected theorem right_inverse.id {g : β → α} {f : α → β} (h : right_inverse g f) : f ∘ g = id :=\nfunext h\n\nend Function\n",
6666
"_type": "text"}]

test/playground/infoTree.lean.leanInk.expected

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,4 +11,4 @@
1111
"goals": [],
1212
"contents": "#print",
1313
"_type": "sentence"},
14-
{"contents": " xor\ninstance : Inhabited", "_type": "text"}]
14+
{"contents": " xor\ninstance : Inhabited Nat where\n\nmacro", "_type": "text"}]

test/test.sh

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -43,10 +43,10 @@ run_leanink () {
4343
# If the folder in which the file resides contains a lakefile we will use it to resolve any dependencies for the file
4444
if [[ -f "$directory/lakefile.lean" ]]; then
4545
echo "Running LeanInk with lakefile.lean - $file"
46-
(cd $directory && $LEANINK analyze $filename --lake lakefile.lean) || error "LeanInk failed - $file"
46+
(cd $directory && $LEANINK analyze $filename --lake lakefile.lean --verbose) || error "LeanInk failed - $file"
4747
else
4848
echo "Running LeanInk - $file"
49-
(cd $directory && $LEANINK analyze $filename) || error "LeanInk failed - $file"
49+
(cd $directory && $LEANINK analyze $filename --verbose) || error "LeanInk failed - $file"
5050
fi
5151
}
5252

test/theorem_proving/005.lean.leanInk.expected

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -33,4 +33,4 @@
3333
"goals": [],
3434
"contents": "#check",
3535
"_type": "sentence"},
36-
{"contents": "", "_type": "text"}]
36+
{"contents": " And", "_type": "text"}]

test/theorem_proving/007.lean.leanInk.expected

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -44,4 +44,4 @@
4444
{"messages": [], "goals": [], "contents": "exact hp", "_type": "sentence"},
4545
{"contents": "\n case left => ", "_type": "text"},
4646
{"messages": [], "goals": [], "contents": "exact hp", "_type": "sentence"},
47-
{"contents": "", "_type": "text"}]
47+
{"contents": "\n", "_type": "text"}]

0 commit comments

Comments
 (0)