Detecting GITHUB_ENV and autoprinting github messages #113
ci.yml
on: pull_request
build
/
build
19m 59s
nix
/
fstar-nix
19m 14s
stale-hints
/
check_stale_hints
9s
Matrix: tests / binary-smoke
Matrix: tests / ocaml-smoke
tests
/
check-stage3
6m 14s
tests
/
test-local
15m 53s
tests
/
perf-canaries
24s
ciok
0s
Annotations
67 warnings and 7 notices
stale-hints / check_stale_hints
ubuntu-latest pipelines will use ubuntu-24.04 soon. For more details, see https://github.com/actions/runner-images/issues/10636
|
nix / fstar-nix
ubuntu-latest pipelines will use ubuntu-24.04 soon. For more details, see https://github.com/actions/runner-images/issues/10636
|
build / build
ubuntu-latest pipelines will use ubuntu-24.04 soon. For more details, see https://github.com/actions/runner-images/issues/10636
|
build / build:
FStar/ulib/FStar.UInt.fsti#L435
(271) * Warning 271 at /__w/FStar/FStar/FStar/ulib/FStar.UInt.fsti(435,8-435,51):
- Pattern uses these theory symbols or terms that should not be in an SMT
pattern:
Prims.op_Subtraction
|
build / build:
FStar/ulib/FStar.UInt.fsti#L435
(271) * Warning 271 at /__w/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 /__w/FStar/FStar/FStar/ulib/FStar.UInt.fsti(435,8-435,51)
|
build / build:
FStar/ulib/FStar.UInt.fsti#L435
(271) * Warning 271 at /__w/FStar/FStar/FStar/ulib/FStar.UInt.fsti(435,8-435,51):
- Pattern uses these theory symbols or terms that should not be in an SMT
pattern:
Prims.op_Subtraction
|
build / build:
FStar/ulib/FStar.Stubs.Tactics.V2.Builtins.fsti#L446
(288) * Warning 288 at /__w/FStar/FStar/FStar/ulib/FStar.Reflection.V2.Arith.fst(116,20-116,31):
- FStar.Stubs.Tactics.V2.Builtins.term_eq_old is deprecated
- Use Reflection.term_eq instead
- See also /__w/FStar/FStar/FStar/ulib/FStar.Stubs.Tactics.V2.Builtins.fsti(446,0-446,42)
|
build / build:
FStar/ulib/FStar.UInt.fsti#L435
(271) * Warning 271 at /__w/FStar/FStar/FStar/ulib/FStar.UInt.fsti(435,8-435,51):
- Pattern uses these theory symbols or terms that should not be in an SMT
pattern:
Prims.op_Subtraction
|
build / build:
FStar/src/data/FStarC.Compiler.RBSet.fst#L105
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/data/FStarC.Compiler.RBSet.fst(105,30-105,31):
- 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/src/data/FStarC.Compiler.RBSet.fst#L105
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/data/FStarC.Compiler.RBSet.fst(105,36-105,37):
- 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/src/basic/FStarC.Compiler.Plugins.fst#L86
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/basic/FStarC.Compiler.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:
FStar/src/basic/FStarC.Compiler.Plugins.fst#L87
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/basic/FStarC.Compiler.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:
FStar/src/basic/FStarC.Compiler.Plugins.fst#L88
(337) * Warning 337 at /__w/FStar/FStar/FStar/src/basic/FStarC.Compiler.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 '@'.
|
tests / check-stage3
ubuntu-latest pipelines will use ubuntu-24.04 soon. For more details, see https://github.com/actions/runner-images/issues/10636
|
tests / check-stage3:
FStar/ulib/FStar.Pervasives.fsti#L1218
(345) * Warning 345 at /__w/FStar/FStar/FStar/ulib/FStar.Pervasives.fsti(1218,66-1218,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(1218,55-1218,56)
|
tests / check-stage3:
FStar/ulib/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 / check-stage3:
FStar/ulib/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 / check-stage3:
FStar/ulib/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 / check-stage3:
FStar/ulib/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 / check-stage3:
dummy#L1
(345) * Warning 345:
- Inserted an unsafe type coercion in generated code from some_ref -> (obj, obj) mreference to some_ref -> (unit, unit) mreference; this may be unsound in F#
|
tests / check-stage3:
FStar/ulib/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 / check-stage3:
FStar/ulib/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 / check-stage3:
FStar/ulib/FStar.FiniteMap.Base.fst#L138
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteMap.Base.fst(138,4-138,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 / check-stage3:
FStar/ulib/FStar.FiniteMap.Base.fst#L145
(344) * Warning 344 at /__w/FStar/FStar/FStar/ulib/FStar.FiniteMap.Base.fst(145,4-145,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 / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest)
ubuntu-latest pipelines will use ubuntu-24.04 soon. For more details, see https://github.com/actions/runner-images/issues/10636
|
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-latest):
dummy#L1
(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):
dummy#L1
(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):
fstar/ulib/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/ulib/FStar.TSet.fst#L28
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.TSet.fst(28,4-28,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/ulib/FStar.GSet.fst#L23
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.GSet.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):
dummy#L1
(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-latest):
dummy#L1
(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-latest):
fstar/ulib/experimental/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/ulib/experimental/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/ulib/FStar.WellFoundedRelation.fst#L152
(290) * Warning 290 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46):
- In the decreases clause for this function, the SMT solver may not be able to
prove that the types of
wfr_a.decreaser (FStar.Pervasives.dfst xy)
(bound in
/home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46))
and
wfr_a.decreaser (FStar.Pervasives.dfst xy)
(bound in
/home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46))
are equal.
- The type of the first term is:
FStar.WellFoundedRelation.acc_classical wfr_a.relation
(FStar.Pervasives.dfst xy)
- The type of the second term is:
FStar.WellFoundedRelation.acc_classical wfr_a.relation
(FStar.Pervasives.dfst xy)
- If the proof fails, try annotating these with the same type.
|
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-22.04):
dummy#L1
(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-22.04):
dummy#L1
(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-22.04):
fstar/ulib/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-22.04):
fstar/ulib/FStar.TSet.fst#L28
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.TSet.fst(28,4-28,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-22.04):
fstar/ulib/FStar.GSet.fst#L23
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.GSet.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-22.04):
dummy#L1
(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-22.04):
dummy#L1
(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-22.04):
fstar/ulib/experimental/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-22.04):
fstar/ulib/experimental/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-22.04):
fstar/ulib/FStar.WellFoundedRelation.fst#L152
(290) * Warning 290 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46):
- In the decreases clause for this function, the SMT solver may not be able to
prove that the types of
wfr_a.decreaser (FStar.Pervasives.dfst xy)
(bound in
/home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46))
and
wfr_a.decreaser (FStar.Pervasives.dfst xy)
(bound in
/home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46))
are equal.
- The type of the first term is:
FStar.WellFoundedRelation.acc_classical wfr_a.relation
(FStar.Pervasives.dfst xy)
- The type of the second term is:
FStar.WellFoundedRelation.acc_classical wfr_a.relation
(FStar.Pervasives.dfst xy)
- If the proof fails, try annotating these with the same type.
|
tests / ocaml-smoke (fstar-src.tar.gz, ubuntu-20.04):
dummy#L1
(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-20.04):
dummy#L1
(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-20.04):
fstar/ulib/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-20.04):
fstar/ulib/FStar.GSet.fst#L23
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.GSet.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-20.04):
dummy#L1
(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-20.04):
dummy#L1
(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-20.04):
fstar/ulib/experimental/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-20.04):
fstar/ulib/experimental/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-20.04):
fstar/ulib/FStar.TSet.fst#L28
(318) * Warning 318 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.TSet.fst(28,4-28,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-20.04):
fstar/ulib/FStar.WellFoundedRelation.fst#L152
(290) * Warning 290 at /home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46):
- In the decreases clause for this function, the SMT solver may not be able to
prove that the types of
wfr_a.decreaser (FStar.Pervasives.dfst xy)
(bound in
/home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46))
and
wfr_a.decreaser (FStar.Pervasives.dfst xy)
(bound in
/home/runner/work/FStar/FStar/fstar/ulib/FStar.WellFoundedRelation.fst(152,21-152,46))
are equal.
- The type of the first term is:
FStar.WellFoundedRelation.acc_classical wfr_a.relation
(FStar.Pervasives.dfst xy)
- The type of the second term is:
FStar.WellFoundedRelation.acc_classical wfr_a.relation
(FStar.Pervasives.dfst xy)
- If the proof fails, try annotating these with the same type.
|
tests / test-local
ubuntu-latest pipelines will use ubuntu-24.04 soon. For more details, see https://github.com/actions/runner-images/issues/10636
|
tests / test-local:
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 / test-local:
Part2.Free.fst#L132
(350) * Warning 350 at Part2.Free.fst(132,4-134,12):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.Free.fst#L133
(350) * Warning 350 at Part2.Free.fst(133,4-134,12):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.FreeFunExt.fst#L136
(350) * Warning 350 at Part2.FreeFunExt.fst(136,4-138,12):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.FreeFunExt.fst#L137
(350) * Warning 350 at Part2.FreeFunExt.fst(137,4-138,12):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.Par.fst#L40
(350) * Warning 350 at Part2.Par.fst(40,18-40,40):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.Par.fst#L48
(350) * Warning 350 at Part2.Par.fst(48,18-48,40):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.Par.fst#L105
(350) * Warning 350 at Part2.Par.fst(105,4-106,17):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.ST.fst#L26
(350) * Warning 350 at Part2.ST.fst(26,2-28,10):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
tests / test-local:
Part2.ST.fst#L27
(350) * Warning 350 at Part2.ST.fst(27,2-28,10):
- The lightweight do notation [x <-- y; z] or [x ;; z] is deprecated, use let operators (i.e. [let* x = y in z] or [y ;* z], [*] being any sequence of operator characters) instead.
|
ciok
ubuntu-latest pipelines will use ubuntu-24.04 soon. For more details, see https://github.com/actions/runner-images/issues/10636
|
tests / perf-canaries:
DEFS_100#L1
time = 0.15
|
tests / perf-canaries:
DEFS_200#L1
time = 0.15
|
tests / perf-canaries:
DEFS_400#L1
time = 0.17
|
tests / perf-canaries:
DEFS_800#L1
time = 0.23
|
tests / perf-canaries:
DEFS_1600#L1
time = 0.30
|
tests / perf-canaries:
DEFS_3200#L1
time = 0.46
|
tests / perf-canaries:
DEFS_6400#L1
time = 0.82
|
Artifacts
Produced during runtime
Name | Size | |
---|---|---|
fstar-repo
|
311 MB |
|
fstar-src.tar.gz
|
4.97 MB |
|
fstar.tar.gz
|
137 MB |
|