Skip to content

Experiment: Pass tactic proof state using references. #922

Experiment: Pass tactic proof state using references.

Experiment: Pass tactic proof state using references. #922

Triggered via pull request September 11, 2025 03:05
Status Failure
Total duration 40m 39s
Artifacts 3

ci.yml

on: pull_request
Matrix: opam / build
Matrix: tests / ocaml-smoke
pulse  /  build-pulse-plugin
1m 48s
pulse / build-pulse-plugin
Fit to window
Zoom out
Zoom in

Annotations

6 errors, 60 warnings, and 7 notices
pulse / build-pulse-plugin
Process completed with exit code 2.
pulse / build-pulse-plugin: Pulse.Typing.Env.fsti#L228
(40) * Error 40 at /__w/FStar/FStar/pulse/src/checker/Pulse.Typing.Env.fsti(228,58-228,86): - Data constructor FStar.Tactics.Result.Failed not found
tests / tests
Process completed with exit code 2.
tests / tests
Diff failed for files /tests/error-messages/_output/Bug2899.fst.output and /tests/error-messages/Bug2899.fst.output.expected: --- Bug2899.fst.output.expected 2025-09-11 03:30:20.383637422 +0000 +++ _output/Bug2899.fst.output 2025-09-11 03:33:39.135511570 +0000 @@ -2,10 +2,9 @@ - Expected failure: - Tactic failed - Tactic got stuck! - - Reduction stopped at: - FStar.Stubs.Tactics.Result.Success (Prims.admit ()) "(((proofstate)))" + - Reduction stopped at: Prims.admit () - The term contains an `admit`, which will not reduce. Did you mean `tadmit()`? - - See also FStar.Tactics.Effect.fsti(200,48-200,58) + - See also FStar.Tactics.Effect.fsti(198,48-198,58) * Info at Bug2899.fst(10,12-10,18): - Expected failure: @@ -13,21 +12,22 @@ - Tactic got stuck! - Reduction stopped at: Prims.admit () - The term contains an `admit`, which will not reduce. Did you mean `tadmit()`? - - See also FStar.Tactics.Effect.fsti(200,48-200,58) + - See also FStar.Tactics.Effect.fsti(198,48-198,58) * Info at Bug2899.fst(13,12-13,18): - Expected failure: - Tactic failed - Tactic got stuck! - Reduction stopped at: - FStar.Stubs.Tactics.V2.Builtins.dump (Prims.admit ()) "(((proofstate)))" + FStar.Stubs.Tactics.V2.Builtins.dump (Prims.admit ()) + "(((ref proofstate)))" - The term contains an `admit`, which will not reduce. Did you mean `tadmit()`? - - See also FStar.Tactics.Effect.fsti(200,48-200,58) + - See also FStar.Tactics.Effect.fsti(198,48-198,58) * Info at Bug2899.fst(17,50-17,66): - Expected failure: - Tactic failed - Tactic got stuck! - - Reduction stopped at: reify (tac ()) "(((proofstate)))" - - See also FStar.Tactics.Effect.fsti(200,48-200,58) + - Reduction stopped at: reify (tac ()) "(((ref proofstate)))" + - See also FStar.Tactics.Effect.fsti(198,48-198,58)
tests / tests
Diff failed for files /tests/error-messages/_output/Bug2899.fst.json_output and /tests/error-messages/Bug2899.fst.json_output.expected: --- Bug2899.fst.json_output.expected 2025-09-11 03:30:20.383637422 +0000 +++ _output/Bug2899.fst.json_output 2025-09-11 03:33:38.359515591 +0000 @@ -1,4 +1,4 @@ -{"msg":["Expected failure:","Tactic failed","Tactic got stuck!","Reduction stopped at:\n FStar.Stubs.Tactics.Result.Success (Prims.admit ()) \"(((proofstate)))\"","The term contains an `admit`, which will not reduce. Did you mean `tadmit()`?"],"level":"Info","range":{"def":{"file_name":"FStar.Tactics.Effect.fsti","start_pos":{"line":200,"col":48},"end_pos":{"line":200,"col":58}},"use":{"file_name":"Bug2899.fst","start_pos":{"line":7,"col":12},"end_pos":{"line":7,"col":18}}},"number":170,"ctx":["While preprocessing VC with a tactic","While checking for top-level effects","While typechecking the top-level declaration `let test0`","While typechecking the top-level declaration `[@@expect_failure] let test0`"]} -{"msg":["Expected failure:","Tactic failed","Tactic got stuck!","Reduction stopped at: Prims.admit ()","The term contains an `admit`, which will not reduce. Did you mean `tadmit()`?"],"level":"Info","range":{"def":{"file_name":"FStar.Tactics.Effect.fsti","start_pos":{"line":200,"col":48},"end_pos":{"line":200,"col":58}},"use":{"file_name":"Bug2899.fst","start_pos":{"line":10,"col":12},"end_pos":{"line":10,"col":18}}},"number":170,"ctx":["While preprocessing VC with a tactic","While checking for top-level effects","While typechecking the top-level declaration `let test1`","While typechecking the top-level declaration `[@@expect_failure] let test1`"]} -{"msg":["Expected failure:","Tactic failed","Tactic got stuck!","Reduction stopped at:\n FStar.Stubs.Tactics.V2.Builtins.dump (Prims.admit ()) \"(((proofstate)))\"","The term contains an `admit`, which will not reduce. Did you mean `tadmit()`?"],"level":"Info","range":{"def":{"file_name":"FStar.Tactics.Effect.fsti","start_pos":{"line":200,"col":48},"end_pos":{"line":200,"col":58}},"use":{"file_name":"Bug2899.fst","start_pos":{"line":13,"col":12},"end_pos":{"line":13,"col":18}}},"number":170,"ctx":["While preprocessing VC with a tactic","While checking for top-level effects","While typechecking the top-level declaration `let test2`","While typechecking the top-level declaration `[@@expect_failure] let test2`"]} -{"msg":["Expected failure:","Tactic failed","Tactic got stuck!","Reduction stopped at: reify (tac ()) \"(((proofstate)))\"",""],"level":"Info","range":{"def":{"file_name":"FStar.Tactics.Effect.fsti","start_pos":{"line":200,"col":48},"end_pos":{"line":200,"col":58}},"use":{"file_name":"Bug2899.fst","start_pos":{"line":17,"col":50},"end_pos":{"line":17,"col":66}}},"number":170,"ctx":["While preprocessing VC with a tactic","While typechecking the top-level declaration `let eval_tactic`","While typechecking the top-level declaration `[@@expect_failure] let eval_tactic`"]} +{"msg":["Expected failure:","Tactic failed","Tactic got stuck!","Reduction stopped at: Prims.admit ()","The term contains an `admit`, which will not reduce. Did you mean `tadmit()`?"],"level":"Info","range":{"def":{"file_name":"FStar.Tactics.Effect.fsti","start_pos":{"line":198,"col":48},"end_pos":{"line":198,"col":58}},"use":{"file_name":"Bug2899.fst","start_pos":{"line":7,"col":12},"end_pos":{"line":7,"col":18}}},"number":170,"ctx":["While preprocessing VC with a tactic","While checking for top-level effects","While typechecking the top-level declaration `let test0`","While typechecking the top-level declaration `[@@expect_failure] let test0`"]} +{"msg":["Expected failure:","Tactic failed","Tactic got stuck!","Reduction stopped at: Prims.admit ()","The term contains an `admit`, which will not reduce. Did you mean `tadmit()`?"],"level":"Info","range":{"def":{"file_name":"FStar.Tactics.Effect.fsti","start_pos":{"line":198,"col":48},"end_pos":{"line":198,"col":58}},"use":{"file_name":"Bug2899.fst","start_pos":{"line":10,"col":12},"end_pos":{"line":10,"col":18}}},"number":170,"ctx":["While preprocessing VC
ciok
Process completed with exit code 1.
build / build: FStarC.Parser.ToDocument.fst#L1991
(328) * Warning 328 at /__w/FStar/FStar/FStar/src/parser/FStarC.Parser.ToDocument.fst(1991,4-1991,12): - Global binding 'FStarC.Parser.ToDocument.p_tmNoEq' is recursive but not used in its body
build / build: FStarC.Parser.ToDocument.fst#L1727
(328) * Warning 328 at /__w/FStar/FStar/FStar/src/parser/FStarC.Parser.ToDocument.fst(1727,4-1727,21): - Global binding 'FStarC.Parser.ToDocument.p_maybeFocusArrow' is recursive but not used in its body
build / build: FStarC.Parser.ToDocument.fst#L1095
(328) * Warning 328 at /__w/FStar/FStar/FStar/src/parser/FStarC.Parser.ToDocument.fst(1095,4-1095,24): - Global binding 'FStarC.Parser.ToDocument.p_disjunctivePattern' is recursive but not used in its body
build / build: FStarC.Parser.ToDocument.fst#L756
(328) * Warning 328 at /__w/FStar/FStar/FStar/src/parser/FStarC.Parser.ToDocument.fst(756,4-756,13): - Global binding 'FStarC.Parser.ToDocument.p_justSig' is recursive but not used in its body
build / build: FStarC.Parser.ToDocument.fst#L735
(328) * Warning 328 at /__w/FStar/FStar/FStar/src/parser/FStarC.Parser.ToDocument.fst(735,8-735,14): - Global binding 'FStarC.Parser.ToDocument.p_decl' is recursive but not used in its body
build / build: FStarC.Plugins.fst#L88
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/basic/FStarC.Plugins.fst(88,16-88,17): - The operator '@' has been resolved to FStar.List.Tot.append even though FStar.List.Tot is not in scope. Please add an 'open FStar.List.Tot' to stop relying on this deprecated, special treatment of '@'.
build / build: FStarC.Plugins.fst#L87
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/basic/FStarC.Plugins.fst(87,16-87,17): - The operator '@' has been resolved to FStar.List.Tot.append even though FStar.List.Tot is not in scope. Please add an 'open FStar.List.Tot' to stop relying on this deprecated, special treatment of '@'.
build / build: FStarC.Plugins.fst#L86
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/basic/FStarC.Plugins.fst(86,16-86,17): - The operator '@' has been resolved to FStar.List.Tot.append even though FStar.List.Tot is not in scope. Please add an 'open FStar.List.Tot' to stop relying on this deprecated, special treatment of '@'.
build / build: FStarC.Plugins.fst#L85
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/basic/FStarC.Plugins.fst(85,16-85,17): - The operator '@' has been resolved to FStar.List.Tot.append even though FStar.List.Tot is not in scope. Please add an 'open FStar.List.Tot' to stop relying on this deprecated, special treatment of '@'.
build / build: FStar.UInt.fsti#L436
(271) * Warning 271 at /__w/FStar/FStar/FStar/ulib/FStar.UInt.fsti(436,8-436,51): - Pattern uses these theory symbols or terms that should not be in an SMT pattern: Prims.op_Subtraction
pulse / build-pulse-plugin: Pulse.Syntax.Base.fst#L299
(290) * Warning 290 at /__w/FStar/FStar/pulse/src/checker/Pulse.Syntax.Base.fst(299,15-299,17): - In the decreases clause for this function, the SMT solver may not be able to prove that the types of b1 (bound in Pulse.Syntax.Base.fst(299,15-299,17)) and t1 (bound in Pulse.Syntax.Base.fst(173,20-173,22)) are equal. - The type of the first term is: Pulse.Syntax.Base.branch - The type of the second term is: Pulse.Syntax.Base.st_term - If the proof fails, try annotating these with the same type.
pulse / build-pulse-plugin: Pulse.Syntax.Base.fst#L304
(290) * Warning 290 at /__w/FStar/FStar/pulse/src/checker/Pulse.Syntax.Base.fst(304,14-304,16): - In the decreases clause for this function, the SMT solver may not be able to prove that the types of q1 (bound in Pulse.Syntax.Base.fst(304,14-304,16)) and t1 (bound in Pulse.Syntax.Base.fst(173,20-173,22)) are equal. - The type of the first term is: Pulse.Syntax.Base.qualifier - The type of the second term is: Pulse.Syntax.Base.st_term - If the proof fails, try annotating these with the same type.
pulse / build-pulse-plugin: Pulse.Syntax.Base.fst#L123
(290) * Warning 290 at /__w/FStar/FStar/pulse/src/checker/Pulse.Syntax.Base.fst(123,20-123,22): - In the decreases clause for this function, the SMT solver may not be able to prove that the types of p1 (bound in Pulse.Syntax.Base.fst(123,20-123,22)) and pb1 (bound in Pulse.Syntax.Base.fst(139,16-139,19)) are equal. - The type of the first term is: Pulse.Syntax.Base.pattern - The type of the second term is: Pulse.Syntax.Base.pattern & Prims.bool - If the proof fails, try annotating these with the same type.
pulse / build-pulse-plugin: Pulse.Syntax.Base.fst#L139
(290) * Warning 290 at /__w/FStar/FStar/pulse/src/checker/Pulse.Syntax.Base.fst(139,16-139,19): - In the decreases clause for this function, the SMT solver may not be able to prove that the types of pb1 (bound in Pulse.Syntax.Base.fst(139,16-139,19)) and p1 (bound in Pulse.Syntax.Base.fst(123,20-123,22)) are equal. - The type of the first term is: Pulse.Syntax.Base.pattern & Prims.bool - The type of the second term is: Pulse.Syntax.Base.pattern - If the proof fails, try annotating these with the same type.
pulse / build-pulse-plugin: PulseSyntaxExtension.Desugar.fst#L926
(328) * Warning 328 at /__w/FStar/FStar/pulse/src/syntax_extension/PulseSyntaxExtension.Desugar.fst(926,4-926,16): - Global binding 'PulseSyntaxExtension.Desugar.desugar_decl' is recursive but not used in its body
pulse / build-pulse-plugin: Pulse.Common.fst#L84
(337) * Warning 337 at /__w/FStar/FStar/pulse/src/checker/Pulse.Common.fst(84,11-84,12): - The operator '@' has been resolved to FStar.List.Tot.append even though FStar.List.Tot is not in scope. Please add an 'open FStar.List.Tot' to stop relying on this deprecated, special treatment of '@'.
pulse / build-pulse-plugin: PulseSyntaxExtension.Sugar.fst#L659
(337) * Warning 337 at /__w/FStar/FStar/pulse/src/syntax_extension/PulseSyntaxExtension.Sugar.fst(659,47-659,48): - The operator '@' has been resolved to FStar.List.Tot.append even though FStar.List.Tot is not in scope. Please add an 'open FStar.List.Tot' to stop relying on this deprecated, special treatment of '@'.
pulse / build-pulse-plugin: PulseSyntaxExtension.Sugar.fst#L658
(337) * Warning 337 at /__w/FStar/FStar/pulse/src/syntax_extension/PulseSyntaxExtension.Sugar.fst(658,47-658,48): - The operator '@' has been resolved to FStar.List.Tot.append even though FStar.List.Tot is not in scope. Please add an 'open FStar.List.Tot' to stop relying on this deprecated, special treatment of '@'.
pulse / build-pulse-plugin: PulseSyntaxExtension.Sugar.fst#L545
(328) * Warning 328 at /__w/FStar/FStar/pulse/src/syntax_extension/PulseSyntaxExtension.Sugar.fst(545,8-545,17): - Global binding 'PulseSyntaxExtension.Sugar.scan_decl' is recursive but not used in its body
pulse / build-pulse-plugin: PulseSyntaxExtension.Sugar.fst#L397
(328) * Warning 328 at /__w/FStar/FStar/pulse/src/syntax_extension/PulseSyntaxExtension.Sugar.fst(397,8-397,15): - Global binding 'PulseSyntaxExtension.Sugar.eq_decl' is recursive but not used in its body
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.MST.fst#L247
(352) * Warning 352 at /home/runner/work/FStar/FStar/fstar/ulib/experimental/FStar.MST.fst(247,42-247,60): - Combinator FStar.MSTTotal.MSTATETOT ~> FStar.MST.MSTATE is not a substitutive indexed effect combinator, it is better to make it one if possible for better performance and ease of use
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.MST.fst#L222
(330) * Warning 330 at /home/runner/work/FStar/FStar/fstar/ulib/experimental/FStar.MST.fst(222,43-222,55): - Polymonadic binds ((DIV, MSTATE) |> MSTATE) in this case) is an experimental feature;it is subject to some redesign in the future. Please keep us informed (on github etc.) about how you are using it
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.MST.fst#L222
(330) * Warning 330 at /home/runner/work/FStar/FStar/fstar/ulib/experimental/FStar.MST.fst(222,43-222,55): - Polymonadic binds ((DIV, MSTATE) |> MSTATE) in this case) is an experimental feature;it is subject to some redesign in the future. Please keep us informed (on github etc.) about how you are using it
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.UInt.fsti#L436
(271) * Warning 271 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fst(293,8-293,25): - Pattern uses these theory symbols or terms that should not be in an SMT pattern: Prims.op_Subtraction - See also /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fsti(436,8-436,51)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.UInt.fsti#L436
(271) * Warning 271 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fsti(436,8-436,51): - Pattern uses these theory symbols or terms that should not be in an SMT pattern: Prims.op_Subtraction
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): dummy#L0
(242) * Warning 242 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(122,0-131,33): - Definitions of inner let-rec aux and its enclosing top-level letbinding are not encoded to the solver, you will only be able to reason with their types - Also see: /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(126,12-126,15)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): dummy#L0
(242) * Warning 242 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(122,0-131,33): - Definitions of inner let-rec aux and its enclosing top-level letbinding are not encoded to the solver, you will only be able to reason with their types - Also see: /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(86,12-86,15)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.GhostSet.fst#L23
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.GhostSet.fst(23,4-23,7): - Values of type `set` cannot be erased during extraction, but the `must_erase_for_extraction` attribute claims that it can. - Please remove the attribute.
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.UInt.fsti#L436
(271) * Warning 271 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fsti(436,8-436,51): - Pattern uses these theory symbols or terms that should not be in an SMT pattern: Prims.op_Subtraction
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest): FStar.TSet.fst#L26
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.TSet.fst(26,4-26,7): - Values of type `set` cannot be erased during extraction, but the `must_erase_for_extraction` attribute claims that it can. - Please remove the attribute.
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): FStar.MST.fst#L222
(330) * Warning 330 at /home/runner/work/FStar/FStar/fstar/ulib/experimental/FStar.MST.fst(222,43-222,55): - Polymonadic binds ((DIV, MSTATE) |> MSTATE) in this case) is an experimental feature;it is subject to some redesign in the future. Please keep us informed (on github etc.) about how you are using it
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): dummy#L0
(242) * Warning 242 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.LexicographicOrdering.fsti(187,0-194,59): - Definitions of inner let-rec get_acc and its enclosing top-level letbinding are not encoded to the solver, you will only be able to reason with their types - Also see: /home/runner/work/FStar/FStar/fstar/ulib/FStar.LexicographicOrdering.fst(124,10-124,17)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): dummy#L0
(242) * Warning 242 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.LexicographicOrdering.fsti(187,0-194,59): - Definitions of inner let-rec lex_t_wf_aux_y and its enclosing top-level letbinding are not encoded to the solver, you will only be able to reason with their types - Also see: /home/runner/work/FStar/FStar/fstar/ulib/FStar.LexicographicOrdering.fst(75,14-75,28)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): dummy#L0
(242) * Warning 242 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(122,0-131,33): - Definitions of inner let-rec aux and its enclosing top-level letbinding are not encoded to the solver, you will only be able to reason with their types - Also see: /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(126,12-126,15)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): dummy#L0
(242) * Warning 242 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(122,0-131,33): - Definitions of inner let-rec aux and its enclosing top-level letbinding are not encoded to the solver, you will only be able to reason with their types - Also see: /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFounded.fst(86,12-86,15)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): FStar.GhostSet.fst#L23
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.GhostSet.fst(23,4-23,7): - Values of type `set` cannot be erased during extraction, but the `must_erase_for_extraction` attribute claims that it can. - Please remove the attribute.
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): FStar.UInt.fsti#L436
(271) * Warning 271 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fst(293,8-293,25): - Pattern uses these theory symbols or terms that should not be in an SMT pattern: Prims.op_Subtraction - See also /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fsti(436,8-436,51)
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): FStar.UInt.fsti#L436
(271) * Warning 271 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fsti(436,8-436,51): - Pattern uses these theory symbols or terms that should not be in an SMT pattern: Prims.op_Subtraction
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): FStar.UInt.fsti#L436
(271) * Warning 271 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.UInt.fsti(436,8-436,51): - Pattern uses these theory symbols or terms that should not be in an SMT pattern: Prims.op_Subtraction
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-24.04): FStar.TSet.fst#L26
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.TSet.fst(26,4-26,7): - Values of type `set` cannot be erased during extraction, but the `must_erase_for_extraction` attribute claims that it can. - Please remove the attribute.
tests / stage3: FStar.FiniteMap.Base.fst#L90
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteMap.Base.fst(90,4-90,9): - Parameter 0 of items is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.FiniteMap.Base.fst#L83
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteMap.Base.fst(83,4-83,10): - Parameter 0 of values is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.FiniteSet.Base.fst#L151
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteSet.Base.fst(151,4-151,12): - Parameter 0 of disjoint is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.FiniteSet.Base.fst#L144
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteSet.Base.fst(144,4-144,9): - Parameter 0 of equal is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.FiniteSet.Base.fst#L137
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteSet.Base.fst(137,4-137,10): - Parameter 0 of subset is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.FiniteSet.Base.fst#L151
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteSet.Base.fst(151,4-151,12): - Parameter 0 of disjoint is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.FiniteSet.Base.fst#L144
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteSet.Base.fst(144,4-144,9): - Parameter 0 of equal is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.FiniteSet.Base.fst#L137
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteSet.Base.fst(137,4-137,10): - Parameter 0 of subset is unused and must be eliminated for F#; add `[@@ remove_unused_type_parameters [0; ...]]` to the interface signature. - This type definition is being dropped
tests / stage3: FStar.Pervasives.fsti#L55
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.Monotonic.Witnessed.fsti(34,4-34,33): - Expected parameter 'state of witnessed to be unused in its definition and eliminated - See also /__w/FStar/FStar/FStar/ulib/FStar.Pervasives.fsti(55,0-55,56)
tests / stage3: FStar.Pervasives.fsti#L642
(345) * Warning 345 at /__w/FStar/FStar/FStar/ulib/FStar.Pervasives.fsti(642,66-642,67): - Inserted an unsafe type coercion in generated code from unit -> 'a -> 'a to unit -> 'a -> 'b. - This may be unsound in F#. - See also /__w/FStar/FStar/FStar/ulib/FStar.Pervasives.fsti(642,55-642,56)
tests / tests: dummy#L0
(274) * Warning 274: - Implicitly opening namespace 'fstar.list.' shadows module 'pure' in file "Pure.fst". - Rename "Pure.fst" to avoid conflicts.
tests / tests: Hello.fst#L5
(272) * Warning 272 at Hello.fst(5,0-5,28): - Top-level let-bindings must be total; this term may have effects
tests / tests: dummy#L0
(274) * Warning 274: - Implicitly opening namespace 'fstar.' shadows module 'uint32' in file "UInt32.fsti, UInt32.fst". - Rename "UInt32.fsti, UInt32.fst" to avoid conflicts.
tests / tests: dummy#L0
(361) * Warning 361 at AlexOpaque.fst(103,0-125,5): - Some #push-options have not been popped. Current depth is 2.
tests / tests: Test.fst#L21
(272) * Warning 272 at Test.fst(21,0-21,31): - Top-level let-bindings must be total; this term may have effects
tests / tests: dummy#L0
(274) * Warning 274: - Implicitly opening namespace 'fstar.' shadows module 'uint32' in file "UInt32.fsti, UInt32.fst". - Rename "UInt32.fsti, UInt32.fst" to avoid conflicts.
tests / tests: Hello.fst#L5
(272) * Warning 272 at Hello.fst(5,0-5,34): - Top-level let-bindings must be total; this term may have effects
tests / tests: dummy#L0
(274) * Warning 274: - Implicitly opening namespace 'fstar.tactics.' shadows module 'typeclasses' in file "Typeclasses.fst". - Rename "Typeclasses.fst" to avoid conflicts.
tests / tests: dummy#L0
(274) * Warning 274: - Implicitly opening namespace 'fstar.list.' shadows module 'pure' in file "Pure.fst". - Rename "Pure.fst" to avoid conflicts.
tests / tests: dummy#L0
(274) * Warning 274: - Implicitly opening namespace 'fstar.' shadows module 'uint32' in file "UInt32.fsti, UInt32.fst". - Rename "UInt32.fsti, UInt32.fst" to avoid conflicts.
tests / perf-canaries: DEFS_6400#L0
time = 1.08
tests / perf-canaries: DEFS_3200#L0
time = 0.58
tests / perf-canaries: DEFS_1600#L0
time = 0.36
tests / perf-canaries: DEFS_800#L0
time = 0.23
tests / perf-canaries: DEFS_400#L0
time = 0.18
tests / perf-canaries: DEFS_200#L0
time = 0.15
tests / perf-canaries: DEFS_100#L0
time = 0.14

Artifacts

Produced during runtime
Name Size Digest
fstar-repo
192 MB
sha256:21db6234080f4d5fd059b537e65b29520235b0af624d03a3626fe5ef0d89224d
fstar-src.tar.gz
4.16 MB
sha256:2c662ec3d96654a18cec86f357f65ae3641ee1143881bfe5b9dc289803354c47
fstar.tar.gz
133 MB
sha256:c5f1f478ed0d4e12588138da4a39fb24a84b2b0a0f7789a734aa6001a2452d1b