Skip to content

Commit

Permalink
Fix some (valid) regressions
Browse files Browse the repository at this point in the history
  • Loading branch information
mtzguido committed Jan 14, 2025
1 parent 4953e2b commit b93640e
Show file tree
Hide file tree
Showing 4 changed files with 6 additions and 6 deletions.
2 changes: 1 addition & 1 deletion tests/micro-benchmarks/BinderAttributes.fst
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ let default_to (def : 'a) (x : option 'a) : Tot 'a =
| None -> def
| Some a -> a

type description (d : string) = ()
let description (d : string) = ()

type inductive_example =
| CaseExplicit : [@@@ description "x"] x:int -> [@@@ description "y"] y:string -> inductive_example
Expand Down
6 changes: 3 additions & 3 deletions tests/micro-benchmarks/MultipleAttributesBinder.fst
Original file line number Diff line number Diff line change
Expand Up @@ -7,9 +7,9 @@ type attr_value =
| String : v:string -> attr_value
| Int : v:int -> attr_value

type attr1 (v : string) = ()
type attr2 (v : int) = ()
type attr3 (v : attr_value) = ()
let attr1 (v : string) = ()
let attr2 (v : int) = ()
let attr3 (v : attr_value) = ()

let f (#[@@@ attr1 "imp"; attr2 1; attr3 (String "x")] x_imp:int) ([@@@ attr1 "exp"; attr2 2; attr3 (String "y")] y:string) : Tot unit =
()
Expand Down
2 changes: 1 addition & 1 deletion tests/micro-benchmarks/RecordFieldAttributes.fst
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@ module RecordFieldAttributes

module T = FStar.Tactics.V2

type description (d : string) = ()
let description (d : string) = ()

type r =
{
Expand Down
2 changes: 1 addition & 1 deletion tests/micro-benchmarks/Unit1.Basic.fst
Original file line number Diff line number Diff line change
Expand Up @@ -219,7 +219,7 @@ let test_skolem_match (x:int) =
match apply (fun x -> x) 0 with
| 0 -> 0

type _T = (apply (fun x -> x) 0 = 1)
type _T = (apply (fun x -> x) 0 == 1)

val test_skolem_refinement: x:int{_T} -> Tot unit
let test_skolem_refinement x = assert false
Expand Down

0 comments on commit b93640e

Please sign in to comment.