Skip to content

Commit

Permalink
chore: fix tests
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura committed Jun 17, 2024
1 parent 7661c88 commit d4c442a
Show file tree
Hide file tree
Showing 8 changed files with 31 additions and 27 deletions.
8 changes: 4 additions & 4 deletions tests/lean/1682.lean.expected.out
Original file line number Diff line number Diff line change
@@ -1,21 +1,21 @@
1682.lean:1:25-2:17: error: unsolved goals
case a
p : Sort ?u
p : Sort u_1
q r : Prop
⊢ p → q

case b
p : Sort ?u
p : Sort u_1
q r : Prop
⊢ r
1682.lean:4:25-5:26: error: unsolved goals
case a
p : Sort ?u
p : Sort u_1
q r : Prop
h : p
⊢ q

case b
p : Sort ?u
p : Sort u_1
q r : Prop
⊢ r
4 changes: 2 additions & 2 deletions tests/lean/813.lean.expected.out
Original file line number Diff line number Diff line change
@@ -1,12 +1,12 @@
p : Nat → Prop
h : p 1
⊢ p 1
α : Sort ?u
α : Sort u_1
a : α
p : α → Prop
h : p a
⊢ p a
α : Sort ?u
α : Sort u_1
a : α
f : α → α
p : α → Prop
Expand Down
2 changes: 1 addition & 1 deletion tests/lean/autoPPExplicit.lean.expected.out
Original file line number Diff line number Diff line change
Expand Up @@ -5,4 +5,4 @@ argument
has type
Prop : Type
but is expected to have type
α : Sort ?u
α : Sort u_1
12 changes: 6 additions & 6 deletions tests/lean/interactive/plainGoal.lean.expected.out
Original file line number Diff line number Diff line change
Expand Up @@ -82,9 +82,9 @@
{"textDocument": {"uri": "file:///plainGoal.lean"},
"position": {"line": 55, "character": 3}}
{"rendered":
"```lean\nα : Sort ?u\np : α → Prop\na b : α\ninst✝ : DecidablePred p\nh : ∀ {p : α → Prop} [inst : DecidablePred p], p a → p b\n⊢ p a\n```",
"```lean\nα : Sort u_1\np : α → Prop\na b : α\ninst✝ : DecidablePred p\nh : ∀ {p : α → Prop} [inst : DecidablePred p], p a → p b\n⊢ p a\n```",
"goals":
["α : Sort ?u\np : α → Prop\na b : α\ninst✝ : DecidablePred p\nh : ∀ {p : α → Prop} [inst : DecidablePred p], p a → p b\n⊢ p a"]}
["α : Sort u_1\np : α → Prop\na b : α\ninst✝ : DecidablePred p\nh : ∀ {p : α → Prop} [inst : DecidablePred p], p a → p b\n⊢ p a"]}
{"textDocument": {"uri": "file:///plainGoal.lean"},
"position": {"line": 61, "character": 3}}
{"rendered": "```lean\ncase left\n⊢ True\n```", "goals": ["case left\n⊢ True"]}
Expand All @@ -110,15 +110,15 @@
{"textDocument": {"uri": "file:///plainGoal.lean"},
"position": {"line": 82, "character": 53}}
{"rendered":
"```lean\ncase nil\nα : Type ?u\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)\n```",
"```lean\ncase nil\nα : Type u_1\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)\n```",
"goals":
["case nil\nα : Type ?u\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)"]}
["case nil\nα : Type u_1\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)"]}
{"textDocument": {"uri": "file:///plainGoal.lean"},
"position": {"line": 82, "character": 54}}
{"rendered":
"```lean\ncase nil\nα : Type ?u\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)\n```",
"```lean\ncase nil\nα : Type u_1\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)\n```",
"goals":
["case nil\nα : Type ?u\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)"]}
["case nil\nα : Type u_1\nbs cs : List α\n⊢ [] ++ bs ++ cs = [] ++ (bs ++ cs)"]}
{"textDocument": {"uri": "file:///plainGoal.lean"},
"position": {"line": 86, "character": 38}}
{"rendered": "no goals", "goals": []}
Expand Down
2 changes: 1 addition & 1 deletion tests/lean/ppProofs.lean.expected.out
Original file line number Diff line number Diff line change
Expand Up @@ -13,7 +13,7 @@ a : α
h : α = β
⊢ ⋯ ▸ a = b
ppProofs.lean:10:50-10:98: error: unsolved goals
α β : Sort ?u
α β : Sort u_1
b : β
a : α
h : α = β
Expand Down
8 changes: 6 additions & 2 deletions tests/lean/run/1575.lean
Original file line number Diff line number Diff line change
@@ -1,2 +1,6 @@
example [Subsingleton α] (p : α → Prop) : Subsingleton (Subtype p) :=
⟨fun ⟨x, _⟩ ⟨y, _⟩ => Subsingleton.elim x y ▸ sorry
example [Subsingleton α] (p : α → Prop) : Subsingleton (Subtype p) := by
constructor
intro ⟨x, _⟩ ⟨y, _⟩
have := Subsingleton.elim x y
subst this
rfl
6 changes: 3 additions & 3 deletions tests/lean/run/multiTargetCasesInductionIssue.lean
Original file line number Diff line number Diff line change
Expand Up @@ -24,7 +24,7 @@ def Vec.casesOn
| ⟨as, h⟩ => go n as h

/--
info: α : Type _
info: α : Type u_1
n✝ : Nat
a✝ : α
as✝ : Vec α n✝
Expand All @@ -43,7 +43,7 @@ example (n : Nat) (a : α) (as : Vec α n) : Vec.cons a (Vec.cons a as) = Vec.co
constructor

/--
info: α : Type _
info: α : Type u_1
n✝ : Nat
a✝ : α
as✝ : Vec α n✝
Expand All @@ -62,7 +62,7 @@ example (n : Nat) (a : α) (as : Vec α n) : Vec.cons a (Vec.cons a as) = Vec.co
constructor

/--
info: α : Type _
info: α : Type u_1
n : Nat
a : α
as : Vec α n
Expand Down
16 changes: 8 additions & 8 deletions tests/lean/rwEqThms.lean.expected.out
Original file line number Diff line number Diff line change
@@ -1,41 +1,41 @@
α : Type ?u
α : Type u_1
a : α
as bs : List α
h : bs = a :: as
⊢ (?head :: as).length = bs.length

case head
α : Type ?u
α : Type u_1
a : α
as bs : List α
h : bs = a :: as
⊢ α
α : Type ?u
α : Type u_1
b a : α
as bs : List α
h : as = bs
⊢ as.length + 1 + 1 = bs.length + 2
α : Type ?u
α : Type u_1
b a : α
as bs : List α
h : as = bs
⊢ as.length + 1 + 1 = (b :: bs).length + 1
α : Type ?u
α : Type u_1
b a : α
as bs : List α
h : as = bs
⊢ as.length + 1 + 1 = bs.length + 1 + 1
α : Type ?u
α : Type u_1
b a : α
as bs : List α
h : as = bs
⊢ id (a :: b :: as).length = (b :: bs).length + 1
α : Type ?u
α : Type u_1
b a : α
as bs : List α
h : as = bs
⊢ (a :: b :: as).length = (b :: bs).length + 1
α : Type ?u
α : Type u_1
b a : α
as bs : List α
h : as = bs
Expand Down

0 comments on commit d4c442a

Please sign in to comment.