Skip to content

Commit

Permalink
Add a test
Browse files Browse the repository at this point in the history
  • Loading branch information
mtzguido committed Aug 26, 2024
1 parent 7772ca8 commit 3e54ed5
Showing 1 changed file with 31 additions and 0 deletions.
31 changes: 31 additions & 0 deletions tests/tactics/PluginReturned.fst
Original file line number Diff line number Diff line change
@@ -0,0 +1,31 @@
module PluginReturned

open FStar.Tactics.V2

(* This used to trip the normalizer due to an extra Meta_monadic
node on the returned and_elim or inspect (which are plugins). *)

assume val p : prop
assume val q : prop

let foo (b:bool) : Tac (term -> Tac unit) =
if b
then and_elim
else fail "no"

let test (x : squash (p /\ q)) =
assert True by (
let f = foo true in
f (quote x);
dump ""
)

let bar () : Tac (term -> Tac term_view) =
inspect

let test2 () =
assert True by (
let f = bar () in
let tv = f (`1) in
dump ""
)

0 comments on commit 3e54ed5

Please sign in to comment.