Skip to content

Commit d8fe6c0

Browse files
committed
fix imports and tests
1 parent b55e66e commit d8fe6c0

8 files changed

+14
-74
lines changed

REPL/Frontend.lean

-1
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Scott Morrison
55
-/
66
import Lean.Elab.Frontend
7-
import REPL.Util.TermUnsafe
87

98
open Lean Elab
109

REPL/Main.lean

-1
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,6 @@ Authors: Scott Morrison
66
import REPL.JSON
77
import REPL.Frontend
88
import REPL.Util.Path
9-
import REPL.Util.TermUnsafe
109
import REPL.Lean.ContextInfo
1110
import REPL.Lean.Environment
1211
import REPL.Lean.InfoTree

REPL/Snapshots.lean

+1
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Scott Morrison
55
-/
66
import Lean.Replay
7+
import Lean.Elab.Command
78
import REPL.Util.Pickle
89

910
open Lean Elab

REPL/Util/Pickle.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2023 Mario Carneiro. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mario Carneiro
55
-/
6-
import REPL.Util.TermUnsafe
6+
import Lean.Environment
77

88
/-!
99
# Pickling and unpickling objects

REPL/Util/TermUnsafe.lean

-63
This file was deleted.

test/by_cases.expected.out

+5-5
Original file line numberDiff line numberDiff line change
@@ -12,14 +12,14 @@
1212

1313
{"proofState": 1,
1414
"goals":
15-
["case inl\nx : Int\nh : x < 0\n⊢ x = x",
16-
"case inr\nx : Int\nh : ¬x < 0\n⊢ x = x"]}
15+
["case pos\nx : Int\nh : x < 0\n⊢ x = x",
16+
"case neg\nx : Int\nh : ¬x < 0\n⊢ x = x"]}
1717

18-
{"proofState": 2, "goals": ["case inr\nx : Int\nh : ¬x < 0\n⊢ x = x"]}
18+
{"proofState": 2, "goals": ["case neg\nx : Int\nh : ¬x < 0\n⊢ x = x"]}
1919

2020
{"sorries":
21-
[{"proofState": 3, "goal": "case inl\nx : Int\nh : x < 0\n⊢ x = x"},
22-
{"proofState": 4, "goal": "case inr\nx : Int\nh : ¬x < 0\n⊢ x = x"}],
21+
[{"proofState": 3, "goal": "case pos\nx : Int\nh : x < 0\n⊢ x = x"},
22+
{"proofState": 4, "goal": "case neg\nx : Int\nh : ¬x < 0\n⊢ x = x"}],
2323
"proofState": 5,
2424
"goals": []}
2525

test/by_cases.in

+1-1
Original file line numberDiff line numberDiff line change
@@ -2,7 +2,7 @@
22

33
{"proofState" : 0, "tactic": "by_cases h : x < 0"}
44

5-
{"proofState" : 1, "tactic": "case inl => rfl"}
5+
{"proofState" : 1, "tactic": "case pos => rfl"}
66

77
{"proofState" : 1, "tactic": "all_goals sorry"}
88

test/name_generator.expected.out

+6-2
Original file line numberDiff line numberDiff line change
@@ -23,11 +23,15 @@
2323
"proofState": 5,
2424
"goals": []}
2525

26-
{"traces": ["[Meta.Tactic.simp.rewrite] h0:1000, x > 0 ==> True"],
26+
{"traces":
27+
["[Meta.Tactic.simp.rewrite] @gt_iff_lt:1000, x > 0 ==> 0 < x",
28+
"[Meta.Tactic.simp.rewrite] h0:1000, 0 < x ==> True"],
2729
"proofState": 6,
2830
"goals": []}
2931

30-
{"traces": ["[Meta.Tactic.simp.rewrite] h0:1000, x > 0 ==> True"],
32+
{"traces":
33+
["[Meta.Tactic.simp.rewrite] @gt_iff_lt:1000, x > 0 ==> 0 < x",
34+
"[Meta.Tactic.simp.rewrite] h0:1000, 0 < x ==> True"],
3135
"proofState": 7,
3236
"goals": []}
3337

0 commit comments

Comments
 (0)