Question about ulib files and naming conventions #3077
Answered
by
nikswamy
chandradeepdey
asked this question in
Q&A
-
Hi! I wanted to add the following to ulib. Could someone please tell me what files I need to change in the PR and any naming conventions that I need to follow? Also, what about let rec list_all_mem_implies_subset_lemma (#a: eqtype) (la lb: list a)
: Lemma (requires (forall x. List.Tot.mem x la ==> List.Tot.mem x lb))
(ensures (List.Tot.subset la lb)) =
match la with
| [] -> ()
| hd :: tl -> list_all_mem_implies_subset_lemma tl lb
let list_subset_self_lemma (#a: eqtype) (l: list a) : Lemma (List.Tot.subset l l) =
list_all_mem_implies_subset_lemma l l |
Beta Was this translation helpful? Give feedback.
Answered by
nikswamy
Oct 31, 2023
Replies: 1 comment 1 reply
-
I would put this in FStar.List.Tot.Properties. For naming and other conventions, see https://github.com/FStarLang/FStar/wiki/Style-guide I would be inclined to remove FStar.List.Pure and merge it into FStar.List.Tot, but that's a separate, larger issue. |
Beta Was this translation helpful? Give feedback.
1 reply
Answer selected by
chandradeepdey
Sign up for free
to join this conversation on GitHub.
Already have an account?
Sign in to comment
I would put this in FStar.List.Tot.Properties.
For naming and other conventions, see https://github.com/FStarLang/FStar/wiki/Style-guide
I would be inclined to remove FStar.List.Pure and merge it into FStar.List.Tot, but that's a separate, larger issue.