Skip to content

Commit

Permalink
test: update test output following stage0 update
Browse files Browse the repository at this point in the history
this is a consequenc of #4807 that only shows up once that change made
it to stage0, it seem.
  • Loading branch information
nomeata committed Jul 23, 2024
1 parent ee6737a commit 5d522c0
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 7 deletions.
4 changes: 2 additions & 2 deletions tests/lean/ppMotives.lean.expected.out
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ fun x x_1 =>
(fun x f x_2 =>
(match x_2, x with
| a, Nat.zero => fun x => a
| a, b.succ => fun x => (x.fst.fst a).succ)
| a, b.succ => fun x => (x.1 a).succ)
f)
x
protected def Nat.add : Nat → Nat → Nat :=
Expand All @@ -13,7 +13,7 @@ fun x x_1 =>
(fun x f x_2 =>
(match (motive := Nat → (x : Nat) → Nat.below (motive := fun x => Nat → Nat) x → Nat) x_2, x with
| a, Nat.zero => fun x => a
| a, b.succ => fun x => (x.fst.fst a).succ)
| a, b.succ => fun x => (x.1 a).succ)
f)
x
theorem ex.{u} : ∀ {α β : Sort u} (h : α = β) (a : α), HEq (cast h a) a :=
Expand Down
6 changes: 2 additions & 4 deletions tests/lean/run/diagRec.lean
Original file line number Diff line number Diff line change
Expand Up @@ -12,11 +12,9 @@ info: [reduction] unfolded declarations (max: 407, num: 3):
Or.rec ↦ 144
Acc.rec ↦ 108[reduction] unfolded reducible declarations (max: 352, num: 3):
Acc.rec ↦ 108[reduction] unfolded reducible declarations (max: 352, num: 2):
Nat.casesOn ↦ 352
Or.casesOn ↦ 144
PProd.fst ↦ 126use `set_option diagnostics.threshold <num>` to control threshold for reporting counters
Or.casesOn ↦ 144use `set_option diagnostics.threshold <num>` to control threshold for reporting counters
-/
#guard_msgs in
set_option diagnostics true in
Expand Down
2 changes: 1 addition & 1 deletion tests/lean/unusedLet.lean.expected.out
Original file line number Diff line number Diff line change
Expand Up @@ -8,5 +8,5 @@ fun x =>
| 0 => fun x => 1
| n.succ => fun x =>
let y := 42;
2 * x.1.1)
2 * x.1)
f

0 comments on commit 5d522c0

Please sign in to comment.