Skip to content

Commit

Permalink
chore: stop running compiler twice during tests (#6321)
Browse files Browse the repository at this point in the history
The reason given for this in the comment seemingly no longer holds.

Co-authored-by: Cameron Zwarich <cameron@lean-fro.org>
  • Loading branch information
zwarich and zwarich authored Dec 13, 2024
1 parent 7530fd6 commit aa00725
Show file tree
Hide file tree
Showing 5 changed files with 0 additions and 15 deletions.
3 changes: 0 additions & 3 deletions tests/lean/run/CompilerCSE.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,9 +6,6 @@ import Lean.Elab.Command
open Lean
open Lean.Compiler.LCNF

-- Run compilation twice to avoid the output caused by the inliner
run_meta Compiler.compile #[``Lean.Meta.synthInstance, ``Lean.Elab.Term.Do.elabDo]

@[cpass]
def cseFixTest : PassInstaller := Testing.assertIsAtFixPoint |>.install `cse `cseFix

Expand Down
3 changes: 0 additions & 3 deletions tests/lean/run/CompilerFindJoinPoints.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,9 +6,6 @@ import Lean.Elab.Command
open Lean
open Lean.Compiler.LCNF

-- Run compilation twice to avoid the output caused by the inliner
run_meta Compiler.compile #[``Lean.Meta.synthInstance, ``Lean.Elab.Term.Do.elabDo, ``Lean.MetavarContext.MkBinding.collectForwardDeps]

@[cpass]
def findJoinPointFixTest : PassInstaller := Testing.assertIsAtFixPoint |>.install `findJoinPoints `findJoinPointsFix

Expand Down
3 changes: 0 additions & 3 deletions tests/lean/run/CompilerFloatLetIn.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,9 +6,6 @@ import Lean.Elab.Command
open Lean
open Lean.Compiler.LCNF

-- Run compilation twice to avoid the output caused by the inliner
run_meta Compiler.compile #[``Lean.Meta.synthInstance, ``Lean.Elab.Term.Do.elabDo]

-- #eval fails if we uncomment this pass after I added a `floatLetIn` pass at the mono phase
-- @[cpass]
-- def floatLetInFixTest : PassInstaller := Testing.assertIsAtFixPoint |>.install `floatLetIn `floatLetInFix
Expand Down
3 changes: 0 additions & 3 deletions tests/lean/run/CompilerPullInstances.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,9 +6,6 @@ import Lean.Elab.Command
open Lean
open Lean.Compiler.LCNF

-- Run compilation twice to avoid the output caused by the inliner
run_meta Compiler.compile #[``Lean.Meta.synthInstance, ``Lean.Elab.Term.Do.elabDo]

@[cpass]
def pullInstancesFixTest : PassInstaller := Testing.assertIsAtFixPoint |>.install `pullInstances `pullInstancesFix

Expand Down
3 changes: 0 additions & 3 deletions tests/lean/run/CompilerSimp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,9 +6,6 @@ import Lean.Elab.Command
open Lean
open Lean.Compiler.LCNF

-- Run compilation twice to avoid the output caused by the inliner
run_meta Compiler.compile #[``Lean.Meta.synthInstance, ``Lean.Elab.Term.Do.elabDo]

@[cpass]
def simpFixTest : PassInstaller := Testing.assertIsAtFixPoint |>.install `simp `simpFix

Expand Down

0 comments on commit aa00725

Please sign in to comment.