FStar
FStar copied to clipboard
Crash when extracting inner let rec in tactics
module Bug
open FStar.Tactics.Effect
let crash () : Tac int =
let rec aux () : Tac int = 123 in
let r = aux () in
r
$ ./bin/fstar.exe Bug.fst --odir o --codegen OCaml | clip.exe
Extracted module FStar.Pervasives.Native
Extracted module FStar.Preorder
Extracted module FStar.Monotonic.Pure
Unexpected error; please file a bug report, ideally with a minimized version of the source program that triggered the error.
Failure("This should not happen (should have been handled at Tm_abs level for effect FStar.Tactics.Effect.TAC)")
Hit this today