From 272bfd5439963a3c7603dd80c069276a65b714e7 Mon Sep 17 00:00:00 2001 From: Dzomo the everest Yak Date: Fri, 14 Sep 2018 06:17:50 +0000 Subject: [PATCH] [CI] regenerate hints + ocaml snapshot --- doc/tutorial/code/exercises/Ex03a.fst.hints | 4 +- doc/tutorial/code/exercises/Ex03b.fst.hints | 4 +- doc/tutorial/code/exercises/Ex03c.fst.hints | 4 +- doc/tutorial/code/exercises/Ex04a.fst.hints | 8 +- doc/tutorial/code/exercises/Ex04b.fst.hints | 8 +- doc/tutorial/code/exercises/Ex04c.fst.hints | 8 +- doc/tutorial/code/exercises/Ex04e.fst.hints | 4 +- doc/tutorial/code/exercises/Ex04f.fst.hints | 8 +- doc/tutorial/code/exercises/Ex05a.fst.hints | 12 +- doc/tutorial/code/exercises/Ex05b.fst.hints | 8 +- doc/tutorial/code/exercises/Ex06b.fst.hints | 24 +- doc/tutorial/code/exercises/Ex06e.fst.hints | 8 +- doc/tutorial/code/exercises/Ex07a.fst.hints | 20 +- doc/tutorial/code/exercises/Ex07b.fst.hints | 28 +- doc/tutorial/code/exercises/Ex07c.fst.hints | 28 +- doc/tutorial/code/exercises/Ex07d.fst.hints | 28 +- doc/tutorial/code/exercises/Ex11a.fst.hints | 4 +- .../code/exercises/LowStar.Ex2.fst.hints | 4 +- .../code/exercises/LowStar.Ex3.fst.hints | 14 +- doc/tutorial/code/solutions/Ex03a.fst.hints | 4 +- doc/tutorial/code/solutions/Ex03b.fst.hints | 4 +- doc/tutorial/code/solutions/Ex03c.fst.hints | 6 +- doc/tutorial/code/solutions/Ex04a.fst.hints | 8 +- doc/tutorial/code/solutions/Ex04b.fst.hints | 8 +- doc/tutorial/code/solutions/Ex04c.fst.hints | 8 +- doc/tutorial/code/solutions/Ex04e.fst.hints | 8 +- doc/tutorial/code/solutions/Ex04f.fst.hints | 14 +- doc/tutorial/code/solutions/Ex04h.fst.hints | 8 +- doc/tutorial/code/solutions/Ex05a.fst.hints | 12 +- doc/tutorial/code/solutions/Ex05b.fst.hints | 20 +- doc/tutorial/code/solutions/Ex06a.fst.hints | 4 +- doc/tutorial/code/solutions/Ex06b.fst.hints | 24 +- doc/tutorial/code/solutions/Ex06c.fst.hints | 28 +- doc/tutorial/code/solutions/Ex06d.fst.hints | 24 +- doc/tutorial/code/solutions/Ex06e.fst.hints | 16 +- doc/tutorial/code/solutions/Ex07a.fst.hints | 20 +- doc/tutorial/code/solutions/Ex07b.fst.hints | 32 +- doc/tutorial/code/solutions/Ex07c.fst.hints | 28 +- doc/tutorial/code/solutions/Ex07d.fst.hints | 28 +- doc/tutorial/code/solutions/Ex11a.fst.hints | 4 +- .../code/solutions/LowStar.Ex2.fst.hints | 12 +- .../code/solutions/LowStar.Ex3.fst.hints | 38 +- examples/algorithms/BinarySearch.fst.hints | 8 +- examples/algorithms/Huffman.fst.hints | 36 +- examples/algorithms/InsertionSort.fst.hints | 12 +- examples/algorithms/IntSort.fst.hints | 4 +- examples/algorithms/MergeSort.fst.hints | 12 +- examples/algorithms/QuickSort.List.fst.hints | 16 +- examples/algorithms/QuickSort.Seq.fst.hints | 8 +- examples/algorithms/Unification.fst.hints | 40 +- examples/bug-reports/Bug1423.fst.hints | 2 +- examples/bug-reports/Bug1502.fst.hints | 2 +- examples/bug-reports/Bug1536.fst.hints | 61 ++ examples/bug-reports/ExtractionBug2.fst.hints | 4 +- examples/bug-reports/bug024.fst.hints | 2 +- examples/bug-reports/bug025.fst.hints | 2 +- examples/bug-reports/bug026.fst.hints | 2 +- examples/bug-reports/bug056.fst.hints | 2 +- examples/bug-reports/bug058.fst.hints | 2 +- examples/bug-reports/bug058b.fst.hints | 2 +- examples/bug-reports/bug1091.fst.hints | 24 +- examples/bug-reports/bug1206.fst.hints | 4 +- examples/bug-reports/bug1319b.fst.hints | 2 +- examples/bug-reports/bug1361.fst.hints | 4 +- examples/bug-reports/bug1362.fst.hints | 6 +- examples/bug-reports/bug138.fst.hints | 6 +- examples/bug-reports/bug1414.fst.hints | 12 +- examples/bug-reports/bug1535b.fst.hints | 70 ++ examples/bug-reports/bug161.fst.hints | 2 +- examples/bug-reports/bug162.fst.hints | 2 +- examples/bug-reports/bug173.fst.hints | 8 +- examples/bug-reports/bug185.fst.hints | 2 +- examples/bug-reports/bug279.fst.hints | 2 +- examples/bug-reports/bug281.fst.hints | 6 +- examples/bug-reports/bug379.fst.hints | 2 +- examples/bug-reports/bug463b.fst.hints | 2 +- examples/bug-reports/bug466.fst.hints | 2 +- examples/bug-reports/bug579.fst.hints | 4 +- examples/bug-reports/bug589.fst.hints | 2 +- examples/bug-reports/bug590.fst.hints | 2 +- examples/bug-reports/bug606.fst.hints | 4 +- examples/bug-reports/bug989.fst.hints | 2 +- examples/crypto/CntProtocol.fst.hints | 2 +- examples/crypto/EtM.AE.fst.hints | 4 +- examples/crypto/EtM.CPA.fst.hints | 2 +- examples/csl/Examples.fst.hints | 112 +-- examples/csl/Lang.fst.hints | 4 +- examples/csl/SL.AutoTactic.fst.hints | 112 +-- examples/csl/SL.ConcurrentExamples.fst.hints | 124 ++-- examples/csl/SL.ExamplesAuto.fst.hints | 52 +- examples/csl/SL.ExamplesLocks.fst.hints | 168 ++--- examples/csl/SL.ExamplesLocks2.fst.hints | 82 +-- examples/csl/SL.ExamplesPar.fst.hints | 44 +- examples/csl/SL.Heap.fst.hints | 4 +- examples/csl/SL.Heap.fsti.hints | 4 +- examples/csl/SL.Tactics.fst.hints | 26 +- .../data_structures/ArrayRealized.fst.hints | 8 +- .../BinarySearchTree.fst.hints | 39 +- .../BinarySearchTree0.fst.hints | 8 +- .../BinarySearchTreeBasic.fst.hints | 63 +- .../BinarySearchTreeFirst.fst.hints | 12 +- .../data_structures/BinaryTrees.fst.hints | 40 +- .../BinaryTreesEnumeration.fst.hints | 14 +- examples/data_structures/MerkleTree.fst.hints | 18 +- examples/data_structures/RBTree.fst.hints | 28 +- examples/data_structures/Vector.fst.hints | 32 +- examples/dm4free/FStar.DM4F.Heap.ST.fst.hints | 4 +- examples/kv_parsing/EnumParsing.fst.hints | 170 ++--- examples/kv_parsing/IntegerParsing.fst.hints | 234 +++--- examples/kv_parsing/KeyValue.fst.hints | 68 +- examples/kv_parsing/Parsing.fst.hints | 88 +-- examples/kv_parsing/PureEncoder.fst.hints | 8 +- examples/kv_parsing/PureParser.fst.hints | 12 +- examples/kv_parsing/PureValidator.fst.hints | 44 +- examples/kv_parsing/Serializer.fst.hints | 80 +-- examples/kv_parsing/Serializing.fst.hints | 4 +- examples/kv_parsing/ValidatedAccess.fst.hints | 22 +- examples/kv_parsing/ValidatedParser.fst.hints | 86 +-- examples/kv_parsing/Validator.fst.hints | 16 +- examples/kv_parsing/VectorParsing.fst.hints | 72 +- examples/low-mitls-experiments/HSL.fst.hints | 96 ++- examples/lowparse/LowParse.Bytes32.fst.hints | 20 +- .../lowparse/LowParse.SLow.Base.fst.hints | 62 +- .../LowParse.SLow.Combinators.fst.hints | 134 ++-- .../lowparse/LowParse.SLow.Enum.fst.hints | 66 +- .../lowparse/LowParse.Spec.Base.fst.hints | 4 +- .../lowparse/LowParse.Spec.Enum.fst.hints | 12 +- examples/metatheory/LambdaOmega.fst.hints | 84 +-- examples/metatheory/ParSubst.fst.hints | 4 +- examples/metatheory/StackMachine.fst.hints | 42 +- .../metatheory/StlcCbvDbParSubst.fst.hints | 28 +- .../StlcCbvDbPntSubstNoLists.fst.hints | 24 +- .../metatheory/StlcStrongDbParSubst.fst.hints | 20 +- examples/metatheory/indind.fst.hints | 28 +- .../micro-benchmarks/DoNotation.fst.hints | 4 +- .../micro-benchmarks/FirstProofs.fst.hints | 16 +- .../IntNormalization.fst.hints | 8 +- .../NegativeTests.Termination.fst.hints | 4 +- .../micro-benchmarks/Normalization.fst.hints | 4 +- examples/micro-benchmarks/Pruning.fst.hints | 4 +- .../micro-benchmarks/TwoPhaseTC.fst.hints | 60 +- .../micro-benchmarks/UnifyMatch.fst.hints | 32 +- .../micro-benchmarks/Unit1.Basic.fst.hints | 46 +- .../Unit1.RecursiveTypeFunctions.fst.hints | 20 +- .../miniparse/MiniParse.Impl.Base.fst.hints | 14 +- .../MiniParse.Impl.Combinators.fst.hints | 76 +- .../miniparse/MiniParse.Impl.Int.fst.hints | 24 +- .../miniparse/MiniParse.Impl.List.fst.hints | 121 ++-- .../miniparse/MiniParse.Impl.TSum.fst.hints | 8 +- .../miniparse/MiniParse.Spec.Int.fst.hints | 6 +- .../miniparse/MiniParse.Spec.List.fst.hints | 8 +- .../miniparse/MiniParse.Spec.TEnum.fst.hints | 20 +- .../miniparse/MiniParse.Tac.Base.fst.hints | 20 +- .../miniparse/MiniParse.Tac.Impl.fst.hints | 14 +- .../miniparse/MiniParse.Tac.Spec.fst.hints | 8 +- examples/miniparse/MiniParseExample.fst.hints | 2 +- .../miniparse/MiniParseExample2.fst.hints | 20 +- .../miniparse/MiniParseExample3.fst.hints | 2 +- examples/native_tactics/Arith.fst.hints | 30 +- examples/native_tactics/BV.Test.fst.hints | 28 +- examples/native_tactics/BV.fst.hints | 108 +-- examples/native_tactics/Bane.fst.hints | 4 +- examples/native_tactics/Canon.Test.fst.hints | 8 +- examples/native_tactics/CanonDeep.fst.hints | 6 +- examples/native_tactics/Clear.fst.hints | 4 +- .../native_tactics/DependentSynth.fst.hints | 2 +- examples/native_tactics/Evens.fst.hints | 18 +- examples/native_tactics/Imp.fst.hints | 4 +- .../native_tactics/Plugins.Test.fst.hints | 12 +- examples/native_tactics/Print.Test.fst.hints | 2 +- examples/native_tactics/Pruning.fst.hints | 6 +- .../native_tactics/Registers.List.fst.hints | 16 +- examples/native_tactics/Sequences.fst.hints | 6 +- examples/native_tactics/Simple.fst.hints | 18 +- .../SimpleTactic.Test.fst.hints | 2 +- examples/native_tactics/Split.fst.hints | 2 +- examples/native_tactics/Tutorial.fst.hints | 8 +- examples/native_tactics/Unify.fst.hints | 2 +- examples/printf/SimplePrintf.fst.hints | 12 +- examples/rel/Benton2004.DDCC.fst.hints | 6 +- examples/rel/Benton2004.RHL.fst.hints | 4 +- .../rel/Benton2004.SmithVolpano.fst.hints | 4 +- examples/rel/Benton2004.fst.hints | 8 +- examples/rel/IfcDelimitedRelease.fst.hints | 12 +- .../rel/IfcDelimitedReleaseReify.fst.hints | 4 +- examples/rel/IfcRecursiveReify.fst.hints | 12 +- examples/rel/IfcRules.fst.hints | 2 +- examples/rel/IfcRulesReify.fst.hints | 2 +- examples/rel/IfcTypechecker.fst.hints | 4 +- examples/rel/Loops.fst.hints | 12 +- examples/rel/Memo.fst.hints | 54 +- examples/rel/ProgramEquivalence.fst.hints | 8 +- examples/rel/ProgramOptimizations.fst.hints | 20 +- examples/rel/Recursive.fst.hints | 6 +- examples/rel/UnionFind.Forest.fst.hints | 4 +- examples/rel/UnionFind.Functions.fst.hints | 8 +- examples/rel/While.fst.hints | 12 +- examples/rel/WhileReify.fst.hints | 8 +- examples/seplogic/Examples.fst.hints | 112 +-- examples/seplogic/SL.Examples.fst.hints | 382 +++++----- examples/seplogic/SL.ExamplesAuto.fst.hints | 130 ++-- .../software_foundations/SfBasic.fst.hints | 24 +- .../software_foundations/SfLists.fst.hints | 42 +- .../software_foundations/SfPoly.fst.hints | 48 +- examples/tactics/Alt.fst.hints | 8 +- examples/tactics/AnnoyingVCs.fst.hints | 6 +- examples/tactics/Arith.fst.hints | 60 +- examples/tactics/Bane.Lib.fst.hints | 10 +- examples/tactics/Bug1252.fst.hints | 4 +- examples/tactics/Bug1256.fst.hints | 2 +- examples/tactics/Bug1270.fst.hints | 8 +- examples/tactics/Bug1299.fst.hints | 4 +- examples/tactics/Canon.fst.hints | 14 +- examples/tactics/CanonCommMonoid.fst.hints | 112 +-- .../tactics/CanonCommMonoidSimple.fst.hints | 90 +-- examples/tactics/CanonCommSemiring.fst.hints | 136 ++-- examples/tactics/CanonCommSwaps.fst.hints | 20 +- examples/tactics/CanonMonoid.fst.hints | 42 +- examples/tactics/Cases.fst.hints | 14 +- examples/tactics/Change.fst.hints | 8 +- examples/tactics/Clear.fst.hints | 12 +- examples/tactics/DeltaDepth.fst.hints | 16 +- examples/tactics/DependentSynth.fst.hints | 4 +- examples/tactics/Destruct.fst.hints | 188 ++--- examples/tactics/Easy.fst.hints | 8 +- examples/tactics/Even.fst.hints | 26 +- examples/tactics/FailFlow.fst.hints | 30 +- examples/tactics/Fresh.fst.hints | 8 +- examples/tactics/GRewrite.fst.hints | 28 +- examples/tactics/Goals.fst.hints | 8 +- examples/tactics/HoleBy.fst.hints | 6 +- examples/tactics/Imp.fst.hints | 120 ++-- examples/tactics/Inlining.fst.hints | 18 +- examples/tactics/Join.fst.hints | 224 +++--- examples/tactics/Labels.fst.hints | 8 +- examples/tactics/LemmaArgs.fst.hints | 14 +- examples/tactics/MetaArgs.fst.hints | 14 +- examples/tactics/MkList.fst.hints | 8 +- examples/tactics/Neg.fst.hints | 4 +- examples/tactics/NormBinderType.fst.hints | 4 +- examples/tactics/Normalization.fst.hints | 32 +- examples/tactics/Poly.fst.hints | 12 +- examples/tactics/Pose.fst.hints | 4 +- examples/tactics/Postprocess.fst.hints | 56 +- examples/tactics/Printers.fst.hints | 60 +- examples/tactics/Pruning.fst.hints | 12 +- examples/tactics/Raise.fst.hints | 115 +++ examples/tactics/Rewrite.Monoid.fst.hints | 10 +- examples/tactics/Sequences.fst.hints | 10 +- examples/tactics/Setopts.fst.hints | 8 +- examples/tactics/Splice.fst.hints | 4 +- examples/tactics/Splice2.fst.hints | 8 +- examples/tactics/State.fst.hints | 4 +- examples/tactics/StringPrinter.Base.fst.hints | 122 ++-- examples/tactics/StringPrinter.Rec.fst.hints | 18 +- examples/tactics/StringPrinter.RecC.fst.hints | 40 +- .../tactics/StringPrinterTest.Aux.fst.hints | 52 +- examples/tactics/StringPrinterTest.fst.hints | 8 +- examples/tactics/Syntax.fst.hints | 4 +- examples/tactics/Synthesis.fst.hints | 36 +- examples/tactics/Tautology.fst.hints | 4 +- examples/tactics/TestBV.fst.hints | 44 +- examples/tactics/Trace.fst.hints | 38 +- examples/tactics/Trans.fst.hints | 2 +- examples/tactics/Tutorial.fst.hints | 16 +- examples/tactics/Unfold.fst.hints | 2 +- examples/tactics/Unify.fst.hints | 4 +- examples/tactics/UnitTests.fst.hints | 82 +-- examples/tactics/UserTactics.fst.hints | 34 +- examples/tactics/WeakVsHNF.fst.hints | 6 +- examples/tactics/Wild.fst.hints | 4 +- examples/termination/CPS.Double.fst.hints | 4 +- .../termination/CPS.DoubleDefun.fst.hints | 12 +- .../CPS.DoubleLambdaLifting2.fst.hints | 4 +- examples/termination/CPS.Simple.fst.hints | 4 +- .../termination/CPS.SimpleDefun.fst.hints | 8 +- .../CPS.SimpleLambdaLifting.fst.hints | 4 +- examples/termination/Eval.DB.fst.hints | 8 +- examples/termination/mcCarthy91.fst.hints | 4 +- examples/termination/termination.fst.hints | 76 +- examples/typeclasses/Add.fst.hints | 44 +- examples/typeclasses/Enum.fst.hints | 32 +- examples/typeclasses/EnumEq.fst.hints | 4 +- examples/typeclasses/Eq.fst.hints | 76 +- examples/typeclasses/Loop2.fst.hints | 12 +- examples/typeclasses/Monad.fst.hints | 12 +- examples/typeclasses/Tests.fst.hints | 20 +- examples/vale/Asm1.fst.hints | 4 +- examples/vale/Calc.fst.hints | 16 +- .../vale/X64.Poly1305.Bitvectors_i.fst.hints | 170 ++--- examples/vale/X64.Poly1305.Math_i.fst.hints | 78 +- examples/vale/X64.Poly1305.Spec_s.fst.hints | 4 +- examples/vale/X64.Poly1305.fst.hints | 86 +-- examples/vale/X64.Print_s.fst.hints | 12 +- examples/vale/X64.Semantics_s.fst.hints | 12 +- examples/vale/X64.Vale.StrongPost_i.fst.hints | 6 +- examples/verifythis/2015/Problem01.fst.hints | 8 +- ulib/FStar.BitVector.fst.hints | 24 +- ulib/FStar.BufferNG.fst.hints | 8 +- ulib/FStar.Bytes.fsti.hints | 72 +- ulib/FStar.Crypto.fst.hints | 12 +- ulib/FStar.Fin.fst.hints | 12 +- ulib/FStar.GSet.fst.hints | 4 +- ulib/FStar.List.Pure.Base.fst.hints | 8 +- ulib/FStar.List.Tot.Base.fst.hints | 140 ++-- ulib/FStar.List.Tot.Properties.fst.hints | 14 +- ulib/FStar.Math.Lemmas.fst.hints | 2 +- ulib/FStar.Math.Lib.fst.hints | 8 +- ulib/FStar.Monotonic.DependentMap.fst.hints | 6 +- ulib/FStar.Monotonic.HyperHeap.fst.hints | 8 +- ulib/FStar.Monotonic.HyperStack.fst.hints | 12 +- ulib/FStar.Monotonic.Seq.fst.hints | 10 +- ulib/FStar.OrdMapProps.fst.hints | 4 +- ulib/FStar.OrdSet.fst.hints | 24 +- ulib/FStar.OrdSetProps.fst.hints | 4 +- ulib/FStar.Order.fst.hints | 4 +- ulib/FStar.Pervasives.fst.hints | 2 +- ulib/FStar.Pointer.Base.fst.hints | 49 +- ulib/FStar.Pointer.Base.fsti.hints | 6 +- ulib/FStar.Printf.fst.hints | 12 +- ulib/FStar.Reflection.Arith.fst.hints | 184 ++--- ulib/FStar.Reflection.Data.fst.hints | 4 +- .../FStar.Reflection.Derived.Lemmas.fst.hints | 4 +- ulib/FStar.Reflection.Derived.fst.hints | 48 +- ulib/FStar.Reflection.Formula.fst.hints | 112 +-- ulib/FStar.Seq.Base.fst.hints | 26 +- ulib/FStar.Seq.Properties.fst.hints | 56 +- ulib/FStar.Seq.Sorted.fst.hints | 4 +- ulib/FStar.Set.fst.hints | 4 +- ulib/FStar.TSet.fst.hints | 4 +- ulib/FStar.Tactics.BV.fst.hints | 124 ++-- ulib/FStar.Tactics.Builtins.fst.hints | 2 +- ulib/FStar.Tactics.Canon.fst.hints | 42 +- ulib/FStar.Tactics.Derived.fst.hints | 177 ++--- ulib/FStar.Tactics.Effect.fst.hints | 34 +- ulib/FStar.Tactics.Logic.fst.hints | 46 +- ulib/FStar.Tactics.PatternMatching.fst.hints | 170 ++--- ulib/FStar.Tactics.Result.fst.hints | 24 +- ulib/FStar.Tactics.Simplifier.fst.hints | 22 +- ulib/FStar.Tactics.Typeclasses.fst.hints | 70 +- ulib/FStar.Tactics.Types.fsti.hints | 20 +- ulib/FStar.Tactics.Util.fst.hints | 16 +- ulib/FStar.TaggedUnion.fst.hints | 4 +- ulib/FStar.TaggedUnion.fsti.hints | 4 +- ulib/FStar.Tcp.fsti.hints | 6 +- ulib/FStar.UInt.fst.hints | 16 +- ulib/FStar.WellFounded.fst.hints | 4 +- ulib/LowStar.Buffer.fst.hints | 44 +- ulib/LowStar.BufferCompat.fst.hints | 14 +- ulib/LowStar.BufferOps.fst.hints | 14 +- ulib/LowStar.BufferView.fst.hints | 88 ++- ulib/LowStar.BufferView.fsti.hints | 26 +- ulib/LowStar.ImmutableBuffer.fst.hints | 30 +- ulib/LowStar.Monotonic.Buffer.fst.hints | 183 +++-- ulib/LowStar.Monotonic.Buffer.fsti.hints | 98 ++- ulib/LowStar.ToFStarBuffer.fst.hints | 102 +-- ulib/LowStar.UninitializedBuffer.fst.hints | 679 ++++++++++++++++++ ulib/prims.fst.hints | 4 +- 358 files changed, 6049 insertions(+), 5034 deletions(-) create mode 100644 examples/bug-reports/Bug1536.fst.hints create mode 100644 examples/bug-reports/bug1535b.fst.hints create mode 100644 examples/tactics/Raise.fst.hints create mode 100644 ulib/LowStar.UninitializedBuffer.fst.hints diff --git a/doc/tutorial/code/exercises/Ex03a.fst.hints b/doc/tutorial/code/exercises/Ex03a.fst.hints index 74ea363ab45..c34f4c17a0b 100644 --- a/doc/tutorial/code/exercises/Ex03a.fst.hints +++ b/doc/tutorial/code/exercises/Ex03a.fst.hints @@ -15,7 +15,7 @@ "well-founded-ordering-on-nat" ], 0, - "b6687cbc476fd20d31713c942f9711a8" + "76e3147de1d785692c5752d090cd976c" ], [ "Ex03a.factorial", @@ -31,7 +31,7 @@ "well-founded-ordering-on-nat" ], 0, - "dae73103b13efa0e57bbb6d6fa73a752" + "61401b1e8c4405bd2c79cca75fdba980" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex03b.fst.hints b/doc/tutorial/code/exercises/Ex03b.fst.hints index 2775ad9dd6b..ea3ba553b3c 100644 --- a/doc/tutorial/code/exercises/Ex03b.fst.hints +++ b/doc/tutorial/code/exercises/Ex03b.fst.hints @@ -15,7 +15,7 @@ "well-founded-ordering-on-nat" ], 0, - "3eb5e92cb6a537be8d1562e9a90a1cec" + "c313cdc06a906f357649d990ed699f23" ], [ "Ex03b.fibonacci", @@ -31,7 +31,7 @@ "well-founded-ordering-on-nat" ], 0, - "46fe0bf374bd12ea112c360478137bed" + "d9ff4730065f2704b795c2a11474c97b" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex03c.fst.hints b/doc/tutorial/code/exercises/Ex03c.fst.hints index 931d8f5f3e0..857f0d1edd1 100644 --- a/doc/tutorial/code/exercises/Ex03c.fst.hints +++ b/doc/tutorial/code/exercises/Ex03c.fst.hints @@ -17,7 +17,7 @@ "well-founded-ordering-on-nat" ], 0, - "936f98103cc4eda3bf0b1856bc235614" + "dc68bcbafa2a36619037586e34925bde" ], [ "Ex03c.fibonacci", @@ -35,7 +35,7 @@ "well-founded-ordering-on-nat" ], 0, - "88d40100c5f9008931d0c6f2945c8e40" + "2aa0d7cecafadad8438221ebb8b2c576" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex04a.fst.hints b/doc/tutorial/code/exercises/Ex04a.fst.hints index 457ae5aeb79..0b6b7189504 100644 --- a/doc/tutorial/code/exercises/Ex04a.fst.hints +++ b/doc/tutorial/code/exercises/Ex04a.fst.hints @@ -16,7 +16,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "fab9dc3186a6c9366e799e337907ddd8" + "8ec752beaf705eb747b1ed9629bfb008" ], [ "Ex04a.append", @@ -30,7 +30,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "62c6dfd7e17bd3e923cf192ba32828d5" + "c8fe010178d564da6579e851d6b570b6" ], [ "Ex04a.length", @@ -47,7 +47,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "2004ba46bf4ccbd85339eb44602c0af4" + "bbfbb0b6e69935eac642d74184010fb5" ], [ "Ex04a.append", @@ -61,7 +61,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "51d39c4a679a04d1d493f48354b0dcae" + "cda88999adcc79d06b37207112ed247d" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex04b.fst.hints b/doc/tutorial/code/exercises/Ex04b.fst.hints index aa782bc2502..2ff240244f5 100644 --- a/doc/tutorial/code/exercises/Ex04b.fst.hints +++ b/doc/tutorial/code/exercises/Ex04b.fst.hints @@ -16,7 +16,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "d02d6627e3f392b08c9e8ce1c5230a3b" + "1440708be33e0e7b3c2ce24d8104aa8f" ], [ "Ex04b.append", @@ -31,7 +31,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "9f5b23ca8b769b5039d84b242d12b095" + "7d6dc0fadd12b74725dc84a28134d931" ], [ "Ex04b.append_len", @@ -57,7 +57,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "a26a13220999c9dba765c81fd046892d" + "7d53632089291d3d1d8822a3c7b848e1" ], [ "Ex04b.append", @@ -71,7 +71,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "d569a36a2c96956990dad164d8dfd2ff" + "2163782d98ff5791ada9875a39f7414e" ], [ "Ex04b.append_len", diff --git a/doc/tutorial/code/exercises/Ex04c.fst.hints b/doc/tutorial/code/exercises/Ex04c.fst.hints index 3124ddba62a..acdef3e140d 100644 --- a/doc/tutorial/code/exercises/Ex04c.fst.hints +++ b/doc/tutorial/code/exercises/Ex04c.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "ffc55c0c4e9a74e9122a70f26ef7940c" + "a02ed18a045b3fa57772585d87c790e0" ], [ "Ex04c.mem", @@ -28,7 +28,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "e91339b1985f802aeaa5ecc7af66a197" + "b56970501804ac73a158c189405b8fbc" ], [ "Ex04c.append", @@ -42,7 +42,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "c8cb79f40ab20ab8509802d2f802e9ef" + "df19543978e2c23beac8e29ea9e5d927" ], [ "Ex04c.mem", @@ -57,7 +57,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "258b6c7e64d7b57bb26a3800e846453a" + "c20556427a089e049c7cb71757cfcd0e" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex04e.fst.hints b/doc/tutorial/code/exercises/Ex04e.fst.hints index 6725191dd0f..378cc5af3ef 100644 --- a/doc/tutorial/code/exercises/Ex04e.fst.hints +++ b/doc/tutorial/code/exercises/Ex04e.fst.hints @@ -35,7 +35,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "2793520c35377104b3958d51dbe2fd52" + "41e05aae09d5cb18130195d1cb7f25e8" ], [ "Ex04e.option", @@ -71,7 +71,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "1e4efe914a23e44358491cb7579c5e11" + "330e051f9af1465a63b0afa4212850fb" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex04f.fst.hints b/doc/tutorial/code/exercises/Ex04f.fst.hints index b7712715c8e..ad70e404236 100644 --- a/doc/tutorial/code/exercises/Ex04f.fst.hints +++ b/doc/tutorial/code/exercises/Ex04f.fst.hints @@ -14,7 +14,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "0cb1eb8c0837ad0d30237a5dbd69c088" + "c6ffb06d2e38689fb8a21ef55b2d44de" ], [ "Ex04f.reverse", @@ -29,7 +29,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "f889c9d10cb3dd73edfc158c069bc343" + "994e3bf9a1558d240b021be8a29e4b4c" ], [ "Ex04f.append", @@ -43,7 +43,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "a0ad81cd657dbc4d575ea00911d435f4" + "8cde49732245b28aa6ed72366319cc86" ], [ "Ex04f.reverse", @@ -57,7 +57,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "8391f3c3a60be84fad2d28175d6840a8" + "cba2df6efb3cefd38d3a7942213ca7b5" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex05a.fst.hints b/doc/tutorial/code/exercises/Ex05a.fst.hints index f18e39572b5..9218b88466b 100644 --- a/doc/tutorial/code/exercises/Ex05a.fst.hints +++ b/doc/tutorial/code/exercises/Ex05a.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "314bdb51b5142a141cccd4ea6d59e5c3" + "78f442075beb1f149c88bf49f3f7ce0f" ], [ "Ex05a.reverse", @@ -27,7 +27,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "cb42482a295f6d5bfab4139d7cb3b4e0" + "6ff7a998392647d5a6c13b5e5da50569" ], [ "Ex05a.rev", @@ -42,7 +42,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "239646108938d77861f9fa992a334631" + "123020bf33ba9a1d7994eb890d2c984c" ], [ "Ex05a.append_assoc", @@ -78,7 +78,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "3f1fe816a325d337910683bfd6bd50f4" + "da753a0ea698a7378722f8243822fb4b" ], [ "Ex05a.reverse", @@ -92,7 +92,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "f9097ffca4f4349ce5441ee1a1cbce05" + "bce4032db6caa5e7209e989132c9810d" ], [ "Ex05a.rev", @@ -107,7 +107,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "ab43c71597323ba5db0739edbb064e5d" + "34181cb70dee024a908b80d31648ddcc" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex05b.fst.hints b/doc/tutorial/code/exercises/Ex05b.fst.hints index a2357d2cc20..eaeab438226 100644 --- a/doc/tutorial/code/exercises/Ex05b.fst.hints +++ b/doc/tutorial/code/exercises/Ex05b.fst.hints @@ -17,7 +17,7 @@ "well-founded-ordering-on-nat" ], 0, - "119128aa621c5bd54da8960e175199d0" + "e82513efc45e644b87153b95ef00e167" ], [ "Ex05b.fib", @@ -37,7 +37,7 @@ "well-founded-ordering-on-nat" ], 0, - "f7f1d31925eda0efd4bf3a09d3ea3efa" + "a0519c2f42fff1155377c627f20a84dc" ], [ "Ex05b.fib_is_ok", @@ -67,7 +67,7 @@ "well-founded-ordering-on-nat" ], 0, - "600af676c19c7759ed128ccb318ea275" + "2d622ee58aceb5e0327aed17069b4fb5" ], [ "Ex05b.fib", @@ -87,7 +87,7 @@ "well-founded-ordering-on-nat" ], 0, - "d5d286966c0be7cf11faa649b4f43f2c" + "a6e89d43e37688eda9e2a90fad1ced00" ], [ "Ex05b.fib_is_ok", diff --git a/doc/tutorial/code/exercises/Ex06b.fst.hints b/doc/tutorial/code/exercises/Ex06b.fst.hints index 3f6dd6b5f3b..2600b70ed85 100644 --- a/doc/tutorial/code/exercises/Ex06b.fst.hints +++ b/doc/tutorial/code/exercises/Ex06b.fst.hints @@ -14,7 +14,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "2ff60d0298cc0e28142e9e52cabc37ec" + "79e355fa114904831465b67933e0c610" ], [ "Ex06b.append", @@ -29,7 +29,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "ac24ab1c057ebb31a79189fd2e7a673a" + "d7bc7bf7280b3bfe0dca6e3024d28ed9" ], [ "Ex06b.append_mem", @@ -85,7 +85,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "90d4e2a77c6a4602fbc0cf9b30d4fa6b" + "9b14f9ac63e084b15cb15bd8912e43d5" ], [ "Ex06b.sorted", @@ -104,7 +104,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "6d4c1bb200c2271ab1e8361f3dce5d69" + "5262ee3496783607ad170c6b29d0066f" ], [ "Ex06b.partition", @@ -119,7 +119,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "e363c524126d8ea009eeb61ce74d4e28" + "c31169208e20268b52db721ae3549e1d" ], [ "Ex06b.partition_lemma", @@ -309,7 +309,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "2157fca8679b43c71acb147dd0a1fd1b" + "43afd1cb0b9b0172e78c1159b949c71b" ], [ "Ex06b.mem", @@ -324,7 +324,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "64dc31b2a7c21a411791a0c327d8dc2e" + "b91759864796ebe72892a9a665bfc04f" ], [ "Ex06b.append", @@ -338,7 +338,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "f6e28ca4a1659ebd8fd3f9006444ba83" + "bb182962a6cfbe412c95a7c13ef2b7a3" ], [ "Ex06b.append_mem", @@ -364,7 +364,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "44ed3b809ff05c4106b2d16dcfe09b04" + "bec7386c8dfb94ad59086206da89ae17" ], [ "Ex06b.sorted", @@ -382,7 +382,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "8d26a4f698455a569af0027662c24f4b" + "230d5374768a208e4b6f5015df64002f" ], [ "Ex06b.partition", @@ -396,7 +396,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "1771250da8c25e57e54db55919d43006" + "73e3c3f2e86e2b60fe67803591a8fa46" ], [ "Ex06b.partition_lemma", @@ -514,7 +514,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "720016af44abd1d0613f0816c4c3eeba" + "d9697cc3ddf881e45c7c27b8bff2ab34" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex06e.fst.hints b/doc/tutorial/code/exercises/Ex06e.fst.hints index ef17ee00f96..962504a793c 100644 --- a/doc/tutorial/code/exercises/Ex06e.fst.hints +++ b/doc/tutorial/code/exercises/Ex06e.fst.hints @@ -17,7 +17,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "9b7137e8b518de48dd4a1ee72927972c" + "2f195d592e90253eb34371d21f2480f8" ], [ "Ex06e.mem", @@ -36,7 +36,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "46b254d8093b332b4e6498d301f341eb" + "823f31acf50513706aea3d08582e6b32" ], [ "Ex06e.sorted", @@ -54,7 +54,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "c432aa8d153eb6f7567e6fac45fcd5f4" + "236798206beb319461b17ed47ad1beae" ], [ "Ex06e.mem", @@ -73,7 +73,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "f205862d025b646791949a15db1c0631" + "128731a24297c43780d7b6c37c0371eb" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex07a.fst.hints b/doc/tutorial/code/exercises/Ex07a.fst.hints index 5a366f3a94e..7503aa96c59 100644 --- a/doc/tutorial/code/exercises/Ex07a.fst.hints +++ b/doc/tutorial/code/exercises/Ex07a.fst.hints @@ -193,7 +193,7 @@ "subterm_ordering_Ex07a.EIf" ], 0, - "a0cc790757619071dcdf4963262d51d8" + "261b3a5152fa224e2a5ffcd55abbbe9c" ], [ "Ex07a.step", @@ -213,7 +213,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "e1c90ca1d6083c5903bcaacfea40424f" + "e8e76e2b0bb70552cc952660a5a22783" ], [ "Ex07a.extend", @@ -248,7 +248,7 @@ "typing_tok_Ex07a.TBool@tok" ], 0, - "c5181f3c89df5d82f62a65463afc3bba" + "9a1e1ac6cca98b93201a82212e556752" ], [ "Ex07a.progress", @@ -329,7 +329,7 @@ "subterm_ordering_Ex07a.EApp", "subterm_ordering_Ex07a.EIf" ], 0, - "074e6de73cb96ac7980d92228a83d3f2" + "434fc1161c9303a749b5bc975eee68cf" ], [ "Ex07a.free_in_context", @@ -394,7 +394,7 @@ "typing_tok_Ex07a.TBool@tok" ], 0, - "f75db1287ae0bef52f47201997cb3cb9" + "ebb788d8ea72d3355a74d7badaee19a6" ], [ "Ex07a.typable_empty_closed", @@ -490,7 +490,7 @@ "typing_Ex07a.typing", "typing_tok_Ex07a.TBool@tok", "unit_typing" ], 0, - "5a956b80cc6857dd23061637eeb7a37d" + "fc1d10bbbe8237b5e784d81c60eceda9" ], [ "Ex07a.typing_extensional", @@ -827,7 +827,7 @@ "subterm_ordering_Ex07a.EApp", "subterm_ordering_Ex07a.EIf" ], 0, - "e9aa2a1e7cbd9143f7a9695c9ae872c7" + "146ee7030b8cfc32265ee46fd2d7e141" ], [ "Ex07a.step", @@ -847,7 +847,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "0ea6c00bcd0fb943f0ac5547d3b304fe" + "c5c3c0d2909d392158aa48f9ac070707" ], [ "Ex07a.extend", @@ -882,7 +882,7 @@ "typing_tok_Ex07a.TBool@tok" ], 0, - "8a4542abd0385155bacd8f88efc0ad7a" + "98b607506577b3eee92701f91fa400a0" ], [ "Ex07a.appears_free_in", @@ -901,7 +901,7 @@ "subterm_ordering_Ex07a.EApp", "subterm_ordering_Ex07a.EIf" ], 0, - "835939097132c681be99523ccb9ed6b2" + "247d88439ddbf42e45f5b1b6201c9ecb" ], [ "Ex07a.equal", diff --git a/doc/tutorial/code/exercises/Ex07b.fst.hints b/doc/tutorial/code/exercises/Ex07b.fst.hints index 576c5e90bd0..edfc9bd32ba 100644 --- a/doc/tutorial/code/exercises/Ex07b.fst.hints +++ b/doc/tutorial/code/exercises/Ex07b.fst.hints @@ -212,7 +212,7 @@ "subterm_ordering_Ex07b.EApp", "subterm_ordering_Ex07b.EIf" ], 0, - "ab99fcfa5430924d2e26ac01df42104a" + "9c63e6e6522f42ac0cacc7779604aea1" ], [ "Ex07b.step", @@ -233,7 +233,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "1413b593a983b3d27a37c1419255c21b" + "21700034a0c0dd7727cf4aa09de8b16c" ], [ "Ex07b.extend", @@ -268,7 +268,7 @@ "typing_tok_Ex07b.TBool@tok" ], 0, - "70e11f14ab6f85c210c567804a50a460" + "125a80007ccb5f3dd5aa701135ebfc1c" ], [ "Ex07b.progress", @@ -355,7 +355,7 @@ "subterm_ordering_Ex07b.EIf" ], 0, - "81b54905dcea1355309ae1a6dd69e595" + "70127a14eae85f0fce92b62a94e8929b" ], [ "Ex07b.free_in_context", @@ -420,7 +420,7 @@ "typing_tok_Ex07b.ETrue@tok", "typing_tok_Ex07b.TBool@tok" ], 0, - "8ec82a31c41e48399d04e2b5dfd0e98f" + "5f303c362107d8f90cc242d7909ce53b" ], [ "Ex07b.typable_empty_closed", @@ -516,7 +516,7 @@ "typing_Ex07b.typing", "typing_tok_Ex07b.TBool@tok" ], 0, - "6fe6df32fd9586b6e30310073680fa01" + "4ef7996564f7b16bd702e5901f39a395" ], [ "Ex07b.typing_extensional", @@ -615,7 +615,7 @@ "typing_tok_Ex07b.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "9c33322daefc0bdfb3a1eef201532828" + "ce2f1cf8b84f607c66751f790c7ac3be" ], [ "Ex07b.preservation", @@ -691,7 +691,7 @@ "typing_tok_Ex07b.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "e2ba039e487bfec9a30ed5f60c3736ec" + "55f5eab7891815d6e9eec84ca8959b30" ], [ "Ex07b.ty", @@ -900,7 +900,7 @@ "subterm_ordering_Ex07b.EApp", "subterm_ordering_Ex07b.EIf" ], 0, - "0ac2d4ac2b0423c11232a21a7a5a054e" + "824258788e313800b5dc2ef8db01666a" ], [ "Ex07b.step", @@ -920,7 +920,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "1e8abb6924b118ac88e9cd6ded20f299" + "be1dc786aa143cfc8bae91f93d4667e1" ], [ "Ex07b.extend", @@ -955,7 +955,7 @@ "typing_tok_Ex07b.TBool@tok" ], 0, - "23526bd5fd191803b97c16a3eb7981e4" + "9848d0d2342b5131964916be7e59eb06" ], [ "Ex07b.appears_free_in", @@ -974,7 +974,7 @@ "subterm_ordering_Ex07b.EApp", "subterm_ordering_Ex07b.EIf" ], 0, - "a5ec3154bd35c156a7e9f08027998588" + "60b12482b7d6a349878920ce27f99201" ], [ "Ex07b.equal", @@ -1077,7 +1077,7 @@ "typing_tok_Ex07b.TBool@tok", "unit_typing" ], 0, - "20d4bc84b60239ec24932faee60936d1" + "07779472b8b766d3927c2e5960d33095" ], [ "Ex07b.preservation", @@ -1139,7 +1139,7 @@ "typing_tok_Ex07b.TBool@tok" ], 0, - "db70d1c8ed50d2003b4665eba5005377" + "dd147b71eb0529926671e126c3d2832f" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex07c.fst.hints b/doc/tutorial/code/exercises/Ex07c.fst.hints index 7a219fe7677..64080ed5b93 100644 --- a/doc/tutorial/code/exercises/Ex07c.fst.hints +++ b/doc/tutorial/code/exercises/Ex07c.fst.hints @@ -193,7 +193,7 @@ "subterm_ordering_Ex07c.EIf" ], 0, - "cb3aa75d37d98f6d227b438b40314bb6" + "38f9a58d25596ee0cdab6772be1bfa43" ], [ "Ex07c.step", @@ -213,7 +213,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "7228a6dcba906bee07342b28fc118628" + "67ae53946465416883664b86d8aea213" ], [ "Ex07c.extend", @@ -248,7 +248,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "8335be9249dc0d842e5b6781e2c71c7a" + "7065dbf2af43e6795d27186e3a3dc50b" ], [ "Ex07c.progress", @@ -329,7 +329,7 @@ "subterm_ordering_Ex07c.EApp", "subterm_ordering_Ex07c.EIf" ], 0, - "8bea03148f78853e13e467a61ca5b7b5" + "cfbc2e2d988b2faf3ff8b2b67acbb3d7" ], [ "Ex07c.free_in_context", @@ -396,7 +396,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "b4c12fb962fd3ed118f82315a67a58e9" + "98da45f53649cf7289cd9bebfe4be0e6" ], [ "Ex07c.typable_empty_closed", @@ -491,7 +491,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "dfaa8f882b450440e57d43a97259cfb4" + "2a9d5a271c57793a9753e80ee99f40ed" ], [ "Ex07c.typing_extensional", @@ -592,7 +592,7 @@ "typing_tok_Ex07c.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "97e24c97cea9d3fcd487cf220c40c927" + "c0453250331aa76848def5007ee8b22b" ], [ "Ex07c.preservation", @@ -671,7 +671,7 @@ "typing_tok_Ex07c.TBool@tok", "unit_typing" ], 0, - "ac891a8e0ae22807a75c11ebaf1b892f" + "82c53973381f953d7606bc24ca804e0f" ], [ "Ex07c.ty", @@ -854,7 +854,7 @@ "subterm_ordering_Ex07c.EApp", "subterm_ordering_Ex07c.EIf" ], 0, - "3ec066f884809c92bf1ecadfee0c7184" + "7d20a747fd3c5e5e45d0ea92d11a0504" ], [ "Ex07c.step", @@ -874,7 +874,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "e7cfe932df9995cf75bac5583bd4fbfb" + "6fcfb58b0374666bb1d26d205a629fde" ], [ "Ex07c.extend", @@ -909,7 +909,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "82cd9807f4d741a106a41abb84eb4053" + "30bbab80961654b8c62419043c5cb3dc" ], [ "Ex07c.appears_free_in", @@ -928,7 +928,7 @@ "subterm_ordering_Ex07c.EApp", "subterm_ordering_Ex07c.EIf" ], 0, - "7dea86bdb03f0e77a1cce287c6b73ad8" + "b887a23988b0cadada9033caf1db400c" ], [ "Ex07c.equal", @@ -1031,7 +1031,7 @@ "typing_tok_Ex07c.TBool@tok", "unit_typing" ], 0, - "05375137113d760376e19f675dac7c60" + "6de23669c5661d941e087d7f47ce5eda" ], [ "Ex07c.preservation", @@ -1091,7 +1091,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "ed3de48d958516f64260a3ad3129ecb0" + "01c7813e6e66b937685fc19d8d5c21b9" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/Ex07d.fst.hints b/doc/tutorial/code/exercises/Ex07d.fst.hints index 05bcf5b35db..713d96cc997 100644 --- a/doc/tutorial/code/exercises/Ex07d.fst.hints +++ b/doc/tutorial/code/exercises/Ex07d.fst.hints @@ -193,7 +193,7 @@ "subterm_ordering_Ex07d.EIf" ], 0, - "16f0d4e3314a871b97fa03d5812eb738" + "a8713f25fca38349badb020addcc49b0" ], [ "Ex07d.step", @@ -213,7 +213,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "c160cc089ebf576391c771c8e87c5e11" + "b0b61cf5aacff6e29ec8529dbbb40b22" ], [ "Ex07d.extend", @@ -248,7 +248,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "b9229ada7d86eaeca59926ad59a02fc1" + "1007c5280749da930340cf2bc48bd22a" ], [ "Ex07d.progress", @@ -329,7 +329,7 @@ "subterm_ordering_Ex07d.EApp", "subterm_ordering_Ex07d.EIf" ], 0, - "c065d0cf34d3e59bd72d980a84cd1e88" + "87a4ec00b46966a6b3d7370de1b6b6cd" ], [ "Ex07d.free_in_context", @@ -394,7 +394,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "22964c3693b1ab7ff19472863bbd5418" + "d68746c3f051cadfec29154b0b1e6119" ], [ "Ex07d.typable_empty_closed", @@ -491,7 +491,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "faad885210a10d3c29edb7c94955cd73" + "05142b618e6b95d3aba51bd4448518f5" ], [ "Ex07d.typing_extensional", @@ -592,7 +592,7 @@ "typing_tok_Ex07d.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "aef49b88bc7dd68b1d3f68b5130c533a" + "7f20b255efb0e518ca656bc196479643" ], [ "Ex07d.preservation", @@ -669,7 +669,7 @@ "typing_tok_Ex07d.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "43e7aeffbe3192675cce06355d5cc5b1" + "71e8f08708092b76a261e705ab1d27b8" ], [ "Ex07d.typed_step", @@ -893,7 +893,7 @@ "subterm_ordering_Ex07d.EApp", "subterm_ordering_Ex07d.EIf" ], 0, - "7ccebd1c4ee45684a1ef651681cddee3" + "bb094ae28170c7ff8822505fe1092446" ], [ "Ex07d.step", @@ -913,7 +913,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "e7898ee751fee53860f795c0cd832f39" + "03f1ec48f6d58a9fe6a1579abbef075d" ], [ "Ex07d.extend", @@ -948,7 +948,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "928a8477a9b225ab15befcc301d5c627" + "baeabe23680146795083028d4ecbcd55" ], [ "Ex07d.appears_free_in", @@ -967,7 +967,7 @@ "subterm_ordering_Ex07d.EApp", "subterm_ordering_Ex07d.EIf" ], 0, - "c6b69783963754fd6e51a14b7a4fa7d2" + "6b8b718b1630159556f1e059628a22d7" ], [ "Ex07d.equal", @@ -1070,7 +1070,7 @@ "typing_tok_Ex07d.TBool@tok", "unit_typing" ], 0, - "39fdb1312c1eca1841bfd2c346cd25c5" + "8cd8618cfb4facf53d53735e8a44f965" ], [ "Ex07d.preservation", @@ -1130,7 +1130,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "bc8153ad553f896955a8707ad011573e" + "9dbc67270704f34f321314d85a4bc314" ], [ "Ex07d.typed_step", diff --git a/doc/tutorial/code/exercises/Ex11a.fst.hints b/doc/tutorial/code/exercises/Ex11a.fst.hints index 48a7526cc9e..cb0f956dda9 100644 --- a/doc/tutorial/code/exercises/Ex11a.fst.hints +++ b/doc/tutorial/code/exercises/Ex11a.fst.hints @@ -919,7 +919,7 @@ "subterm_ordering_Ex11a.Cons" ], 0, - "1e8aad52c685464c7094651fa06fd963" + "ab5f42f446164bcb021818544508937c" ], [ "Ex11a.lemma_mem_rid", @@ -1373,7 +1373,7 @@ "subterm_ordering_Ex11a.Cons" ], 0, - "4836912d752681592062b3a1e0d93c35" + "638036cb02a8b0c84c13cfeb5c90b9c3" ], [ "Ex11a.lemma_bots_tl_disjoint", diff --git a/doc/tutorial/code/exercises/LowStar.Ex2.fst.hints b/doc/tutorial/code/exercises/LowStar.Ex2.fst.hints index 2e34e046b29..d7b335b240f 100644 --- a/doc/tutorial/code/exercises/LowStar.Ex2.fst.hints +++ b/doc/tutorial/code/exercises/LowStar.Ex2.fst.hints @@ -23,7 +23,7 @@ "refinement_interpretation_LowStar.Ex2_Tm_refine_e295d1a089abf8fd7758b0cf33f12cde" ], 0, - "f1ff3ce195d5eef1585bc86b8b85fe03" + "cbcb476f06b78263e417338dcd4ebdaf" ], [ "LowStar.Ex2.prefix_equal", @@ -47,7 +47,7 @@ "refinement_interpretation_LowStar.Ex2_Tm_refine_e295d1a089abf8fd7758b0cf33f12cde" ], 0, - "4a24ef2a74aeafb5862fe51ff5064164" + "2087073d6c72ccb4a9b9c680b01db3bc" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/exercises/LowStar.Ex3.fst.hints b/doc/tutorial/code/exercises/LowStar.Ex3.fst.hints index 58ff2e6879e..6ab3b10e6c2 100644 --- a/doc/tutorial/code/exercises/LowStar.Ex3.fst.hints +++ b/doc/tutorial/code/exercises/LowStar.Ex3.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq" ], 0, - "d5c47665922c003c0c15c94fd87fde5f" + "b21608a6734928cb55101f8b955ca6f2" ], [ "LowStar.Ex3.repr", @@ -55,7 +55,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "f27efab94a59dc6b0d7d8f9c6318aff2" + "229b79d57cac4e1e0cd2156013098663" ], [ "LowStar.Ex3.pop", @@ -84,7 +84,7 @@ "typing_LowStar.Buffer.get" ], 0, - "39c9d1884c6472391038b0a000fc9cdd" + "94e12e482c0193e08c3ca6ff3d31b86c" ], [ "LowStar.Ex3.ok", @@ -93,7 +93,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq" ], 0, - "7931ef5d71ff35a9e331e0e7acd36151" + "f9885c0cd199cd916a3acd15de5d2efa" ], [ "LowStar.Ex3.repr", @@ -140,7 +140,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "2921750acfddf7786e24ebd1c49096bd" + "72200ba68959bc67ebd275a0b5592f98" ], [ "LowStar.Ex3.pop", @@ -169,7 +169,7 @@ "typing_LowStar.Buffer.get" ], 0, - "4ed8f175b0d1d3d7f1852e0e5d337b02" + "920e780c06a90898fb2376ca5919ce19" ], [ "LowStar.Ex3.malloc", @@ -186,7 +186,7 @@ "refinement_interpretation_LowStar.Ex3_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "be07695a5b486fcca70fe8124888756c" + "6095475ef20811d56f6d5b8e44c605c7" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex03a.fst.hints b/doc/tutorial/code/solutions/Ex03a.fst.hints index d6193c069af..ef8af6b6bf5 100644 --- a/doc/tutorial/code/solutions/Ex03a.fst.hints +++ b/doc/tutorial/code/solutions/Ex03a.fst.hints @@ -15,7 +15,7 @@ "well-founded-ordering-on-nat" ], 0, - "b6687cbc476fd20d31713c942f9711a8" + "76e3147de1d785692c5752d090cd976c" ], [ "Ex03a.factorial", @@ -31,7 +31,7 @@ "well-founded-ordering-on-nat" ], 0, - "dae73103b13efa0e57bbb6d6fa73a752" + "61401b1e8c4405bd2c79cca75fdba980" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex03b.fst.hints b/doc/tutorial/code/solutions/Ex03b.fst.hints index 7f3f58c4970..4c6458b76c0 100644 --- a/doc/tutorial/code/solutions/Ex03b.fst.hints +++ b/doc/tutorial/code/solutions/Ex03b.fst.hints @@ -16,7 +16,7 @@ "well-founded-ordering-on-nat" ], 0, - "2408f85d7e8cc5f0aa88e1701d99522f" + "91de9ced2c080bd68ebb1502e78bbd25" ], [ "Ex03b.fibonacci", @@ -34,7 +34,7 @@ "well-founded-ordering-on-nat" ], 0, - "05a6ebd478af50eeba0df27997ca112b" + "aac1716a784c61baa5b1e57717e8c3fa" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex03c.fst.hints b/doc/tutorial/code/solutions/Ex03c.fst.hints index ae0249b5378..68fb97dd2bc 100644 --- a/doc/tutorial/code/solutions/Ex03c.fst.hints +++ b/doc/tutorial/code/solutions/Ex03c.fst.hints @@ -17,7 +17,7 @@ "well-founded-ordering-on-nat" ], 0, - "936f98103cc4eda3bf0b1856bc235614" + "9cc88b34cb5f10aab469bda51d8ef760" ], [ "Ex03c.fibonacci_greater_than_arg", @@ -43,7 +43,7 @@ "well-founded-ordering-on-nat" ], 0, - "725b83aaf5b8ba38cdb26cae50e018de" + "15a6b13adb2ce5a21d796329c2c2b2c3" ], [ "Ex03c.fibonacci", @@ -61,7 +61,7 @@ "well-founded-ordering-on-nat" ], 0, - "ad197d371f1a744776d9bb198bb65f92" + "26a2d1520507928b65896d84a3c4d97e" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex04a.fst.hints b/doc/tutorial/code/solutions/Ex04a.fst.hints index 4e34e591ee4..b51ea2f53c6 100644 --- a/doc/tutorial/code/solutions/Ex04a.fst.hints +++ b/doc/tutorial/code/solutions/Ex04a.fst.hints @@ -16,7 +16,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "fab9dc3186a6c9366e799e337907ddd8" + "8ec752beaf705eb747b1ed9629bfb008" ], [ "Ex04a.append", @@ -57,7 +57,7 @@ "typing_Ex04a.length" ], 0, - "e1e2d0653c0eaef78dbb533e06d89efe" + "36e01b5d65d8bcb4e343c8f21fc35fb8" ], [ "Ex04a.length", @@ -74,7 +74,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "f40d1e753736452497a51a6a1b0ffc57" + "614012e71dd23a5716dd5f74fc157952" ], [ "Ex04a.append", @@ -104,7 +104,7 @@ "subterm_ordering_Prims.Cons", "typing_Ex04a.length" ], 0, - "9b63ad314eee60f0d4212f66b74912f1" + "b82bc5a6fb0d529bfc2d96cdfedaaec3" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex04b.fst.hints b/doc/tutorial/code/solutions/Ex04b.fst.hints index d0e3561c3ac..34ad369fd4c 100644 --- a/doc/tutorial/code/solutions/Ex04b.fst.hints +++ b/doc/tutorial/code/solutions/Ex04b.fst.hints @@ -16,7 +16,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "d02d6627e3f392b08c9e8ce1c5230a3b" + "1440708be33e0e7b3c2ce24d8104aa8f" ], [ "Ex04b.append", @@ -31,7 +31,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "9f5b23ca8b769b5039d84b242d12b095" + "7d6dc0fadd12b74725dc84a28134d931" ], [ "Ex04b.append_len", @@ -89,7 +89,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "4f9cc9aa9b1e2d4361a997480a5bcdf6" + "a647932d13e647dc1426ef37dab7c207" ], [ "Ex04b.append", @@ -103,7 +103,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "8e8f4e1313cf6ef31aa23baff446a2e7" + "4ee2c0e5c3321eda5a7f1f639791dde0" ], [ "Ex04b.append_len", diff --git a/doc/tutorial/code/solutions/Ex04c.fst.hints b/doc/tutorial/code/solutions/Ex04c.fst.hints index 7d36158aa2c..23fafd7b4c9 100644 --- a/doc/tutorial/code/solutions/Ex04c.fst.hints +++ b/doc/tutorial/code/solutions/Ex04c.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "ffc55c0c4e9a74e9122a70f26ef7940c" + "a02ed18a045b3fa57772585d87c790e0" ], [ "Ex04c.mem", @@ -28,7 +28,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "e91339b1985f802aeaa5ecc7af66a197" + "9ea824ec7485db8d46127e56de19f6b6" ], [ "Ex04c.append_mem", @@ -75,7 +75,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "5dea882f95f6ca070c49e97298ddde11" + "da9e505048fa8717fc1de02a62144701" ], [ "Ex04c.mem", @@ -90,7 +90,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "0fc94b19d07b04c41f878920cdfcc97e" + "2fbc8381185842c4bd8812b3de9f9282" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex04e.fst.hints b/doc/tutorial/code/solutions/Ex04e.fst.hints index e8cec5e381e..596f4f4363a 100644 --- a/doc/tutorial/code/solutions/Ex04e.fst.hints +++ b/doc/tutorial/code/solutions/Ex04e.fst.hints @@ -37,7 +37,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "7661577b25a2381221ddba29b72ba14e" + "8e3a6f79a5614d24c59b3801d0640ac6" ], [ "Ex04e.find'", @@ -52,7 +52,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "2be959cd8236e39a7226c42d5710c901" + "32cbd9eead24b5f986d610b9b264e649" ], [ "Ex04e.find_some", @@ -170,7 +170,7 @@ "projection_inverse_BoxBool_proj_0", "subterm_ordering_Prims.Cons" ], 0, - "d78c66900317cffceb13e0d2fa8b3e4b" + "ebf65d5a03e06741448726c081f744de" ], [ "Ex04e.find'", @@ -184,7 +184,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "5a058abb8e5a41de3b0683d7fefeccfe" + "f8f607553d7a6f2c6678deeafbb1923a" ], [ "Ex04e.find_some", diff --git a/doc/tutorial/code/solutions/Ex04f.fst.hints b/doc/tutorial/code/solutions/Ex04f.fst.hints index 73c3c143180..907d71ca85e 100644 --- a/doc/tutorial/code/solutions/Ex04f.fst.hints +++ b/doc/tutorial/code/solutions/Ex04f.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "4eddcbe68310e4ec8e460fa8448609ed" + "72289b094b51196f4dcf1b5a14a9d2e3" ], [ "Ex04f.reverse", @@ -27,7 +27,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "2dc89dc48e7f9ebcca8f08a34cf8c1cf" + "f68990e2e8b7ec4900d5f63d3c571399" ], [ "Ex04f.fold_left", @@ -42,7 +42,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "6e48976068f2500fce8b7af5e67ad6c3" + "3dae7e558f2c92bbd0e64ce17c7134e0" ], [ "Ex04f.append_assoc", @@ -92,7 +92,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "3f34a4511b36b1714cb16d1161bdfb93" + "17b90589e02b9ce32159cef45ab68002" ], [ "Ex04f.append", @@ -106,7 +106,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "20ea5b11b1038d0b334e8755ee01e24d" + "77b3b3b8ab9b9a60c527b1617bdfb751" ], [ "Ex04f.reverse", @@ -120,7 +120,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "504a378e415fdfd37ae54b7de9b20a06" + "e0c504f806c0abdff6f074ac15890919" ], [ "Ex04f.fold_left", @@ -134,7 +134,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "72f996301b861803c50231db35ec6990" + "bca687cb97068c637d0ebb9680467725" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex04h.fst.hints b/doc/tutorial/code/solutions/Ex04h.fst.hints index c050a943d33..b2eda3df3f2 100644 --- a/doc/tutorial/code/solutions/Ex04h.fst.hints +++ b/doc/tutorial/code/solutions/Ex04h.fst.hints @@ -16,7 +16,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "989de913748697fe678dfcf56905ba94" + "7e73d3543b8afad1a375c471eaa4193c" ], [ "Ex04h.nth", @@ -43,7 +43,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "9f540db452a5aabb8923bbbf49da4b21" + "851bb0b0a9e9019331c5d286baf86e73" ], [ "Ex04h.length", @@ -60,7 +60,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "49296d445f47fa535f635d7b1e58b210" + "e62fe9fc90fc3abd096ae28066e0c601" ], [ "Ex04h.nth", @@ -89,7 +89,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "301047ebe95b1db2c730765073aa9cf7" + "39d5dfd78e917cc1dc696c9af8fccad2" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex05a.fst.hints b/doc/tutorial/code/solutions/Ex05a.fst.hints index 374d381140d..cdd37395244 100644 --- a/doc/tutorial/code/solutions/Ex05a.fst.hints +++ b/doc/tutorial/code/solutions/Ex05a.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "314bdb51b5142a141cccd4ea6d59e5c3" + "78f442075beb1f149c88bf49f3f7ce0f" ], [ "Ex05a.reverse", @@ -27,7 +27,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "cb42482a295f6d5bfab4139d7cb3b4e0" + "6ff7a998392647d5a6c13b5e5da50569" ], [ "Ex05a.rev", @@ -42,7 +42,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "239646108938d77861f9fa992a334631" + "123020bf33ba9a1d7994eb890d2c984c" ], [ "Ex05a.append_assoc", @@ -136,7 +136,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "904f3683ab32fca6aed63c6a00d5f965" + "28c911dbd4ba428b488cc54b827178e8" ], [ "Ex05a.reverse", @@ -150,7 +150,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "9ce09e1a9cd910f374a2ac249e64ceaa" + "91b403e83f6bde88e8bf8bd65df632f5" ], [ "Ex05a.rev", @@ -165,7 +165,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "9a6402bd23e0769e84d3ecd64c443ec2" + "786d54e2cc70c29688b1dd99d6379247" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex05b.fst.hints b/doc/tutorial/code/solutions/Ex05b.fst.hints index 7f7959bd728..2ce558e33ef 100644 --- a/doc/tutorial/code/solutions/Ex05b.fst.hints +++ b/doc/tutorial/code/solutions/Ex05b.fst.hints @@ -17,7 +17,7 @@ "well-founded-ordering-on-nat" ], 0, - "119128aa621c5bd54da8960e175199d0" + "e82513efc45e644b87153b95ef00e167" ], [ "Ex05b.fib", @@ -37,7 +37,7 @@ "well-founded-ordering-on-nat" ], 0, - "f7f1d31925eda0efd4bf3a09d3ea3efa" + "a0519c2f42fff1155377c627f20a84dc" ], [ "Ex05b.fib_is_ok_aux", @@ -86,7 +86,7 @@ "typing_Ex05b.fibonacci", "well-founded-ordering-on-nat" ], 0, - "60ff5ef5298b4fbe27c49552b52d8526" + "d3e8bdf3a8f9c8b9336bb891167a5a75" ], [ "Ex05b.fib_is_ok", @@ -135,7 +135,7 @@ "well-founded-ordering-on-nat" ], 0, - "931a9ed28522450bd94396f9d4071e70" + "d619cd2df2a0d22728b95dabbf2222d3" ], [ "Ex05b.fib_inner_aux_2", @@ -173,7 +173,7 @@ "typing_Ex05b.fibonacci", "well-founded-ordering-on-nat" ], 0, - "d7964212ea2e801b01128ee283e22d6f" + "d3a94304e2f71839eb1228b177b31603" ], [ "Ex05b.fibonacci", @@ -191,7 +191,7 @@ "well-founded-ordering-on-nat" ], 0, - "665c1d1b3502e220e905e850dd420d05" + "a1b40816e1a8ad1cd22c92a1579d6cdd" ], [ "Ex05b.fib", @@ -211,7 +211,7 @@ "well-founded-ordering-on-nat" ], 0, - "afb1ed616247425d0760b64608f99f66" + "4d1c03c7a232ea8a6bcfa4ab200f0345" ], [ "Ex05b.fib_is_ok_aux", @@ -242,7 +242,7 @@ "typing_Ex05b.fibonacci", "well-founded-ordering-on-nat" ], 0, - "4be6c5121b13c53fbbc9aa2bda902d94" + "66408137acf5134bfc4ef672c7d4526a" ], [ "Ex05b.fib_is_ok", @@ -271,7 +271,7 @@ "well-founded-ordering-on-nat" ], 0, - "8f4fb76926401e5cc3630dcfceeed1ef" + "ce2b0ee1c2e192a7e97eb69f5bd6c1bb" ], [ "Ex05b.fib_inner_aux_2", @@ -297,7 +297,7 @@ "typing_Ex05b.fibonacci", "well-founded-ordering-on-nat" ], 0, - "e84aec29e49e54c0bbd735fd322444a9" + "732dbb2f7a863213ffcb029d225b689f" ], [ "Ex05b.fib_inner_aux_2", diff --git a/doc/tutorial/code/solutions/Ex06a.fst.hints b/doc/tutorial/code/solutions/Ex06a.fst.hints index 727e04e4bbb..3ea2086bcc0 100644 --- a/doc/tutorial/code/solutions/Ex06a.fst.hints +++ b/doc/tutorial/code/solutions/Ex06a.fst.hints @@ -14,7 +14,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "2c9535e4864fd8bfe8f5c598f934babb" + "f9b922eba63ad1e22a54c81c4e6f2658" ], [ "Ex06a.partition", @@ -28,7 +28,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "4f520729cdb25faa95993e52a9e9d581" + "9037c92ebcff282c60164808fc003bbb" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex06b.fst.hints b/doc/tutorial/code/solutions/Ex06b.fst.hints index 10dc2a1c59b..793eb680946 100644 --- a/doc/tutorial/code/solutions/Ex06b.fst.hints +++ b/doc/tutorial/code/solutions/Ex06b.fst.hints @@ -14,7 +14,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "2ff60d0298cc0e28142e9e52cabc37ec" + "79e355fa114904831465b67933e0c610" ], [ "Ex06b.append", @@ -29,7 +29,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "ac24ab1c057ebb31a79189fd2e7a673a" + "d7bc7bf7280b3bfe0dca6e3024d28ed9" ], [ "Ex06b.append_mem", @@ -85,7 +85,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "90d4e2a77c6a4602fbc0cf9b30d4fa6b" + "9b14f9ac63e084b15cb15bd8912e43d5" ], [ "Ex06b.sorted", @@ -104,7 +104,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "765e09e3f1da1bba6b7e8747f2d79ad0" + "b32ed1f54c9568bf1e2ecdc3ebc10af2" ], [ "Ex06b.partition", @@ -119,7 +119,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "596532e3b96f2f9d14a85518f724a625" + "d45e47654ab2c6a397f43e884d0b19d3" ], [ "Ex06b.partition_lemma", @@ -305,7 +305,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "333a9d95f21a5083641dd4357a6dc3eb" + "4128000f36c66beb9bacd68ec84d5751" ], [ "Ex06b.mem", @@ -320,7 +320,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "d61e5fb5a8a47c7161f3266c95ece8d6" + "96cfe73d62885d9d1b7cb55dedf66a9c" ], [ "Ex06b.append", @@ -334,7 +334,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "b818a473acc5e87ab63c8c06d9623dd4" + "f1960f54f03134466dfde2f3f07185fb" ], [ "Ex06b.append_mem", @@ -360,7 +360,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "8505ed8833e5c7997bfd785ddb861ae7" + "1fe9eada3e39cd693b077158ec7160c0" ], [ "Ex06b.sorted", @@ -378,7 +378,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "3bad1751eadabcf3e7eef367903232c9" + "f14c31775f77cf7b2db73079a879069e" ], [ "Ex06b.partition", @@ -392,7 +392,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "8973d11294c5d7fbc21e67069ae8556e" + "4a8f5cf592310b7553632e05cc1debb4" ], [ "Ex06b.partition_lemma", @@ -473,7 +473,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "09f0eb9838cc770b04024590e10d2179" + "f038cca4c9f6dc4839bd540d035a3415" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex06c.fst.hints b/doc/tutorial/code/solutions/Ex06c.fst.hints index 91856ef9225..f9f2a74d725 100644 --- a/doc/tutorial/code/solutions/Ex06c.fst.hints +++ b/doc/tutorial/code/solutions/Ex06c.fst.hints @@ -14,7 +14,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "dd61e6537971ea31a4fe08366bdcffb4" + "5105f34823432108930bdff964d24045" ], [ "Ex06c.append", @@ -29,7 +29,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "30d928dfe2eab14485c24557d68cf6ff" + "69999ae8b879306b30a1df12e7a5d92c" ], [ "Ex06c.append_mem", @@ -87,7 +87,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "24a170db6c86c7303a92ba8b811eac4d" + "a4e87728476a6ceba8c557d78d43ea18" ], [ "Ex06c.sorted", @@ -106,7 +106,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "99888001c2f1f1fcb482aef7d98169df" + "efb030de5fd4c46da998f7ca98d39503" ], [ "Ex06c.partition", @@ -121,7 +121,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "37e52fae4a117e9893e9c79d66dad339" + "1e6cf785c86f0f00fa33909255a4a552" ], [ "Ex06c.partition_lemma", @@ -297,7 +297,7 @@ "typing_Ex06c.sorted", "typing_Prims.__proj__Cons__item__tl" ], 0, - "d031d6c8a1b3bbe36d1286ebbdd01deb" + "2bc7ace4359588d79ca47f27117db880" ], [ "Ex06c.sort", @@ -379,7 +379,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "d73dc5e092bd106902eb4a704c725b09" + "4afa1f387e0615219efc696a081466ff" ], [ "Ex06c.mem", @@ -394,7 +394,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "de8d056b6403ea85540e2d57ed3ffcf5" + "c740957df54bac040bed450d5e91df5b" ], [ "Ex06c.append", @@ -408,7 +408,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "2e19a3eb87d5d2d3313942d5febb6c5d" + "227bd0a09ab99dea4bbc82c902f30522" ], [ "Ex06c.append_mem", @@ -434,7 +434,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "c72c6e86761dd3221002142da36bc5e9" + "6fbbb049823225dcbd4d845cbe19a38b" ], [ "Ex06c.sorted", @@ -452,7 +452,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "f4cef9338c9500dccea59156df437ed0" + "99adbfe838c8ebe8e63b64aa802663e7" ], [ "Ex06c.partition", @@ -466,7 +466,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "74eb83b99eafff95634cdc00aaabfa10" + "6e810c65b2c2d04dcc83481dd3dcb13a" ], [ "Ex06c.partition_lemma", @@ -570,7 +570,7 @@ "typing_Ex06c.sorted", "typing_Prims.__proj__Cons__item__tl" ], 0, - "dd77eff25ff79b8a66f5c7b827824d4c" + "535658590dd17182809f2f7a8ed42650" ], [ "Ex06c.sort", @@ -634,7 +634,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "527b0015847042f9126224634d2127dd" + "4176336db0d85ebf9730993e5bfc60c1" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex06d.fst.hints b/doc/tutorial/code/solutions/Ex06d.fst.hints index c3796e1eef2..bc2d12f0c4c 100644 --- a/doc/tutorial/code/solutions/Ex06d.fst.hints +++ b/doc/tutorial/code/solutions/Ex06d.fst.hints @@ -19,7 +19,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "8a6503a28585d50f243c2ab9eef6a031" + "457ccf2fbb49955c8d324f76453b803c" ], [ "Ex06d.append", @@ -33,7 +33,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "f25668f9546616a7188d5c886307e41c" + "91e9cc555d6c5dc3002eea6791a8e69e" ], [ "Ex06d.append_count", @@ -125,7 +125,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "a17db9cd0d5bebc76897a9c2cddf49b4" + "11c86812e204b900cb7134f016f1f62c" ], [ "Ex06d.sorted", @@ -144,7 +144,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "5d0cdc697147149e5771077d2b674f65" + "c3a8236181559c309095fe8ca8857aef" ], [ "Ex06d.partition", @@ -158,7 +158,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "d419c75e97c5002f3368ae7136876ca8" + "2f82378269ab00659f4427061b3df354" ], [ "Ex06d.partition_lemma", @@ -342,7 +342,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "ba3078b7c9c474aeaa10526edd193241" + "659e944ee4534e09f7f78f4b2cf900c0" ], [ "Ex06d.count", @@ -362,7 +362,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "be94731e746314b3772023431c932f5b" + "fa00dac48d44461e92b8eefb8063c161" ], [ "Ex06d.append", @@ -376,7 +376,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "550f0b39f91a42d6c55f7a786226b82f" + "fae0a7f3714cecb2c02540235b56365c" ], [ "Ex06d.append_count", @@ -411,7 +411,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "218edccca0d583aa90090f02d954a711" + "d5e3eda2c65372ae106d703237c80f30" ], [ "Ex06d.sorted", @@ -429,7 +429,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "30271f5408cd42c360c59f4e22ebc806" + "db273b1d3622dddc2c3b4b1d8338a866" ], [ "Ex06d.partition", @@ -443,7 +443,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "f6b17231b264ebf489958b530fcf3b5a" + "edd31ff2c5a44c39af721a6dd4456277" ], [ "Ex06d.partition_lemma", @@ -511,7 +511,7 @@ "typing_FStar.Pervasives.Native.snd", "well-founded-ordering-on-nat" ], 0, - "5f7b6ad90e80735187946a3218851759" + "342ae9f9a6d2d2441ba36a3485fdb342" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex06e.fst.hints b/doc/tutorial/code/solutions/Ex06e.fst.hints index dc6a787f743..267bce69f02 100644 --- a/doc/tutorial/code/solutions/Ex06e.fst.hints +++ b/doc/tutorial/code/solutions/Ex06e.fst.hints @@ -17,7 +17,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "9b7137e8b518de48dd4a1ee72927972c" + "2f195d592e90253eb34371d21f2480f8" ], [ "Ex06e.mem", @@ -36,7 +36,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "46b254d8093b332b4e6498d301f341eb" + "823f31acf50513706aea3d08582e6b32" ], [ "Ex06e.sorted_smaller", @@ -106,7 +106,7 @@ "typing_Ex06e.mem", "typing_Ex06e.sorted" ], 0, - "a231e2cf62acb8ceaf4b415d21e2846c" + "523d875516bca890d9ca43825af52941" ], [ "Ex06e.sort", @@ -139,7 +139,7 @@ "typing_Ex06e.mem", "typing_Ex06e.sorted" ], 0, - "b9666a1987217a73740f71f9b35ed0fe" + "13dfd5c3b4fd0e27dad97a176a256cb4" ], [ "Ex06e.sorted", @@ -157,7 +157,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "de26bb0af278e1a3a44156f37c77c998" + "4b7ba6732093d39e2323b2944d574439" ], [ "Ex06e.mem", @@ -176,7 +176,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "7104ea107a0d9a036454fff472705004" + "9b0b84ea4a2423f8368e6b9e8b466798" ], [ "Ex06e.insert", @@ -216,7 +216,7 @@ "typing_Ex06e.insert", "typing_Ex06e.mem", "typing_Ex06e.sorted" ], 0, - "ddd390d41266dd53159b4de5ec093ce7" + "61ad9201209e2e21240bdb8424630be6" ], [ "Ex06e.sort", @@ -247,7 +247,7 @@ "typing_Ex06e.mem" ], 0, - "94f840525c3aa173530498d9fa9b1ad8" + "54541c22194f1bd4a7f9af3f2acf7484" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex07a.fst.hints b/doc/tutorial/code/solutions/Ex07a.fst.hints index 79aaaac6457..0b65c537cd5 100644 --- a/doc/tutorial/code/solutions/Ex07a.fst.hints +++ b/doc/tutorial/code/solutions/Ex07a.fst.hints @@ -185,7 +185,7 @@ "subterm_ordering_Ex07a.EIf" ], 0, - "b44452ef1086dd06e882de352c0a49bb" + "249343498838f15207faf48ff451f17c" ], [ "Ex07a.step", @@ -205,7 +205,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "e1c90ca1d6083c5903bcaacfea40424f" + "e8e76e2b0bb70552cc952660a5a22783" ], [ "Ex07a.extend", @@ -240,7 +240,7 @@ "typing_tok_Ex07a.TBool@tok" ], 0, - "c5181f3c89df5d82f62a65463afc3bba" + "9a1e1ac6cca98b93201a82212e556752" ], [ "Ex07a.progress", @@ -326,7 +326,7 @@ "subterm_ordering_Ex07a.EApp", "subterm_ordering_Ex07a.EIf" ], 0, - "d2e797d302231cef9a11533c8c472a8f" + "e75cd01d12b0b24feffdcdbf44560bbd" ], [ "Ex07a.free_in_context", @@ -391,7 +391,7 @@ "typing_tok_Ex07a.TBool@tok" ], 0, - "f75db1287ae0bef52f47201997cb3cb9" + "ebb788d8ea72d3355a74d7badaee19a6" ], [ "Ex07a.typable_empty_closed", @@ -487,7 +487,7 @@ "typing_Ex07a.typing", "typing_tok_Ex07a.TBool@tok", "unit_typing" ], 0, - "5a956b80cc6857dd23061637eeb7a37d" + "fc1d10bbbe8237b5e784d81c60eceda9" ], [ "Ex07a.typing_extensional", @@ -842,7 +842,7 @@ "subterm_ordering_Ex07a.EApp", "subterm_ordering_Ex07a.EIf" ], 0, - "13f23d3298c143b210011ff765a68fd8" + "b6a2ef7fd9f2a83749394d273d9b41c7" ], [ "Ex07a.step", @@ -862,7 +862,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "4d2ef2e90892e42928d77926a29c31bf" + "e434826142495e5598f433c28136e0c8" ], [ "Ex07a.extend", @@ -897,7 +897,7 @@ "typing_tok_Ex07a.TBool@tok" ], 0, - "af0222316c52a55bc9eedd9323f05ce8" + "cb6f4e4b836f57d9e4db43be50a2302d" ], [ "Ex07a.appears_free_in", @@ -916,7 +916,7 @@ "subterm_ordering_Ex07a.EApp", "subterm_ordering_Ex07a.EIf" ], 0, - "8db234eb77057bf2c8c0112ba09f52a5" + "152ea8c28669cbfcb4f926e1137db5f5" ], [ "Ex07a.equal", diff --git a/doc/tutorial/code/solutions/Ex07b.fst.hints b/doc/tutorial/code/solutions/Ex07b.fst.hints index b5dd8fd72bd..c09825d1183 100644 --- a/doc/tutorial/code/solutions/Ex07b.fst.hints +++ b/doc/tutorial/code/solutions/Ex07b.fst.hints @@ -254,7 +254,7 @@ "subterm_ordering_Ex07b.EPair" ], 0, - "06cc5dd48d068f70d870941e0290e049" + "ecfe60b1734a2dbcc99b52eeae81d2ae" ], [ "Ex07b.subst", @@ -283,7 +283,7 @@ "subterm_ordering_Ex07b.EPair", "subterm_ordering_Ex07b.ESnd" ], 0, - "0de02043a327dec9fd53bb7ab2a6bc28" + "91fc297a867e7aabf1f52ff89654e1f2" ], [ "Ex07b.step", @@ -305,7 +305,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "34728210a9dc9139089f71d649bb1f9f" + "1fc8b3fca23178f4b09ae4181ffc260b" ], [ "Ex07b.extend", @@ -343,7 +343,7 @@ "typing_tok_Ex07b.TBool@tok" ], 0, - "60c0bfdffa2e3b7642574417a05ceca7" + "e367f44099d0e412acafb5826c8d3df4" ], [ "Ex07b.progress", @@ -454,7 +454,7 @@ "subterm_ordering_Ex07b.ESnd" ], 0, - "d111e82f4b20545ab8f2d758469a6ecf" + "7b494569fe6aab667fed730f3f917937" ], [ "Ex07b.free_in_context", @@ -533,7 +533,7 @@ "typing_tok_Ex07b.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "6a8ccc4a1e8557a183c8e573b9e9baad" + "dc479f1cfecf09d34a094fa787d13f59" ], [ "Ex07b.typable_empty_closed", @@ -640,7 +640,7 @@ "typing_Ex07b.typing", "typing_tok_Ex07b.TBool@tok", "unit_typing" ], 0, - "94bdd2b9cc124a7dc1fc8a90eff1630e" + "57e71a0b869dcff35644d6215465e4d4" ], [ "Ex07b.typing_extensional", @@ -749,7 +749,7 @@ "typing_tok_Ex07b.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "1d9ebe13f35823cc4d39ae712bd007e5" + "12498356219b4ee79e979546f8a6bf37" ], [ "Ex07b.preservation", @@ -839,7 +839,7 @@ "typing_tok_Ex07b.TBool@tok" ], 0, - "845beb1020a84b9a6ff4e97110168a7f" + "f1707902b97e75607930e137a7ac17b4" ], [ "Ex07b.ty", @@ -1094,7 +1094,7 @@ "subterm_ordering_Ex07b.EPair" ], 0, - "de2883fb3bfd65ab8432a3d12837f851" + "5217a371088e6c28725fe4a2ad9ff99f" ], [ "Ex07b.subst", @@ -1116,7 +1116,7 @@ "subterm_ordering_Ex07b.EPair", "subterm_ordering_Ex07b.ESnd" ], 0, - "42ecc76962406d0c10ce7a0c4b8f8527" + "9274c31f659a00d1e7a4c0bd7d015e76" ], [ "Ex07b.step", @@ -1138,7 +1138,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "eaef8f108e0935d1cbf81f57d0e46046" + "c7f09e355af99599d7d3006988cdf1ca" ], [ "Ex07b.extend", @@ -1176,7 +1176,7 @@ "typing_tok_Ex07b.TBool@tok" ], 0, - "b41af93dedaed4a52c349b2f9264d218" + "eed12a54496905ce58bfd1e8db8af7da" ], [ "Ex07b.appears_free_in", @@ -1198,7 +1198,7 @@ "subterm_ordering_Ex07b.EPair", "subterm_ordering_Ex07b.ESnd" ], 0, - "ba4c69a75decd8a91d33c0878d2ee507" + "00385231c8f832e85a4b95cf0302e79d" ], [ "Ex07b.equal", @@ -1311,7 +1311,7 @@ "typing_tok_Ex07b.TBool@tok", "unit_typing" ], 0, - "d044b17795d0ee7a69cd2ff9ed429340" + "48c7ef1c52ddc8a5f4927fc544eb666f" ], [ "Ex07b.preservation", @@ -1389,7 +1389,7 @@ "typing_tok_Ex07b.TBool@tok" ], 0, - "2482faf7b7476f38eccd9af83d0ae8d9" + "473d70910b2af6028f9b8fffb94b5cff" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex07c.fst.hints b/doc/tutorial/code/solutions/Ex07c.fst.hints index 1ce91dc4be4..c2a0713b66c 100644 --- a/doc/tutorial/code/solutions/Ex07c.fst.hints +++ b/doc/tutorial/code/solutions/Ex07c.fst.hints @@ -228,7 +228,7 @@ "subterm_ordering_Ex07c.ELet" ], 0, - "512ba5011384ff72102948ae0b5b5112" + "0b837cd8675a6506b4ec5ec3ed2af92f" ], [ "Ex07c.step", @@ -250,7 +250,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "123344c292dcf7c60ad5ebd0ac928082" + "d4ee22bd4e9c622d2e406566ad5e2293" ], [ "Ex07c.extend", @@ -286,7 +286,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "c85fc91e4a1828fe57b92818421f27c6" + "2ebf96830212fa71fc5d79557cd564a4" ], [ "Ex07c.progress", @@ -382,7 +382,7 @@ "subterm_ordering_Ex07c.ELet" ], 0, - "0b5023eac68e52e8b6ebc6ccbf2e9ece" + "61ca92b051c04c718446b4c965f31855" ], [ "Ex07c.free_in_context", @@ -453,7 +453,7 @@ "unit_inversion" ], 0, - "1d7855891cbc80804a369c93fcfbf8c9" + "33628a60bc281eaea872e56214138c4b" ], [ "Ex07c.typable_empty_closed", @@ -565,7 +565,7 @@ "typing_tok_Ex07c.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "fe8b87d78ad4fccbb7cd3c9823d47a84" + "42a251418b5e8694f8efcca4068682c8" ], [ "Ex07c.typing_extensional", @@ -675,7 +675,7 @@ "typing_tok_Ex07c.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "c8f0e1d3dcb32a231e8ff7dda01cb1dc" + "de58146cf8454302c130c15d94bcfcd2" ], [ "Ex07c.preservation", @@ -754,7 +754,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "9f5440308496887d54a14ea3d3825310" + "ff501aa1dc85c18594366f693f845302" ], [ "Ex07c.ty", @@ -977,7 +977,7 @@ "subterm_ordering_Ex07c.EIf", "subterm_ordering_Ex07c.ELet" ], 0, - "151ef0024cef8c6367a9473966d39a47" + "dc8d6af536c5158c5be80f12f60eddda" ], [ "Ex07c.step", @@ -998,7 +998,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "c4a4590de4b5e7994fb480308c3e65c1" + "f8d6eece0f9e17a986bb65d3a86f1268" ], [ "Ex07c.extend", @@ -1034,7 +1034,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "48b09b2013f565196065080a11318e84" + "722f659edac9cf0f2f816eda23c0f7ac" ], [ "Ex07c.appears_free_in", @@ -1054,7 +1054,7 @@ "subterm_ordering_Ex07c.EIf", "subterm_ordering_Ex07c.ELet" ], 0, - "7c2e7661e17b7fdfa95c7f4434e934ff" + "9ce9189209a525eded2e176c5933f408" ], [ "Ex07c.equal", @@ -1168,7 +1168,7 @@ "typing_tok_Ex07c.TBool@tok", "unit_typing" ], 0, - "b42b566dfa15a28b6001d7d0f132e1e2" + "76173ffdb57577fb90b68f3bab7778e6" ], [ "Ex07c.preservation", @@ -1235,7 +1235,7 @@ "typing_tok_Ex07c.TBool@tok" ], 0, - "83fa442e9b6c4d24cc57ce64225a5bee" + "f6b57dc513acb630e52db626f5dcbd00" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/Ex07d.fst.hints b/doc/tutorial/code/solutions/Ex07d.fst.hints index 3cf460db03e..9358203dcb9 100644 --- a/doc/tutorial/code/solutions/Ex07d.fst.hints +++ b/doc/tutorial/code/solutions/Ex07d.fst.hints @@ -185,7 +185,7 @@ "subterm_ordering_Ex07d.EIf" ], 0, - "653d6d39f830302d1535fe18cf06b463" + "74376ad328b0c258de301c1d16aa6583" ], [ "Ex07d.step", @@ -205,7 +205,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "c160cc089ebf576391c771c8e87c5e11" + "b0b61cf5aacff6e29ec8529dbbb40b22" ], [ "Ex07d.extend", @@ -240,7 +240,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "b9229ada7d86eaeca59926ad59a02fc1" + "1007c5280749da930340cf2bc48bd22a" ], [ "Ex07d.progress", @@ -326,7 +326,7 @@ "subterm_ordering_Ex07d.EApp", "subterm_ordering_Ex07d.EIf" ], 0, - "3ba4a819d88785f1d9ee845c668cd741" + "83955281903f17556206bb8772d80a73" ], [ "Ex07d.free_in_context", @@ -391,7 +391,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "22964c3693b1ab7ff19472863bbd5418" + "d68746c3f051cadfec29154b0b1e6119" ], [ "Ex07d.typable_empty_closed", @@ -488,7 +488,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "faad885210a10d3c29edb7c94955cd73" + "05142b618e6b95d3aba51bd4448518f5" ], [ "Ex07d.typing_extensional", @@ -589,7 +589,7 @@ "typing_tok_Ex07d.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "362dbd74a050e0ae214b9d055a2c16df" + "38335670e3ba800f62cd8ba24a33883a" ], [ "Ex07d.preservation", @@ -666,7 +666,7 @@ "typing_tok_Ex07d.TBool@tok", "unit_inversion", "unit_typing" ], 0, - "43e7aeffbe3192675cce06355d5cc5b1" + "71e8f08708092b76a261e705ab1d27b8" ], [ "Ex07d.typed_step", @@ -989,7 +989,7 @@ "subterm_ordering_Ex07d.EApp", "subterm_ordering_Ex07d.EIf" ], 0, - "ddac5ba5faa3aa785178cf1b25a522bc" + "56285aad524c2357ff21ac826ca32ae1" ], [ "Ex07d.step", @@ -1009,7 +1009,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "5b5524e5cb41a0aae2f92fd140f97baa" + "311a9ed319b4035705ec17a57788271c" ], [ "Ex07d.extend", @@ -1044,7 +1044,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "682b9cb03674d79b857abe20cdb26f25" + "2b52c97f2707a566af3ddc16b9a593af" ], [ "Ex07d.appears_free_in", @@ -1063,7 +1063,7 @@ "subterm_ordering_Ex07d.EApp", "subterm_ordering_Ex07d.EIf" ], 0, - "a0a211826e3bbf7bebeec0f5151a422e" + "6984e36097b802d65c543821b964ccd2" ], [ "Ex07d.equal", @@ -1166,7 +1166,7 @@ "typing_tok_Ex07d.TBool@tok", "unit_typing" ], 0, - "59e22f197ee76a45462f68bf9b1d9563" + "22625a0c95ef5957f217c5350c6a34f3" ], [ "Ex07d.preservation", @@ -1226,7 +1226,7 @@ "typing_tok_Ex07d.TBool@tok" ], 0, - "51580d9690b0581cc5b286ccf7c9b743" + "ff5e477161cb366c65f2ccbc33a65782" ], [ "Ex07d.typed_step", diff --git a/doc/tutorial/code/solutions/Ex11a.fst.hints b/doc/tutorial/code/solutions/Ex11a.fst.hints index e0394103042..771e55ee850 100644 --- a/doc/tutorial/code/solutions/Ex11a.fst.hints +++ b/doc/tutorial/code/solutions/Ex11a.fst.hints @@ -916,7 +916,7 @@ "subterm_ordering_Ex11a.Cons" ], 0, - "1e8aad52c685464c7094651fa06fd963" + "5de05d164b600fbaa67882181d581c85" ], [ "Ex11a.lemma_mem_rid", @@ -1531,7 +1531,7 @@ "subterm_ordering_Ex11a.Cons" ], 0, - "c0cec488b22a3bc9e3503a365b443d53" + "f354294412f54b807aab651458ecbadc" ], [ "Ex11a.lemma_bots_tl_disjoint", diff --git a/doc/tutorial/code/solutions/LowStar.Ex2.fst.hints b/doc/tutorial/code/solutions/LowStar.Ex2.fst.hints index 77af9d5ee13..7831c5b10e0 100644 --- a/doc/tutorial/code/solutions/LowStar.Ex2.fst.hints +++ b/doc/tutorial/code/solutions/LowStar.Ex2.fst.hints @@ -48,7 +48,7 @@ "typing_LowStar.Monotonic.Buffer.loc_buffer" ], 0, - "5b88e69aa36a5dd95fe81787138d922e" + "14c8c930488af25989edc822dc3e97ec" ], [ "LowStar.Ex2.prefix_equal", @@ -72,7 +72,7 @@ "refinement_interpretation_LowStar.Ex2_Tm_refine_e295d1a089abf8fd7758b0cf33f12cde" ], 0, - "5aed8cc8e724549cb6089917f0399dae" + "b2910aa792f1f2851835eb9ce95c229f" ], [ "LowStar.Ex2.copy_correct", @@ -156,7 +156,7 @@ "typing_LowStar.Monotonic.Buffer.loc_buffer" ], 0, - "b673d6c5282245b1cdd6a5676eeab745" + "9a908f283a61ab2c50fa6a31d563d94b" ], [ "LowStar.Ex2.swap", @@ -172,7 +172,7 @@ "projection_inverse_FStar.Integers.Unsigned__0" ], 0, - "1b8cdfc26d256cd73ed45cfd29c2ce0e" + "caa6edbcb189354dcfa3192ced603cae" ], [ "LowStar.Ex2.prefix_equal", @@ -196,7 +196,7 @@ "refinement_interpretation_LowStar.Ex2_Tm_refine_e295d1a089abf8fd7758b0cf33f12cde" ], 0, - "949614abe068f814470d80dbf7ea0dc6" + "1dd20b338f1445ac79003d087c62948b" ], [ "LowStar.Ex2.copy_correct", @@ -209,7 +209,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "c52f4af11980fbd5af9d613eb0b78bb3" + "059db4684c486760072d482c6684c084" ] ] ] \ No newline at end of file diff --git a/doc/tutorial/code/solutions/LowStar.Ex3.fst.hints b/doc/tutorial/code/solutions/LowStar.Ex3.fst.hints index 0bb495a6628..1e6fde6fda9 100644 --- a/doc/tutorial/code/solutions/LowStar.Ex3.fst.hints +++ b/doc/tutorial/code/solutions/LowStar.Ex3.fst.hints @@ -12,7 +12,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_573cfed777dae20cc82e8fef9622857e" ], 0, - "fd396582463f63e9123e75619096c4dc" + "a603d3ce9227aea007d0478cf734173b" ], [ "LowStar.Ex3.ok", @@ -21,7 +21,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq" ], 0, - "69caa66538edeb8462ad182cae3734f3" + "99c1755e4c5aa36a55afe0b5de6a0be2" ], [ "LowStar.Ex3.repr", @@ -69,7 +69,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "227ac0c28c8b88c691ed6221df61a90f" + "cdc86f2be8d7f5be62199d5b43bf3a56" ], [ "LowStar.Ex3.full", @@ -83,7 +83,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "d28aa4453fbcdbc2be32b5d1307ad9e7" + "9dcc24bbe0b57481ed6cb64ff64e51dc" ], [ "LowStar.Ex3.pop", @@ -191,7 +191,7 @@ "typing_LowStar.Monotonic.Buffer.loc_union" ], 0, - "86bc83edb797e2146693a2da60b8fd8d" + "e0aa74025e361bb18119d839902a381c" ], [ "LowStar.Ex3.push", @@ -296,7 +296,7 @@ "typing_LowStar.Monotonic.Buffer.loc_buffer" ], 0, - "9b58e4de64307d3532e3416748fabc3e" + "ded0c8068fca632c8a02245b266a7d3d" ], [ "LowStar.Ex3.create", @@ -416,7 +416,7 @@ "typing_LowStar.Monotonic.Buffer.mgsub" ], 0, - "f78d683337a30edfd3be702636d31f99" + "8d14e9692c490f5e569c17a863086ab6" ], [ "LowStar.Ex3.main", @@ -508,7 +508,7 @@ "typing_LowStar.Monotonic.Buffer.length", "typing_Prims.pow2" ], 0, - "3483a06ec719f6477123e0f4c8af2498" + "da09c1915376b3421c80e7f3787c24b5" ], [ "LowStar.Ex3.deref", @@ -521,7 +521,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_573cfed777dae20cc82e8fef9622857e" ], 0, - "1c249e632cf5bffff84ef561d83c2dad" + "33f918f48289592ba1c7ae645c3d9089" ], [ "LowStar.Ex3.ok", @@ -530,7 +530,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq" ], 0, - "e6163843eef382c4eb82979111a8918d" + "8ef6d29310d587a6c712b238336476c5" ], [ "LowStar.Ex3.repr", @@ -578,7 +578,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "07559c7e014aada935ae1cf6f8fb6095" + "f596776b1f2181b5864e243bb6303c49" ], [ "LowStar.Ex3.repr", @@ -593,7 +593,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_573cfed777dae20cc82e8fef9622857e" ], 0, - "19fe45b5f16f7e15d4155ae044e59a67" + "b120e87fafa565b8019d93e4c69e1b93" ], [ "LowStar.Ex3.empty", @@ -608,7 +608,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_573cfed777dae20cc82e8fef9622857e" ], 0, - "2fd7282423add153561537589befd1b4" + "4ab1e0d7da1b381162e3c36cde645eb3" ], [ "LowStar.Ex3.full", @@ -622,7 +622,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "b01620da68f8ff223d1299fdcfc9eb8b" + "2b56cf9e65ad25ff5fcc436a2d090c93" ], [ "LowStar.Ex3.full", @@ -637,7 +637,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_573cfed777dae20cc82e8fef9622857e" ], 0, - "036ca03f62392e572d91eead9bdd1921" + "c2fccf5cdbecf35682fcc393a1b6cf62" ], [ "LowStar.Ex3.pop", @@ -667,7 +667,7 @@ "typing_LowStar.Monotonic.Buffer.get" ], 0, - "8bca263fb51113fc7e362e9df52a5913" + "8648c3eeb05e7768707c713672ee1b7f" ], [ "LowStar.Ex3.push", @@ -680,7 +680,7 @@ "refinement_interpretation_LowStar.Ex3_Tm_refine_652bbbdf45596729c838daeb8e71aa70" ], 0, - "2139dc747a22e614d531aef263433ceb" + "76b3316e421e6745075df9bdef2651ae" ], [ "LowStar.Ex3.malloc", @@ -697,7 +697,7 @@ "refinement_interpretation_LowStar.Ex3_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "c253bd9fa0a241daea815fefb2fd79b9" + "a67b81e0233e8fd5fbd909d2aa4b1a5c" ], [ "LowStar.Ex3.create", @@ -713,7 +713,7 @@ "projection_inverse_FStar.Integers.Unsigned__0" ], 0, - "e1a484252916dc57129723e914c5d181" + "72007854c5b3596b96cc2bd7e9474c75" ] ] ] \ No newline at end of file diff --git a/examples/algorithms/BinarySearch.fst.hints b/examples/algorithms/BinarySearch.fst.hints index 170b51c4f4b..1e069df35e9 100644 --- a/examples/algorithms/BinarySearch.fst.hints +++ b/examples/algorithms/BinarySearch.fst.hints @@ -23,7 +23,7 @@ "well-founded-ordering-on-nat" ], 0, - "0afb9dafc7433c27ffecb424f6a9719c" + "cce691a0bc51cde2a48ae5a756a00dc6" ], [ "BinarySearch.bsearch", @@ -81,7 +81,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "4500f7487ee6f9ab9eb20be913d2e3fd" + "d095d7c21ccc9ca1361fee18b1bc32a2" ], [ "BinarySearch.bsearch_correct", @@ -229,7 +229,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "35c358dc2fa362e638c3f0118804eb0d" + "1598c8832c69d1d0a8cb5448da0a46c3" ], [ "BinarySearch.bsearch_complete", @@ -279,7 +279,7 @@ "well-founded-ordering-on-nat" ], 0, - "e1e86b90c3eb9594fd9cdbd76cf0fb18" + "7d82fd851f258713951f2f2b49acddb3" ], [ "BinarySearch.bsearch", diff --git a/examples/algorithms/Huffman.fst.hints b/examples/algorithms/Huffman.fst.hints index 5890c16701b..9c4ae64859b 100644 --- a/examples/algorithms/Huffman.fst.hints +++ b/examples/algorithms/Huffman.fst.hints @@ -111,7 +111,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "1586e5ed7f1f76eff1e7f46523838e0d" + "c665b56964d1eb84470a80c5947c9a1c" ], [ "Huffman.permutation", @@ -212,7 +212,7 @@ "typing_Huffman.sorted" ], 0, - "e826509ee1c155ceeddb077beaa31d1c" + "c4b5403adcd0484e45eefbe88134bf01" ], [ "Huffman.insertion_sort", @@ -242,7 +242,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "d77d1e7858cd3792f501c22ca9491faa" + "0212ce2167043fe189ef9c43ebaa62c2" ], [ "Huffman.huffman_trie", @@ -292,7 +292,7 @@ "typing_Huffman.weight", "well-founded-ordering-on-nat" ], 0, - "16fb184244c2b6d87aff53620e78a567" + "0dbc2015c6687d436e7650ab0c165a13" ], [ "Huffman.huffman", @@ -346,7 +346,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "b54d441356eaa8e3cfe54910f9534e34" + "caa77e90c185a198aa83aff8b899396d" ], [ "Huffman.encode", @@ -395,7 +395,7 @@ "typing_FStar.Pervasives.Native.__proj__Some__item__v" ], 0, - "fc54725ac2464878a57d8c5aa595be41" + "eb3f75f6871bb26ba393844baa3619f6" ], [ "Huffman.decode_one", @@ -440,7 +440,7 @@ "subterm_ordering_Huffman.Node" ], 0, - "eea0196fdddd31419e10b037742b7d46" + "6523468d1e3ba1f110ac0a0c7aeb8814" ], [ "Huffman.decode'", @@ -483,7 +483,7 @@ "well-founded-ordering-on-nat" ], 0, - "8e95eb3549b8167047583264efdc3a1c" + "7a3ff22eea15c021502b35ff7c67aceb" ], [ "Huffman.decode_aux", @@ -540,7 +540,7 @@ "typing_Huffman.uu___is_Node", "well-founded-ordering-on-nat" ], 0, - "a117ed52d4958c30845aef9c0fc50c5e" + "1ad43ab1468f4329b617ad1d3713d969" ], [ "Huffman.decode", @@ -906,7 +906,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "9ea389c08da1d4b866c1872d9c03ce84" + "61d58610ce0e45b65fca6394e5120d12" ], [ "Huffman.permutation", @@ -998,7 +998,7 @@ "typing_Huffman.sorted" ], 0, - "f2224f7940c492df74f23477574f8fa9" + "0b4180dd362382e62632ecf61bead624" ], [ "Huffman.insertion_sort", @@ -1028,7 +1028,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "04c99cef8582b5ca3d8498da5830f225" + "d5183d6a36bbb550d4838987919e45bf" ], [ "Huffman.huffman_trie", @@ -1078,7 +1078,7 @@ "typing_Huffman.weight", "well-founded-ordering-on-nat" ], 0, - "0733ebb43832f8b44dcbc15836c1cfa4" + "8b6ea5641daab70f9c7b5f522b7c40fb" ], [ "Huffman.huffman", @@ -1128,7 +1128,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "50c99b7676bf5b7968c789978ffbd39c" + "8ca3f924cd28fe68b43ef747fc37dbbc" ], [ "Huffman.encode", @@ -1177,7 +1177,7 @@ "typing_FStar.Pervasives.Native.__proj__Some__item__v" ], 0, - "8b231c37de9fa6b6a04112fdd4679110" + "c21cc492688860967d9475150e4131d2" ], [ "Huffman.decode_one", @@ -1222,7 +1222,7 @@ "subterm_ordering_Huffman.Node" ], 0, - "d2f71a78907a3b09fd25a8308f4808e8" + "df18f77e712889548dbe61b26baf8bb0" ], [ "Huffman.decode'", @@ -1265,7 +1265,7 @@ "well-founded-ordering-on-nat" ], 0, - "d9632076bcdb24b39c7fd8320d49588f" + "911a13dcf427024121fd1099b333bf1a" ], [ "Huffman.decode_aux", @@ -1321,7 +1321,7 @@ "typing_Huffman.uu___is_Node", "well-founded-ordering-on-nat" ], 0, - "6aeab72126ffe6db386d0adf416b6e52" + "0e01adefa8f88611894f6bbd4208d2c7" ], [ "Huffman.decode", diff --git a/examples/algorithms/InsertionSort.fst.hints b/examples/algorithms/InsertionSort.fst.hints index cab18ff01a8..98381f21a75 100644 --- a/examples/algorithms/InsertionSort.fst.hints +++ b/examples/algorithms/InsertionSort.fst.hints @@ -38,7 +38,7 @@ "subterm_ordering_Prims.Cons", "typing_IntSort.sorted" ], 0, - "1c4ea081041afc9c3b1f0dcfb7297512" + "c1aa50ce183d58b9d118039c6bce8071" ], [ "InsertionSort.insert_implicit", @@ -75,7 +75,7 @@ "subterm_ordering_Prims.Cons", "typing_IntSort.sorted" ], 0, - "35c8bd124b34e5056868794b665f3829" + "e4f6a5d3f6fdc8887b109ea6719d4c26" ], [ "InsertionSort.sort", @@ -108,7 +108,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "e0b0b52d58aa48c1c5860d414ef342c3" + "c0286acc77dc8251ccadef35cc6fcb50" ], [ "InsertionSort.insert", @@ -149,7 +149,7 @@ "typing_IntSort.sorted" ], 0, - "bc94598a6f0509ce08f8b3667e4976ab" + "1a1975a459f931c0f402fc3b1e4403af" ], [ "InsertionSort.insert_implicit", @@ -186,7 +186,7 @@ "subterm_ordering_Prims.Cons", "typing_IntSort.sorted" ], 0, - "5a03186b34f30015cef8f089f526914d" + "a34d372b98168c0f7a4a8dfe0a6028e6" ], [ "InsertionSort.sort", @@ -219,7 +219,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "f5a83dd942caf994c6ff1dbea414e21a" + "f442582134d9514d8919a211bc9acedb" ] ] ] \ No newline at end of file diff --git a/examples/algorithms/IntSort.fst.hints b/examples/algorithms/IntSort.fst.hints index 6b51ada7104..1d1c1333a34 100644 --- a/examples/algorithms/IntSort.fst.hints +++ b/examples/algorithms/IntSort.fst.hints @@ -17,7 +17,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "2334fa44a94d0c65b487038b209cd4eb" + "e8ddafe97dc1e7c9ac05a94aa7b0662a" ], [ "IntSort.test_sorted", @@ -149,7 +149,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "9782ecd60b4ecdaa2ba87462b12a7c21" + "b8b288ac5473406b7515dff9b31d8a39" ], [ "IntSort.test_sorted", diff --git a/examples/algorithms/MergeSort.fst.hints b/examples/algorithms/MergeSort.fst.hints index 453ebc48824..bc71576d18d 100644 --- a/examples/algorithms/MergeSort.fst.hints +++ b/examples/algorithms/MergeSort.fst.hints @@ -45,7 +45,7 @@ "typing_Prims.__proj__Cons__item__tl", "typing_Prims.uu___is_Cons" ], 0, - "30ec7d0f7cb1f1c1fca0849e89f767b8" + "88a649b1992fc20896ba5395aa264a63" ], [ "MergeSort.merge_inv", @@ -103,7 +103,7 @@ "typing_FStar.List.Tot.Base.mem", "typing_IntSort.sorted" ], 0, - "a57dd8f718b053ef2a219fac81e8ea4a" + "605d9310f8bf634cda5df123e0db736b" ], [ "MergeSort.mergesort", @@ -142,7 +142,7 @@ "typing_Prims.__proj__Cons__item__tl", "well-founded-ordering-on-nat" ], 0, - "c85b5fe7b837a1031468e280b561191c" + "e23ad898f7c7c949841881611a6068f8" ], [ "MergeSort.split", @@ -188,7 +188,7 @@ "typing_Prims.__proj__Cons__item__tl", "typing_Prims.uu___is_Cons" ], 0, - "c2cb3424a41d6e27fb69c059bab8af1f" + "d7ff3ba9054386cbb5d8464aa71e8d8e" ], [ "MergeSort.merge_inv", @@ -247,7 +247,7 @@ "typing_FStar.List.Tot.Base.mem", "typing_IntSort.sorted" ], 0, - "5849a63bf016a7b9e1573b8e9bc47527" + "5f0263b7bc3fa5d2152caf76f73175c3" ], [ "MergeSort.mergesort", @@ -286,7 +286,7 @@ "typing_Prims.__proj__Cons__item__tl", "well-founded-ordering-on-nat" ], 0, - "60954f611f1e1557ec9ac422853029ae" + "7322ef81c75f7c7eb9d8f3cd8c4b24de" ] ] ] \ No newline at end of file diff --git a/examples/algorithms/QuickSort.List.fst.hints b/examples/algorithms/QuickSort.List.fst.hints index f25da985d9a..b6a10cb6b07 100644 --- a/examples/algorithms/QuickSort.List.fst.hints +++ b/examples/algorithms/QuickSort.List.fst.hints @@ -12,7 +12,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "a7902346730c9a65f29fb7e763850179" + "0a47bae42578677da3422db893f2e475" ], [ "QuickSort.List.count", @@ -33,7 +33,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "624f02f5ad0279f961630d4601a7ada1" + "39a2aaa0624b77b556b50d01590c6d2f" ], [ "QuickSort.List.mem_count", @@ -88,7 +88,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "096a273b6f5b7cc47ac4acef8aaa6d07" + "86206f991ffa460b9f182a7f39e81b21" ], [ "QuickSort.List.partition_lemma", @@ -343,7 +343,7 @@ "well-founded-ordering-on-nat" ], 0, - "835aaf6f4f88c7e89f25d1a749f031a0" + "2f707f81b8883753ece55e96a2bc2d05" ], [ "QuickSort.List.sorted", @@ -356,7 +356,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "0eedf0ee7ba053a4da2ea15e8b89f824" + "925fb0f7aff6bbf71edb2209107cc9f9" ], [ "QuickSort.List.count", @@ -377,7 +377,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "a6edbf3fff8b0c65149cf0d094f169d9" + "a36adeca263399f8561b238a75016a2c" ], [ "QuickSort.List.mem_count", @@ -400,7 +400,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "de9d144699cf437077367b828a3f818d" + "7aff191ae95aaeaf917cd961c90342c6" ], [ "QuickSort.List.partition_lemma", @@ -486,7 +486,7 @@ "well-founded-ordering-on-nat" ], 0, - "e1695cb36deaa41312d2a1c95d4f1b86" + "183dd631f272ff62f2fea1982c11b4c8" ] ] ] \ No newline at end of file diff --git a/examples/algorithms/QuickSort.Seq.fst.hints b/examples/algorithms/QuickSort.Seq.fst.hints index 6b5ef8341bf..9229616f132 100644 --- a/examples/algorithms/QuickSort.Seq.fst.hints +++ b/examples/algorithms/QuickSort.Seq.fst.hints @@ -80,7 +80,7 @@ "typing_FStar.Seq.Properties.mem", "well-founded-ordering-on-nat" ], 0, - "cbbc8ff7c805829bd51a2760baec5d33" + "8db77ae4508d993afce4917ac4caaf35" ], [ "QuickSort.Seq.sort", @@ -141,7 +141,7 @@ "typing_FStar.Seq.Properties.mem", "well-founded-ordering-on-nat" ], 0, - "98737ffb89dfc6872103dd50eb500489" + "09415cb45fda822d7279c3b557f5d8a1" ], [ "QuickSort.Seq.partition", @@ -213,7 +213,7 @@ "typing_FStar.Seq.Properties.mem", "well-founded-ordering-on-nat" ], 0, - "77c60eb0f1f97a03e3401eb54b59ff61" + "3c83468e3f910118413f0faf8c13dff3" ], [ "QuickSort.Seq.sort", @@ -274,7 +274,7 @@ "typing_FStar.Seq.Properties.mem", "well-founded-ordering-on-nat" ], 0, - "c7c43b8037fbc072e9baee22a16256b2" + "a343d25f24d9b59d1297c87eb86e7131" ] ] ] \ No newline at end of file diff --git a/examples/algorithms/Unification.fst.hints b/examples/algorithms/Unification.fst.hints index df325f59847..d408db0426a 100644 --- a/examples/algorithms/Unification.fst.hints +++ b/examples/algorithms/Unification.fst.hints @@ -157,7 +157,7 @@ "subterm_ordering_Unification.F" ], 0, - "e5ae546cd158ddafa68984fe1c385043" + "2c59c15c867a9551899e8c17b16a90c8" ], [ "Unification.evars", @@ -174,7 +174,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "a7cf5fb76f2133771ec03658fd462e70" + "96352e41d102849fba8d2d88c7b0cd30" ], [ "Unification.n_evars", @@ -203,7 +203,7 @@ "subterm_ordering_Unification.F" ], 0, - "f7d7b605af7fa4c5736baa5cd6259cfc" + "df1777fd06aaea557df944fa5e9c40e1" ], [ "Unification.efuns", @@ -222,7 +222,7 @@ "subterm_ordering_Prims.Cons", "typing_Unification.funs" ], 0, - "ae1c44903c72ff92f48e81eb34f78fbd" + "a43be9ae0f3607d0dd59ea0422955f2a" ], [ "Unification.n_flex_rhs", @@ -241,7 +241,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "555f0b1fbf5f859f5433f27392c207aa" + "0defd56967d68f0b6a7703b78c8b9e63" ], [ "Unification.subst_term", @@ -266,7 +266,7 @@ "subterm_ordering_Unification.F" ], 0, - "2fb720594dda5713d03679b3fb72721b" + "c087cbb65fd89fe868a4e385408a6d58" ], [ "Unification.occurs", @@ -293,7 +293,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "86c183dc0c5354e19a3b924f5f5a851a" + "9a6060ea98df3a0660a7f94ed4b1150f" ], [ "Unification.lemma_lsubst_eqns_nil", @@ -679,7 +679,7 @@ "typing_Unification.vars", "well-founded-ordering-on-nat" ], 0, - "78ae0e1126987ecd500b099017449e30" + "fdf297983f128485ffe7138640e421b3" ], [ "Unification.solved", @@ -695,7 +695,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "350899817fdd48e365568e061008297b" + "00d10386296c3b73f3b22b7293d2f14a" ], [ "Unification.lsubst_distributes_over_F", @@ -1658,7 +1658,7 @@ "well-founded-ordering-on-nat" ], 0, - "2e46ca702112dec4b312d4406332d950" + "abb0a6c0b9a682abe7e820b4e1aac672" ], [ "Unification.unify_eqns_correct", @@ -1813,7 +1813,7 @@ "subterm_ordering_Unification.F" ], 0, - "8234304769598f47d26f251983ae3fe3" + "b1574f07c5eb6cdf08cbf989d18395ac" ], [ "Unification.evars", @@ -1830,7 +1830,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "d0b2b090e4ae90c9f56e20e3ed0c7430" + "7af03cd646e536506b9cc2334bb9283b" ], [ "Unification.n_evars", @@ -1859,7 +1859,7 @@ "subterm_ordering_Unification.F" ], 0, - "c8543035c1e485a69543c1b89edd7d34" + "e77bb0f748f4be280b2b7797c4dba855" ], [ "Unification.efuns", @@ -1878,7 +1878,7 @@ "subterm_ordering_Prims.Cons", "typing_Unification.funs" ], 0, - "41d5f05ac239a834db850bbaa1ca635b" + "bf8bfe2ba46432be9073f0e0d7eaeb06" ], [ "Unification.n_flex_rhs", @@ -1897,7 +1897,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "1a1d4713cf22cdfedf1a0dab2e0780da" + "cc4715f26d8ba6d84741ef09c45154af" ], [ "Unification.subst_term", @@ -1922,7 +1922,7 @@ "subterm_ordering_Unification.F" ], 0, - "b3f5c968e6b8352b7618b3bb4b928a0a" + "917a771dae8692db59f109f7e29b252a" ], [ "Unification.occurs", @@ -1949,7 +1949,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "7ae44cddbbc5c423c30eabfc1137322b" + "95944e2fe2050dc0f1b9fd7c70b6390a" ], [ "Unification.lemma_lsubst_eqns_nil", @@ -2171,7 +2171,7 @@ "typing_Unification.vars", "well-founded-ordering-on-nat" ], 0, - "97e15bc07e0b7662b1d4cb7dbe7af8ec" + "0e1fbf29170bea136068b6feca5dd8da" ], [ "Unification.solved", @@ -2187,7 +2187,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "6ba22ef63158f2ad3f248612b9720b70" + "253a4556b764620ded6b95a6e22b77e8" ], [ "Unification.lsubst_distributes_over_F", @@ -2502,7 +2502,7 @@ "well-founded-ordering-on-nat" ], 0, - "6cf37051cf46efd2781db5eac7ab98c4" + "d9a313fc1b8aba0085acae0c5c78e818" ], [ "Unification.unify_eqns_correct", diff --git a/examples/bug-reports/Bug1423.fst.hints b/examples/bug-reports/Bug1423.fst.hints index 71cc317ee5f..ecd105c51b5 100755 --- a/examples/bug-reports/Bug1423.fst.hints +++ b/examples/bug-reports/Bug1423.fst.hints @@ -11,7 +11,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "1dc0dfa290a95009905b71f9dd375a9c" + "2d22bc28a647dc96bf4493cc66d4f425" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/Bug1502.fst.hints b/examples/bug-reports/Bug1502.fst.hints index 5f1e5a1e1ec..6efda271f1e 100644 --- a/examples/bug-reports/Bug1502.fst.hints +++ b/examples/bug-reports/Bug1502.fst.hints @@ -8,7 +8,7 @@ 0, [ "@query" ], 0, - "979c0e53e05d12b8dd4643619f3d33d1" + "7ff2e587c97867b657f454e11df6fa39" ], [ "Bug1502.disjoint", diff --git a/examples/bug-reports/Bug1536.fst.hints b/examples/bug-reports/Bug1536.fst.hints new file mode 100644 index 00000000000..9c6c2943e1c --- /dev/null +++ b/examples/bug-reports/Bug1536.fst.hints @@ -0,0 +1,61 @@ +[ + "Wd\u0006\u001fFQ", + [ + [ + "Bug1536.bind_ex", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Bug1536_interpretation_Tm_arrow_f2d128b41b807a50fc4bea0cd4f225d8", + "disc_equation_FStar.Pervasives.Inl", + "disc_equation_FStar.Pervasives.Inr", "equation_Bug1536.ex", + "fuel_guarded_inversion_FStar.Pervasives.either", "unit_typing" + ], + 0, + "b71b3014e8e1063bcbe6df0f8e0fa413" + ], + [ + "Bug1536._dm4f_EXN_bind_wp", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "disc_equation_FStar.Pervasives.Inl", + "disc_equation_FStar.Pervasives.Inr", + "fuel_guarded_inversion_FStar.Pervasives.either" + ], + 0, + "4c65288b611341da394a7e40b23dade7" + ], + [ + "Bug1536._dm4f_EXN___proj__EXN__item__raise_elab", + 1, + 2, + 1, + [ "@query" ], + 0, + "cc034a01fa60329b2cb936e4589beb78" + ], + [ + "Bug1536.EXN", + 1, + 2, + 1, + [ "@query" ], + 0, + "c8a3c9bfc1ec20f419eb8522a5f21748" + ], + [ + "Bug1536.ret", + 1, + 2, + 1, + [ "@query" ], + 0, + "56b5590609cd19f33112b67514ae1aa5" + ] + ] +] \ No newline at end of file diff --git a/examples/bug-reports/ExtractionBug2.fst.hints b/examples/bug-reports/ExtractionBug2.fst.hints index 5c8619316b3..4d96ee02238 100644 --- a/examples/bug-reports/ExtractionBug2.fst.hints +++ b/examples/bug-reports/ExtractionBug2.fst.hints @@ -42,7 +42,7 @@ "subterm_ordering_FStar.Pervasives.Native.Mktuple2" ], 0, - "c4bbe084a02527b21441415367934842" + "29539dd95bdce4360872d82185f32f7c" ], [ "ExtractionBug2.app", @@ -56,7 +56,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "800197427aaeae6338eef142fde4eebc" + "a495699a5297d7ef81f605efc7d085e6" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug024.fst.hints b/examples/bug-reports/bug024.fst.hints index c8a19ce33ad..832fa2a608e 100644 --- a/examples/bug-reports/bug024.fst.hints +++ b/examples/bug-reports/bug024.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list" ], 0, - "7cda35ed7e7c12289b91e5ef2e2b14cb" + "83a3ae59bbb34760b1fd9066de29e23e" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug025.fst.hints b/examples/bug-reports/bug025.fst.hints index f2187cb7ad4..e124fd6fa04 100644 --- a/examples/bug-reports/bug025.fst.hints +++ b/examples/bug-reports/bug025.fst.hints @@ -16,7 +16,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "6ea1af061b63f318de2db8cb61222e03" + "7c88b011c791f27523e6ea82ac9eef4b" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug026.fst.hints b/examples/bug-reports/bug026.fst.hints index 057a8b08309..70a4c4e0011 100644 --- a/examples/bug-reports/bug026.fst.hints +++ b/examples/bug-reports/bug026.fst.hints @@ -31,7 +31,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "719f4867f110d5a62f2934bc4347a4bc" + "db5f6063c004ef00ba367053a6094a03" ], [ "Bug026.test_filter1", diff --git a/examples/bug-reports/bug056.fst.hints b/examples/bug-reports/bug056.fst.hints index 7202655a302..20a05d697b2 100644 --- a/examples/bug-reports/bug056.fst.hints +++ b/examples/bug-reports/bug056.fst.hints @@ -17,7 +17,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "b5296b0f36fbc29cc1f7e06f9613cb5d" + "2a844e292c0e216758dc0f33bb8ea11f" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug058.fst.hints b/examples/bug-reports/bug058.fst.hints index e8ab8582690..0b1a96b69d1 100644 --- a/examples/bug-reports/bug058.fst.hints +++ b/examples/bug-reports/bug058.fst.hints @@ -20,7 +20,7 @@ "well-founded-ordering-on-nat" ], 0, - "7286531e05d3c8104c4991f9e362e156" + "8e01a8fda7b96efcbf963adb46563bd4" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug058b.fst.hints b/examples/bug-reports/bug058b.fst.hints index bbc935607c8..ff59b7ff62f 100644 --- a/examples/bug-reports/bug058b.fst.hints +++ b/examples/bug-reports/bug058b.fst.hints @@ -23,7 +23,7 @@ "well-founded-ordering-on-nat" ], 0, - "133393c6574dcf4cbc2086f16ac5922c" + "c892c44a8dca76b2dd2425e645d8c25b" ], [ "Bug058b.fibonacci", diff --git a/examples/bug-reports/bug1091.fst.hints b/examples/bug-reports/bug1091.fst.hints index e85a7e00380..2512414aee4 100644 --- a/examples/bug-reports/bug1091.fst.hints +++ b/examples/bug-reports/bug1091.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_FStar.UInt64.t__uu___haseq" ], 0, - "daf01c79d677462426171692e3c1b523" + "7019589552d4c4ad6b2cd14ae1e4a20b" ], [ "Bug1091.jun21_2017_logand_fail", @@ -25,7 +25,7 @@ "uvar_typing_19" ], 0, - "75d5340e3993a1e450433a79886a15b2" + "4a548eb5c4990a2dd552002ad5158e47" ], [ "Bug1091.jun21_2017_logand", @@ -37,7 +37,7 @@ "haseqFStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87" ], 0, - "196b022ac40cd6fe25981e1dab262e39" + "5ffa103e129a11c07f703ba27d27d822" ], [ "Bug1091.apr19_2017_mem", @@ -52,7 +52,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "e14227763a72e0c7c0b57a2e84b1e8f1" + "32f5b7785a1a55e7851c20a4f2f18ce6" ], [ "Bug1091.apr19_2017_mem_sanity", @@ -64,7 +64,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "6210dd046936ce71e2e0aa798092f9bb" + "0ebd5bed926cf228498e3e91712f8ca4" ], [ "Bug1091.apr19_2017_mem_sanity", @@ -76,7 +76,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "c313d9035cd2a423b525b19f8517b4f7" + "e13a4aac06e40a4e1d1c974eacc7e5de" ], [ "Bug1091.apr19_2017_mem_sanity", @@ -88,7 +88,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "1bf5c27ea5dc6498827ee3d0e0a88c3b" + "b6c494ac63653f109a8255b45a68e9c7" ], [ "Bug1091.apr21_2017_ackermann_fail", @@ -97,7 +97,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "da2e12130b44c9c25cf3c95107d16b1f" + "121e736ed8a2c5da2ea2d533412a1a25" ], [ "Bug1091.apr21_2017_ackermann_fail", @@ -106,7 +106,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "af0a172f9e84b73d30bb03abb9a63827" + "8ba5c93b3f0c42d99836ddfa3f114202" ], [ "Bug1091.apr21_2017_ackermann", @@ -128,7 +128,7 @@ "well-founded-ordering-on-nat" ], 0, - "014df66faca7a0b3f091c4f27ac1fe97" + "b629be3887b29fe284e2cb504908028d" ], [ "Bug1091.apr21_2017_ackermann", @@ -137,7 +137,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "bb821680c3efc4b029ed5714eb1abfad" + "254ac4af892f2de6615f5a162f5c4dbb" ], [ "Bug1091.apr21_2017_ackermann", @@ -146,7 +146,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "b82f81bacd249d6b4d003cc4297a0d10" + "8c2820beee4dbbdd05a55fa74d08fbef" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug1206.fst.hints b/examples/bug-reports/bug1206.fst.hints index f30b7645fd5..1b193e32ceb 100644 --- a/examples/bug-reports/bug1206.fst.hints +++ b/examples/bug-reports/bug1206.fst.hints @@ -11,7 +11,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "c18a1a328e3e30b4e37113dd584b5a7e" + "32000cac5b9ba3cfbcf85d266243747c" ], [ "Bug1206.ser_id", @@ -26,7 +26,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option" ], 0, - "670a4c06540ae6084256b03035ec3b56" + "fd0ef1a36db90aadea0b0c765636812f" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug1319b.fst.hints b/examples/bug-reports/bug1319b.fst.hints index 032009dfd9c..1317bee04f1 100644 --- a/examples/bug-reports/bug1319b.fst.hints +++ b/examples/bug-reports/bug1319b.fst.hints @@ -12,7 +12,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "8b8570b857164784e0087b4218e7f865" + "0f2bbf8c3ba6070ceb10f6e271141b59" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug1361.fst.hints b/examples/bug-reports/bug1361.fst.hints index 6c6fb1f249c..b5672a76267 100644 --- a/examples/bug-reports/bug1361.fst.hints +++ b/examples/bug-reports/bug1361.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list" ], 0, - "9d9d280dfb16a9cd4788ccce984bb23f" + "a6d569048ff1d7d0ef5d1eb7cc4de76d" ], [ "Bug1361.f2", @@ -25,7 +25,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "e5f7786b9f84e20d16da28c4d3caac73" + "a2e64ef8814f336d8fc060158837d980" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug1362.fst.hints b/examples/bug-reports/bug1362.fst.hints index 1eb59da576f..6983c618893 100644 --- a/examples/bug-reports/bug1362.fst.hints +++ b/examples/bug-reports/bug1362.fst.hints @@ -30,7 +30,7 @@ "well-founded-ordering-on-nat" ], 0, - "b335c28079f15f036b044677ba94a098" + "59c45be048e57db5a5bccca5b465eb96" ], [ "Bug1362.f2", @@ -55,7 +55,7 @@ 1, [ "@query" ], 0, - "75e285f7c3e94678bf755a8939636d2c" + "2c2464361d35c1c282bd0935be73ccb4" ], [ "Bug1362.f4", @@ -70,7 +70,7 @@ "projection_inverse_BoxInt_proj_0", "well-founded-ordering-on-nat" ], 0, - "d443fc8f323bdbc8dd7b7e0f5f43bc8e" + "76103f5abdbbf14e785169671c7f8f52" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug138.fst.hints b/examples/bug-reports/bug138.fst.hints index 568b3134c23..886625e64f5 100644 --- a/examples/bug-reports/bug138.fst.hints +++ b/examples/bug-reports/bug138.fst.hints @@ -14,7 +14,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "2fb2bf08cb37de4bd741583e31611032" + "b09b2ae2fd41f642da72f6848dab030a" ], [ "Bug138.foo", @@ -27,7 +27,7 @@ "well-founded-ordering-on-nat" ], 0, - "e4c0989849871d003f94f4db90f0a80d" + "9de9fddc28e956ccb6e793f903b42f12" ], [ "Bug138.arg_precede", @@ -61,7 +61,7 @@ "well-founded-ordering-on-nat" ], 0, - "f55d15a0008cccf2bcbf8accd72725bb" + "fadfd22b0f3fb1a1e223dd7750801d16" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug1414.fst.hints b/examples/bug-reports/bug1414.fst.hints index b117961dc85..2e0b1f05bf4 100755 --- a/examples/bug-reports/bug1414.fst.hints +++ b/examples/bug-reports/bug1414.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "projection_inverse_BoxBool_proj_0" ], 0, - "8353bde54b1cb4e9d504d3008488691d" + "fa3b8bf6bf8a9a946bd1e4decbd7e1cb" ], [ "Bug1414.f'", @@ -17,7 +17,7 @@ 1, [ "@query", "projection_inverse_BoxBool_proj_0" ], 0, - "ae3c8efacc83cbfcc4dd583e8968c10b" + "93a3cb215ae9866863d92f401cef03fe" ], [ "Bug1414.list", @@ -26,7 +26,7 @@ 1, [ "@query" ], 0, - "794aff59027a73a1ce4844d050604771" + "77292a6f5acbc24a27e7be28eef877c1" ], [ "Bug1414.__proj__Cons__item__hd", @@ -39,7 +39,7 @@ "refinement_interpretation_Bug1414_Tm_refine_1dc6a56c5c49f7722088b41ebcd5d2a7" ], 0, - "5bc59c7f66bf5ef4f7ae6553efcdb888" + "6bd4106e84dcafeb11b2c0d0d0692e96" ], [ "Bug1414.__proj__Cons__item__tl", @@ -52,7 +52,7 @@ "refinement_interpretation_Bug1414_Tm_refine_1dc6a56c5c49f7722088b41ebcd5d2a7" ], 0, - "4804d3db30a87906e641537f380339d3" + "1506f9a85f696f2129a8ecd74be021ff" ], [ "Bug1414.f''", @@ -61,7 +61,7 @@ 1, [ "@query", "projection_inverse_BoxBool_proj_0" ], 0, - "d4e44fe647bc865a2f7e1bb84a20ca8d" + "3f14b483b917c1ce5cb59a8af19b719d" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug1535b.fst.hints b/examples/bug-reports/bug1535b.fst.hints new file mode 100644 index 00000000000..a8ffb03dc81 --- /dev/null +++ b/examples/bug-reports/bug1535b.fst.hints @@ -0,0 +1,70 @@ +[ + "m\u001bMY֙", + [ + [ + "Bug1535b.__proj__G0__item__uu___", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", "disc_equation_Bug1535b.G0", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_Bug1535b_Tm_refine_5490163dcc20b59eece3a3cb5fde2ddf" + ], + 0, + "c90202968d1f6ef414c7294fb8a45534" + ], + [ + "Bug1535b.__proj__G1__item__uu___", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", "disc_equation_Bug1535b.G1", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_Bug1535b_Tm_refine_0e544009a6977444a0a5b71b19a94454" + ], + 0, + "59f70295f2453ee475eaefd736d54edc" + ], + [ + "Bug1535b.__proj__G2__item__uu___", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", "disc_equation_Bug1535b.G2", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_Bug1535b_Tm_refine_efed3dc492c71bf16b1a349b091dfe3e" + ], + 0, + "a8b14afeec765857dc476bc5a54b99d8" + ], + [ + "Bug1535b.__proj__G3__item__uu___", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", "disc_equation_Bug1535b.G3", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_Bug1535b_Tm_refine_db9134a200c9dc0ea59a9397653002dd" + ], + 0, + "d20a9039eaebd9d611a409d5961bf373" + ], + [ + "Bug1535b.__proj__G4__item__uu___", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", "disc_equation_Bug1535b.G4", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_Bug1535b_Tm_refine_1390932e4576fe0cad88c7523895958b" + ], + 0, + "c23d67e1d61a0a1094d1e712c68b46e8" + ] + ] +] \ No newline at end of file diff --git a/examples/bug-reports/bug161.fst.hints b/examples/bug-reports/bug161.fst.hints index 86a0fbe4b97..4d6cade4a7f 100644 --- a/examples/bug-reports/bug161.fst.hints +++ b/examples/bug-reports/bug161.fst.hints @@ -19,7 +19,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "0d41f34f9cb0306b56d6aec66ede8efd" + "169676ddc1d864a3c3d5717fe15b959b" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug162.fst.hints b/examples/bug-reports/bug162.fst.hints index 65236535d37..87834b6b655 100644 --- a/examples/bug-reports/bug162.fst.hints +++ b/examples/bug-reports/bug162.fst.hints @@ -21,7 +21,7 @@ "well-founded-ordering-on-nat" ], 0, - "e4f133213f89ded0e4e75552246d633b" + "be20bbe9c5dfcfe8eac1ed92bfbaba93" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug173.fst.hints b/examples/bug-reports/bug173.fst.hints index 5c93e26bd40..ffd8a7facc1 100644 --- a/examples/bug-reports/bug173.fst.hints +++ b/examples/bug-reports/bug173.fst.hints @@ -321,7 +321,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "2323dcc336d90833307938041f6edccd" + "3a35e7debb2d149abf9b6bc6099f6275" ], [ "Bug173.step", @@ -350,7 +350,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "e41f81ab86ddfc55ef42bd0ddc3eca4c" + "e4dd85861c53253ff2a37195c012d26f" ], [ "Bug173.op_type", @@ -394,7 +394,7 @@ "subterm_ordering_Bug173.Op" ], 0, - "fc28db0fca1b15a72e8480ead4a67db4" + "e9745f3d8f9fcf04cc4b949371e27fa3" ], [ "Bug173.typing", @@ -421,7 +421,7 @@ "typing_FStar.Pervasives.Native.uu___is_None" ], 0, - "61e4bb817608762031ce4a2794f2a5bb" + "401a7d47915a193ce14d74fd5d28bcec" ], [ "Bug173.typed_heap", diff --git a/examples/bug-reports/bug185.fst.hints b/examples/bug-reports/bug185.fst.hints index fe4434d5e8e..db931e4d26e 100644 --- a/examples/bug-reports/bug185.fst.hints +++ b/examples/bug-reports/bug185.fst.hints @@ -25,7 +25,7 @@ "token_correspondence_Bug185.verified" ], 0, - "fa1f55b95eab824f2facd7fcb557c470" + "9b1e3ecaf9ca55b374eebb6ad27e24e7" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug279.fst.hints b/examples/bug-reports/bug279.fst.hints index 1f60abb7bfe..cf9255a0139 100644 --- a/examples/bug-reports/bug279.fst.hints +++ b/examples/bug-reports/bug279.fst.hints @@ -23,7 +23,7 @@ "subterm_ordering_Bug279.T" ], 0, - "830d97c3e7ae9e0c13f775b99b11cbe4" + "3a35779fceef98a7a5d20f6e5a9f7dd0" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug281.fst.hints b/examples/bug-reports/bug281.fst.hints index 6bfa350b603..381b961ce28 100644 --- a/examples/bug-reports/bug281.fst.hints +++ b/examples/bug-reports/bug281.fst.hints @@ -101,8 +101,8 @@ "projection_inverse_BoxBool_proj_0", "projection_inverse_BoxInt_proj_0", "projection_inverse_Bug281.EVar__0", - "refinement_interpretation_Bug281_Tm_refine_9d6b80f9e4c15b60d3b9076b8f1917b6", "refinement_interpretation_Bug281_Tm_refine_9eeb2fe43433bda3ba01b74f4dd6684d", + "refinement_interpretation_Bug281_Tm_refine_e5b6f23e0788b61e7a0d92ee3e3afeb2", "refinement_interpretation_FStar.StrongExcludedMiddle_Tm_refine_94f72bfda5e23ac3960136c8bc3f958c", "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", "token_correspondence_Bug281.sub_einc", "typing_Bug281.esubst", @@ -112,7 +112,7 @@ "well-founded-ordering-on-nat" ], 0, - "2b384de7d75245786a754e372bf039a5" + "2d79c9c3c423c3aa72891468ff7b0484" ], [ "Bug281.sub_elam", @@ -142,7 +142,7 @@ "well-founded-ordering-on-nat" ], 0, - "5d74e39513c4a74100cca69d693d17fc" + "bd01d3a29ba96a106cd91b4871d11882" ], [ "Bug281.lemma", diff --git a/examples/bug-reports/bug379.fst.hints b/examples/bug-reports/bug379.fst.hints index fcbb2395ad4..20d65e6dc59 100644 --- a/examples/bug-reports/bug379.fst.hints +++ b/examples/bug-reports/bug379.fst.hints @@ -15,7 +15,7 @@ "well-founded-ordering-on-nat" ], 0, - "ee7aaaaba3dbd56b7ddae5ab3a298f37" + "cd5714b2ee545a1aba59bd96de227855" ], [ "Bug379.test3", diff --git a/examples/bug-reports/bug463b.fst.hints b/examples/bug-reports/bug463b.fst.hints index 3dd5dc288f5..9079344b163 100644 --- a/examples/bug-reports/bug463b.fst.hints +++ b/examples/bug-reports/bug463b.fst.hints @@ -24,7 +24,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.mem" ], 0, - "c054f48a82a74a77bb83cfab04ca117f" + "38d5f58d653b732a862f2b17458b79ef" ], [ "Bug463b.eq1", diff --git a/examples/bug-reports/bug466.fst.hints b/examples/bug-reports/bug466.fst.hints index fd3c496aa9e..4dcb841a6e2 100644 --- a/examples/bug-reports/bug466.fst.hints +++ b/examples/bug-reports/bug466.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "75d1e52f27ae03791fd97bc5c1a2c71d" + "41fdce5795704cd1ce45a7a014bd963b" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug579.fst.hints b/examples/bug-reports/bug579.fst.hints index de4e86333af..cb2423c001b 100644 --- a/examples/bug-reports/bug579.fst.hints +++ b/examples/bug-reports/bug579.fst.hints @@ -47,7 +47,7 @@ "subterm_ordering_Bug579.TyEqu" ], 0, - "1bfac48c468b47739303dcf11f982c12" + "88883055fd602ec30ff883e627216e21" ], [ "Bug579.progress", @@ -63,7 +63,7 @@ "projection_inverse_Bug579.TyEqu_t1", "subterm_ordering_Bug579.TyEqu" ], 0, - "debc34c594152c8654e03781fe6a3d42" + "77bfab93c180c3be8917c6cc73ba8979" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug589.fst.hints b/examples/bug-reports/bug589.fst.hints index 9ed1b4c3bd3..863ee331924 100644 --- a/examples/bug-reports/bug589.fst.hints +++ b/examples/bug-reports/bug589.fst.hints @@ -12,7 +12,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "1cc8c89966b8d42d1743b28043c3ac9b" + "4e56349bcc4cd110fa1c06de8e1dd079" ] ] ] \ No newline at end of file diff --git a/examples/bug-reports/bug590.fst.hints b/examples/bug-reports/bug590.fst.hints index bbf5de891ca..689749f4171 100644 --- a/examples/bug-reports/bug590.fst.hints +++ b/examples/bug-reports/bug590.fst.hints @@ -30,7 +30,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "f52ae86a6e9de72c90b7c73c17045345" + "60c17bedf00a0a07209a79f522c70fcf" ], [ "Bug590.blah2", diff --git a/examples/bug-reports/bug606.fst.hints b/examples/bug-reports/bug606.fst.hints index 7e0ca7c5e6b..5b4040742e1 100644 --- a/examples/bug-reports/bug606.fst.hints +++ b/examples/bug-reports/bug606.fst.hints @@ -15,7 +15,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "b0c2c0d9199d71f4305e31ebffbc0fbf" + "8a50b18bdc5069176f587bafd1001daa" ], [ "Bug606.g", @@ -31,7 +31,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "21ae8662eb3e876d725babd465da4579" + "8f4eb52d949b72e52517189a7ce923c8" ], [ "Bug606.f_eq_g", diff --git a/examples/bug-reports/bug989.fst.hints b/examples/bug-reports/bug989.fst.hints index 14c1a89752f..aa3acb71fcb 100644 --- a/examples/bug-reports/bug989.fst.hints +++ b/examples/bug-reports/bug989.fst.hints @@ -15,7 +15,7 @@ "well-founded-ordering-on-nat" ], 0, - "41710a87f00212d97082b75c9ce47f34" + "a9b341224af7bf316d69d8f3ae7a45c5" ], [ "Bug989.foo", diff --git a/examples/crypto/CntProtocol.fst.hints b/examples/crypto/CntProtocol.fst.hints index 21864b122bd..24f3bcfd478 100644 --- a/examples/crypto/CntProtocol.fst.hints +++ b/examples/crypto/CntProtocol.fst.hints @@ -59,7 +59,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "6cc9484af6907ab447329f7d2a43df88" + "afc7de206976bd9ecc7bdb9cd131fe9d" ], [ "CntProtocol.max_list", diff --git a/examples/crypto/EtM.AE.fst.hints b/examples/crypto/EtM.AE.fst.hints index 83e395aa8b8..6aecb05902d 100644 --- a/examples/crypto/EtM.AE.fst.hints +++ b/examples/crypto/EtM.AE.fst.hints @@ -83,7 +83,7 @@ "typing_FStar.Seq.Base.seq", "well-founded-ordering-on-nat" ], 0, - "70824fc6111acbf7d15aeee1b5484f08" + "91076a9e20fdccfc35b387f3686bec21" ], [ "EtM.AE.mac_only_cpa_ciphers_snoc", @@ -222,7 +222,7 @@ "typing_FStar.Seq.Base.seq", "well-founded-ordering-on-nat" ], 0, - "1e836042ff77dd43d9fb858afd3efe63" + "a191ec8a0a9984dd79264d88068ad068" ], [ "EtM.AE.mac_and_cpa_refine_ae_snoc", diff --git a/examples/crypto/EtM.CPA.fst.hints b/examples/crypto/EtM.CPA.fst.hints index e9209e01ece..0a7cb964e06 100644 --- a/examples/crypto/EtM.CPA.fst.hints +++ b/examples/crypto/EtM.CPA.fst.hints @@ -225,7 +225,7 @@ "typing_FStar.Seq.Base.seq", "well-founded-ordering-on-nat" ], 0, - "8da6d1a5951f8be2c0dca515d3d1595e" + "eb68d22e5806047fa15abb3fc3443d57" ], [ "EtM.CPA.pairwise_snoc", diff --git a/examples/csl/Examples.fst.hints b/examples/csl/Examples.fst.hints index e5833aaf751..9b967b8f89c 100644 --- a/examples/csl/Examples.fst.hints +++ b/examples/csl/Examples.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "90580ffca3ac3845d60e58ae2f3ed6a9" + "b081c24e12d0bed7ea35bdb6e456f1d2" ], [ "Examples.increment_ok", @@ -25,7 +25,7 @@ "unit_inversion", "unit_typing" ], 0, - "c34b6d68c65bea59cbed06465cb6bfa1" + "c6a76db61f55368e97a1083f3c74e60d" ], [ "Examples.increment_ok", @@ -40,7 +40,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "bbc500162a9ca5bfd2827c552e90ff76" + "b22c1acc30db5ed2376f94daa7b9a38f" ], [ "Examples.increment_ok", @@ -61,7 +61,7 @@ "typing_FStar.SL.Monotonic.Heap.points_to" ], 0, - "abe9d79daaf4962d6ed7965dc20743ac" + "0639eb378a518e8521d4ffdb7527b638" ], [ "Examples.swap_ok", @@ -74,7 +74,7 @@ "true_interp" ], 0, - "e864bb900fa69f4d1643a00752c1ac29" + "2d5aa314158f88031ab24d5a5d66bf05" ], [ "Examples.swap_ok", @@ -86,7 +86,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "88839ef30ccdb3269af5be9278818aec" + "fdd065a665468d225920e1b26b5690ca" ], [ "Examples.swap_ok", @@ -104,7 +104,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "3b0aa66ffc7a18ee68fe78e8d2f2ce0b" + "385dac3af215031feff5a5e040e27fd9" ], [ "Examples.swap_ok", @@ -116,7 +116,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "9b57caa2cc4151dfa47a5d2ac65e2120" + "bd78b1755f7e2860d44a1ddb62d3a3bd" ], [ "Examples.swap_ok", @@ -135,7 +135,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "61d255be7ee0bec90dd4dd4400c42422" + "6401f437a39c8e274374b948cc1d2450" ], [ "Examples.swap_ok", @@ -161,7 +161,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "ca558ce0459175c65c252b2c674a805f" + "1907538cacc96cd332d71dc994f7dd10" ], [ "Examples.swap_ok", @@ -180,7 +180,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "3ba1a3d9cc715ae5dc70faf851895507" + "7fe7db99ba8f3e7a1737d628e3d9cdfc" ], [ "Examples.swap_ok", @@ -201,7 +201,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "4c6e14dd68133a4472f64a170632aeea" + "babdbc776d90e18dc1b880d88ead933a" ], [ "Examples.swap_ok", @@ -222,7 +222,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "eb4654985d2c66b98593bcfb3079e7eb" + "6b564eb9dfd12fe6cc40298d2e7d1139" ], [ "Examples.double_increment_ok", @@ -237,7 +237,7 @@ "unit_inversion", "unit_typing" ], 0, - "3b04a4fc6ae70d1a06f6a1f8b843e98c" + "5c79eb6a68923a8dd19d6457682f886e" ], [ "Examples.double_increment_ok", @@ -252,7 +252,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "547e04e85527721737d034f7351c1113" + "14116bef00c56ad7caa4018c98c269cf" ], [ "Examples.double_increment_ok", @@ -270,7 +270,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "afa8775566a0b29d5a7f515f2c70944d" + "82feba63865562d560a58c4a3710452e" ], [ "Examples.double_increment_ok", @@ -289,7 +289,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "d1fd31204c5a23e8e8d246468864ccb1" + "65391a5479476e7145a92d896dbb8e36" ], [ "Examples.double_increment_ok", @@ -329,7 +329,7 @@ "typing_FStar.UInt64.v" ], 0, - "f8b62062562c0d284f706d534d604769" + "8bc30145f7b5aee10383e9742910a825" ], [ "Examples.init_ok", @@ -369,7 +369,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "b972437f4496441306c6a8b2428ca562" + "e0c26f186798800b788f616f1168859c" ], [ "Examples.init_ok", @@ -407,7 +407,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "919a4c6171b0a21342128c8bd0609f06" + "83db1f2bf1cd5e232d01416e7b13c0fb" ], [ "Examples.copy_ok", @@ -423,7 +423,7 @@ "true_interp" ], 0, - "992e79569ae8eb942ceed4086fc37cce" + "f595c37976385bde12f49eb026c48095" ], [ "Examples.copy_ok", @@ -438,7 +438,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "cc36aa284e1f5ea8b318915b064f7231" + "dff66fc98fadb43585a115e13f8d22f1" ], [ "Examples.copy_ok", @@ -456,7 +456,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "13f942b6706e531803286ae9a6f59696" + "65bcf42475750409e301ae3ebfff34ad" ], [ "Examples.copy_ok", @@ -474,7 +474,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "68be352f0ba43dee90ceb750bd4c2827" + "a516c8fb020cc0c2d6610ddabfab4f7f" ], [ "Examples.copy_ok", @@ -495,7 +495,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "0dc21839bd2441a46107f5c8db999c7e" + "9eff316ef0fe0063c980a65326867e71" ], [ "Examples.copy_ok", @@ -513,7 +513,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "62aa586a8fd703098374257c9834de2a" + "8c0f4eb9d38ccc2bc41661ce51fcf1e6" ], [ "Examples.copy_ok", @@ -525,7 +525,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "757e26d8e38e292f3f7e5eddfff47860" + "15d76793f10d00dd76d52c336f68e7e9" ], [ "Examples.copy_ok", @@ -537,7 +537,7 @@ "refinement_interpretation_Examples_Tm_refine_27e663d45ab46f5b4e6a1f9a37782360" ], 0, - "b1c3ac19fb86f4508cfad0fecce34a5c" + "bedc54efc7cfa48738376111b7fc2b28" ], [ "Examples.write_ok", @@ -546,7 +546,7 @@ 1, [ "@query" ], 0, - "4863961780b78db24b90ba9330d4a701" + "22c4fede55eb2c5f8a8de29dde4d3de6" ], [ "Examples.increment_ok", @@ -555,7 +555,7 @@ 1, [ "@query" ], 0, - "4560e100d016a361e182d702db21a2c4" + "b9d28640b7059a7737dac92335199a8e" ], [ "Examples.increment_ok", @@ -570,7 +570,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "9c2ac9e5b94e9be6b2722b95497dfede" + "a15da1f4ffdf9d5fbec0bffe887c0ba9" ], [ "Examples.increment_ok", @@ -591,7 +591,7 @@ "typing_FStar.SL.Monotonic.Heap.points_to" ], 0, - "0df5d154fe1eb21f2a212ab6c823f4a5" + "bf4d55308c08fd9de82efecc6b6fd721" ], [ "Examples.swap_ok", @@ -604,7 +604,7 @@ "true_interp" ], 0, - "1c3d807c6c55fcc19188cbb590c3cae5" + "7590bd59d2f5ac70efd682a1be127203" ], [ "Examples.swap_ok", @@ -613,7 +613,7 @@ 1, [ "@query" ], 0, - "f86c7ed5666685c07584c33f28a911a0" + "1439c021b3b8ba97782612ceaacfb513" ], [ "Examples.swap_ok", @@ -631,7 +631,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "ace8a418e9357263247f0c2481b4b71c" + "4a2156e115b8d2ab1c411833868a6ba1" ], [ "Examples.swap_ok", @@ -643,7 +643,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "59f606d9950a9b19635a3f59844b9046" + "f2e4c4de055b32efd545a2da65c3da6c" ], [ "Examples.swap_ok", @@ -664,7 +664,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "60e056a5afe47297cd16abec15bf8c81" + "1821afa4635977c4958c306b61ea0fb3" ], [ "Examples.swap_ok", @@ -690,7 +690,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "078679c41d7a74b09a0abaa2fd2e0e1a" + "17ea168747532e4a00060185c8a423a9" ], [ "Examples.swap_ok", @@ -709,7 +709,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "7bd0c0e548be220dbdd2d4ebcae13b47" + "39a5f9172567d0e7ff5a27ebea87aefd" ], [ "Examples.swap_ok", @@ -730,7 +730,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "388b5cbe2c4d7028854016e3f9af76ea" + "ecc2caf196950eb9398110a389bd9f70" ], [ "Examples.swap_ok", @@ -751,7 +751,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "9e725593054e0093b62a2295a6502234" + "af714e98ce9e6bc271f4a9263d3e560b" ], [ "Examples.double_increment_ok", @@ -760,7 +760,7 @@ 1, [ "@query" ], 0, - "ea4b1d49dca01b9716480138f9383913" + "fd7285429f2585971a991a29d458edc2" ], [ "Examples.double_increment_ok", @@ -775,7 +775,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "f21ddcc5214ac48ff671f749dff802bb" + "4b656b1156d678339d86090b54e2c951" ], [ "Examples.double_increment_ok", @@ -793,7 +793,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "d3342235cb9550c955c1d5146ba6081a" + "36324045ad9348bb35ceed3f63f6d118" ], [ "Examples.double_increment_ok", @@ -812,7 +812,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "a56ca78646e192be49359f35b71ce9c2" + "77feb38005bfc12d2257104aed7b9078" ], [ "Examples.double_increment_ok", @@ -852,7 +852,7 @@ "typing_FStar.UInt64.v" ], 0, - "326d0494bdb908657d28f0a7161c8f72" + "a1552e00887d02d2bd7a1a84ad062938" ], [ "Examples.init_ok", @@ -892,7 +892,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "ffaa7ff52e6dacda46de9779acc2d04c" + "6b1f6100ef53dd2efaa1293e897c09cc" ], [ "Examples.init_ok", @@ -930,7 +930,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "743246f97a2dd4e7e065e32920f2fd3f" + "2b6ff616b336206df2c09adf14244409" ], [ "Examples.copy_ok", @@ -946,7 +946,7 @@ "true_interp" ], 0, - "46bb60eb702aec0a8552ee94182bcd33" + "50c94f990488c28d6ba77e4fbe54175e" ], [ "Examples.copy_ok", @@ -955,7 +955,7 @@ 1, [ "@query" ], 0, - "d30e9008e499665d1bf65a2dba43d2c5" + "1f2e46cb22af60d506fb99b4355290d7" ], [ "Examples.copy_ok", @@ -973,7 +973,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "6d898d26c86a57992135e887ca2b30ff" + "13f5a6bc0a8240d5c43a84f5ee8e4a90" ], [ "Examples.copy_ok", @@ -991,7 +991,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "554655e4b3988ad5ee4e145ec648a250" + "79a506e6a2d1782fa54975af38b140d1" ], [ "Examples.copy_ok", @@ -1012,7 +1012,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "bd0512577989805cd029a664d524de91" + "18f17fff02121a85d428f890f68885bc" ], [ "Examples.copy_ok", @@ -1030,7 +1030,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "43c49b43d08817b159251d4e9ffb80ed" + "37485d213c277d0df37b1ee789e1de08" ], [ "Examples.copy_ok", @@ -1042,7 +1042,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "177c34d14b88c071b169b42d3d3d3d81" + "77b3da2fff8256b4c854091b0b93e56c" ], [ "Examples.copy_ok", @@ -1054,7 +1054,7 @@ "refinement_interpretation_Examples_Tm_refine_27e663d45ab46f5b4e6a1f9a37782360" ], 0, - "4a23bdf4edde5a8921e47bf6100c570d" + "64150216ae19a2cdd0611eda500a82de" ] ] ] \ No newline at end of file diff --git a/examples/csl/Lang.fst.hints b/examples/csl/Lang.fst.hints index 136ba3246ee..7186891dd46 100644 --- a/examples/csl/Lang.fst.hints +++ b/examples/csl/Lang.fst.hints @@ -141,7 +141,7 @@ "unit_typing" ], 0, - "b65d9cd839706b4ff9f6a714e74e4a8f" + "d556ef50a16e5fc39c6e745ace85821e" ], [ "Lang.__proj__Return__item__a", @@ -283,7 +283,7 @@ "typing_tok_Lang.Alloc@tok", "unit_typing" ], 0, - "b9f0c12feb3c6e9d79548df39a18bf93" + "97dc73eb13a2711dac30885ac5c27c60" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.AutoTactic.fst.hints b/examples/csl/SL.AutoTactic.fst.hints index a49b871f895..6cdd6e4e187 100644 --- a/examples/csl/SL.AutoTactic.fst.hints +++ b/examples/csl/SL.AutoTactic.fst.hints @@ -11,7 +11,7 @@ "lemma_SL.Heap.lemma_sep_comm" ], 0, - "12e7a6a34400969b5bd312ef5b1ae4d3" + "4e5b9cf806c58fba7502fd43c1e46244" ], [ "SL.AutoTactic.fv_is", @@ -20,7 +20,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "f31c30f7f741a4af7d60262e94c09e5b" + "dbd28f5d12e383ba4f628097959aaff5" ], [ "SL.AutoTactic.frame_wp_lemma", @@ -34,7 +34,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "94445f7cebb13c334faec73bf3eebdfd" + "a041def2eada0a2046bc96a5fccd6ba4" ], [ "SL.AutoTactic.ite_wp_lemma", @@ -47,7 +47,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "5e8838acb0e307391e8213f1a74136bc" + "1e718ac7c1f1693d47186ad2a9139844" ], [ "SL.AutoTactic.if_then_else_wp_lemma", @@ -61,7 +61,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "858da99c011ee292181568661b3116c0" + "2bbffd5fff40e822a92d5f43c4f92afa" ], [ "SL.AutoTactic.close_wp_lemma", @@ -71,11 +71,11 @@ [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", "equation_Prims.squash", "equation_SL.Effect.st_close_wp", - "l_quant_interp__9943", + "l_quant_interp__9969", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "e75b87dda4bd0396b3aea5be6aa20380" + "1f9711674690076ffc2bca5e7c7a3b55" ], [ "SL.AutoTactic.assume_p_lemma", @@ -89,7 +89,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "30466c7f3cb06ebb0458380a3be8aa9f" + "0c6d2ba720b13970d11df4a72f25484a" ], [ "SL.AutoTactic.compare_b", @@ -98,7 +98,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "5d571e80cf486f43ffbd42d1588e7101" + "aadca0d333fb11de5f146e2b89b73388" ], [ "SL.AutoTactic.sort_sl_correct", @@ -116,7 +116,7 @@ "token_correspondence_CanonCommMonoid.sortWith" ], 0, - "205642a5286ba1cf8917abedb13faff2" + "7306e74d9d0d753d56c187e0e81989cf" ], [ "SL.AutoTactic.__proj__Frame__item__ta", @@ -130,7 +130,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "5256f03b3689b203a89d7a8123aac18a" + "424f6e8429a5e0f01faf9db1bffe0199" ], [ "SL.AutoTactic.__proj__Frame__item__twp", @@ -144,7 +144,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "a561ec4b59904a4ecae2d26ecfefb8d0" + "79c5823f516edecd1bba19340acc688a" ], [ "SL.AutoTactic.__proj__Frame__item__tpost", @@ -158,7 +158,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "fe293e75612d260986a17691e250d77f" + "d07ad3385bea0693a87e7ec548963dda" ], [ "SL.AutoTactic.__proj__Frame__item__tm", @@ -172,7 +172,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "3462ae1c0c0894e337036c141f550225" + "e24d240eb160aca3b7bc7f7c503a5b22" ], [ "SL.AutoTactic.__proj__ParWP__item__twpa", @@ -186,7 +186,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_215fd0fa36578f49ef025a1f95319e74" ], 0, - "857d60cedcdaf4f9b6be9a8250876a74" + "c9e2642f4815dd3fc52c5d52516a4747" ], [ "SL.AutoTactic.__proj__ParWP__item__twpb", @@ -200,7 +200,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_215fd0fa36578f49ef025a1f95319e74" ], 0, - "d65965ab57275d28f6bfddc502229432" + "82c473a433c4511ff84890de34d12f99" ], [ "SL.AutoTactic.__proj__ParWP__item__th0", @@ -214,7 +214,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_215fd0fa36578f49ef025a1f95319e74" ], 0, - "c519cb1d07a2855243370d207383cca8" + "046b3cec668ebc5e96730227f2ae7e12" ], [ "SL.AutoTactic.__proj__Unknown__item___0", @@ -228,7 +228,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_ef99333c406db249fc03d4edb1fd9534" ], 0, - "604c2da4489cd2cb8ed57d156cec39e4" + "95f2a302e9093d39111fa640a214de65" ], [ "SL.AutoTactic.__lem_eq_sides", @@ -241,7 +241,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "c0c42245b95fd41cdb95c9e8704769c3" + "cefc96bf984c59ca5d946129643fdb57" ], [ "SL.AutoTactic.__and_elim", @@ -255,7 +255,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_b889b19b3d1b749e7e6619d0022a6af7" ], 0, - "12b8eac9e61c6a28b4b24c888942429d" + "d07486f1b1067d586be7da095e9f24ef" ], [ "SL.AutoTactic.destruct_and", @@ -270,14 +270,14 @@ "constructor_distinct_FStar.Tactics.Result.Success", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v", "unit_typing" ], 0, - "ffaaf0da57eab11b7ab03d5c9eb3a118" + "046f5c89c880c93e3be8c02116d854a2" ], [ "SL.AutoTactic.canon_binder_mem_eq", @@ -292,14 +292,14 @@ "constructor_distinct_FStar.Tactics.Result.Success", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v", "unit_typing" ], 0, - "768c081cc7444f51f681486b8d32f265" + "e6543382d44413af3b5c5abc25d9837b" ], [ "SL.AutoTactic.unfold_first_occurrence", @@ -311,7 +311,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "f89b31d46e0914bd8c6321378885efda" + "0b5d524a539c0199a946a578c8e1b37a" ], [ "SL.AutoTactic.__tcut", @@ -324,7 +324,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "a0d1810f88552744c016f29126b332b4" + "1ad06e2d0a9997f4fb5d1f9a190bf296" ], [ "SL.AutoTactic.__elim_fp", @@ -338,7 +338,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "de626da6f66a8b9f03cf1f72066d5055" + "28bb2d3e26e34c128e680947ffb4e81b" ], [ "SL.AutoTactic.__unif_helper", @@ -347,7 +347,7 @@ 1, [ "@query", "lemma_SL.Heap.lemma_sep_unit" ], 0, - "c7f9f2308b9ec625692db31e6967f296" + "71e8bd04cbc332a3898e409bd662d307" ], [ "SL.AutoTactic.find_frame", @@ -371,7 +371,7 @@ "lemma_FStar.Pervasives.invertOption", "projection_inverse_BoxInt_proj_0", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -380,7 +380,7 @@ "typing_FStar.UInt.fits", "unit_typing" ], 0, - "520e2482fa0d12bdb246e085ff46b2ee" + "3e1f8721927a8464745ef1b2ad4db746" ], [ "SL.AutoTactic.sl", @@ -410,7 +410,7 @@ "projection_inverse_BoxBool_proj_0", "projection_inverse_BoxInt_proj_0", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -421,7 +421,7 @@ "typing_FStar.UInt.fits", "unit_typing" ], 0, - "2d078602afa81d979e1d64aef0f2fd47" + "dda7b862432c86c9b754c856f0dd06b4" ], [ "SL.AutoTactic.__elim_exists_as_forall", @@ -430,12 +430,12 @@ 1, [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", - "equation_Prims.squash", "l_quant_interp__10460", + "equation_Prims.squash", "l_quant_interp__10486", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5", "refinement_interpretation_SL.AutoTactic_Tm_refine_d16de86ec5446f55c1622708945a0449" ], 0, - "58fb9b970371d8cd49e168255f34ee72" + "b60f50f49acfd250d0ac2adf00170814" ], [ "SL.AutoTactic.ddump", @@ -452,7 +452,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "5436a941d0afa3b606b6bc2f4046cd5f" + "8ff23c5fe1b80c37b08ee3072a1d21a7" ], [ "SL.AutoTactic.memory_cm", @@ -464,7 +464,7 @@ "lemma_SL.Heap.lemma_sep_comm" ], 0, - "ca95461905d0dd9e91a93d7c33d598b9" + "08350d2e26ad7ee32691669d12659337" ], [ "SL.AutoTactic.fv_is", @@ -473,7 +473,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "b3ed2a14c613aa9ed277a98f2c408d6b" + "22ddbf74014d7bc2722476eeb7a4da07" ], [ "SL.AutoTactic.frame_wp_lemma", @@ -487,7 +487,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "085f7bfa561b9781eea9b6feb33e90af" + "5cc0b9925bf313b9e4b7b7deb852fc70" ], [ "SL.AutoTactic.compare_b", @@ -496,7 +496,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "c261953f498211382e1ebea06d58fabf" + "767f0b84c5fdd4e8afaf4ff5c3b21163" ], [ "SL.AutoTactic.__proj__Frame__item__ta", @@ -510,7 +510,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "adb6339a90af1d5546244153ba62c5dd" + "8cccb9b2982200c013a7e1d233f20c13" ], [ "SL.AutoTactic.__proj__Frame__item__twp", @@ -524,7 +524,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "58cbf04119d22630973927da6fc6d734" + "9a68902bc604720e943a0251eb9d64dc" ], [ "SL.AutoTactic.__proj__Frame__item__tpost", @@ -538,7 +538,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "99db4899177a2b22f5e8d8f07965f0c5" + "208fe1e2f01aaa931372b08367aa389f" ], [ "SL.AutoTactic.__proj__Frame__item__tm", @@ -552,7 +552,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_2d47d28c80466f25c27aa06b4aa5a22b" ], 0, - "ca9d642a5047c982500920f9d75daf8f" + "fe5f448e0dec50138746e7559526b026" ], [ "SL.AutoTactic.__proj__ParWP__item__twpa", @@ -566,7 +566,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_215fd0fa36578f49ef025a1f95319e74" ], 0, - "4a621a9d7bf6e9ab1d224ed2a56c1387" + "ecaa28e84af5223008538c48bcceccf4" ], [ "SL.AutoTactic.__proj__ParWP__item__twpb", @@ -580,7 +580,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_215fd0fa36578f49ef025a1f95319e74" ], 0, - "e9ac2799957f5451e60731a413b90dc4" + "ed43f33ee44d5662493e1eb1df412ff7" ], [ "SL.AutoTactic.__proj__ParWP__item__th0", @@ -594,7 +594,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_215fd0fa36578f49ef025a1f95319e74" ], 0, - "a14e840a6656c8f15e8d41758da95a80" + "1b511e0100368130d29558fa7c3925d3" ], [ "SL.AutoTactic.__proj__Unknown__item___0", @@ -608,7 +608,7 @@ "refinement_interpretation_SL.AutoTactic_Tm_refine_ef99333c406db249fc03d4edb1fd9534" ], 0, - "f8b6d40740af7a7ed11751c63c35a3b8" + "93ab2d6e7cd0d50acf472100cba575e4" ], [ "SL.AutoTactic.destruct_and", @@ -623,14 +623,14 @@ "constructor_distinct_FStar.Tactics.Result.Success", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v", "unit_typing" ], 0, - "1dd6d7df8bd2662fe5c9819f50b7a8ca" + "21574e1f3e93c102b0e7ea56a588b2cc" ], [ "SL.AutoTactic.canon_binder_mem_eq", @@ -645,14 +645,14 @@ "constructor_distinct_FStar.Tactics.Result.Success", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v", "unit_typing" ], 0, - "09a509b95949e7b22f870327259ccbcd" + "a09e0f407261e1e704dc2775cc6b303d" ], [ "SL.AutoTactic.unfold_first_occurrence", @@ -664,7 +664,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "746029380b2467405607074dab09ab84" + "e3115dfb7fd27f3636028a373d569a85" ], [ "SL.AutoTactic.find_frame", @@ -688,7 +688,7 @@ "lemma_FStar.Pervasives.invertOption", "projection_inverse_BoxInt_proj_0", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -697,7 +697,7 @@ "typing_FStar.UInt.fits", "unit_typing" ], 0, - "e5867f7ffff7480640a7e7601f646004" + "5a832058d192985d2d2a2bc5c1c7f07d" ], [ "SL.AutoTactic.sl", @@ -727,7 +727,7 @@ "projection_inverse_BoxBool_proj_0", "projection_inverse_BoxInt_proj_0", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -738,7 +738,7 @@ "typing_FStar.UInt.fits", "unit_typing" ], 0, - "fcb9c20ca38f4446a22197ed00ca2b51" + "20bfde6a4eb575c260fa17fe3d3cc689" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.ConcurrentExamples.fst.hints b/examples/csl/SL.ConcurrentExamples.fst.hints index 1ec61cc7908..17a8a9b347b 100644 --- a/examples/csl/SL.ConcurrentExamples.fst.hints +++ b/examples/csl/SL.ConcurrentExamples.fst.hints @@ -13,7 +13,7 @@ "unit_inversion" ], 0, - "10d45f6ef7aa424c2f2f9b13d9e39a09" + "e7103b3fa957381d46ebf71e97446cc3" ], [ "SL.ConcurrentExamples.test17", @@ -25,7 +25,7 @@ "refinement_interpretation_SL.ConcurrentExamples_Tm_refine_cd225dd77bc8476b2ce0cc839b0de7bb" ], 0, - "dd425f58e2c59fb1b48d4250a63b08f3" + "1a6f95dbafac5026a4690091aba015cd" ], [ "SL.ConcurrentExamples.test17'", @@ -39,7 +39,7 @@ "unit_inversion" ], 0, - "995be1bf2b6faa78e81b486c914c4d2c" + "c3dd97e8289e76de888a765c74362197" ], [ "SL.ConcurrentExamples.test17'", @@ -53,7 +53,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "48a758797df3b76d252100a65e36d3d5" + "5637895adea37fa169ab73a1160c10ba" ], [ "SL.ConcurrentExamples.test18", @@ -67,7 +67,7 @@ "unit_inversion" ], 0, - "55bee8a4a8dfe8a7da70922d73f0205c" + "af0bb8aac93ea2597f25f1d86860eb62" ], [ "SL.ConcurrentExamples.test18", @@ -88,7 +88,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "c7a293241e98e5d13b6718ebba31883f" + "e199ff6b7028940bb6c3f2d248ca6338" ], [ "SL.ConcurrentExamples.test18", @@ -107,7 +107,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "a27c53f85d53a7580e80411d8edac790" + "d390649200d235116342cc6222811989" ], [ "SL.ConcurrentExamples.test18", @@ -119,7 +119,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "dab0d4b4b8d89a19184da627f6e63099" + "0db70872405f77054b2911e7862fa507" ], [ "SL.ConcurrentExamples.test19", @@ -133,7 +133,7 @@ "unit_inversion" ], 0, - "8b9d5cad54f6687820225e69ddcfcc92" + "8bf76a56bd09c99f3b79cb4d1b4ffc9d" ], [ "SL.ConcurrentExamples.test19", @@ -154,7 +154,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "af48899f519ca368575afed65726d80e" + "08d33f2334fcacacd5a853d969910a2d" ], [ "SL.ConcurrentExamples.test19", @@ -173,7 +173,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "e58a5fc090e33daa89ff7c59417f308f" + "39a81c47cd7725729fb65d35eff2397c" ], [ "SL.ConcurrentExamples.test19", @@ -185,7 +185,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "476db5aa543307b5dc00264787aa8e85" + "817786b5fa579f9031ca55e7c7bb0867" ], [ "SL.ConcurrentExamples.test20", @@ -206,7 +206,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "5606e29cb6a174c11dc5c41727fc6cc5" + "1b4e504cf34142dfc4329ad4013b048a" ], [ "SL.ConcurrentExamples.test20", @@ -215,7 +215,7 @@ 1, [ "@query" ], 0, - "27af949d6ec3ec80d5ba01a01d96b19f" + "afc98a5d8f05e9d5fbe2e8d6df17ed71" ], [ "SL.ConcurrentExamples.test20", @@ -236,7 +236,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "d727cd9ae53c998927c29d53f6b06e11" + "2a9b5cca2c6944fb8be3e11b2f1abe3a" ], [ "SL.ConcurrentExamples.test20", @@ -255,7 +255,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "03a79c801190b0404a7726b4dd09b6aa" + "45e509bb9c758f9d1063b9f928a0fc6e" ], [ "SL.ConcurrentExamples.test20", @@ -267,7 +267,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "b6d3bafaaf54535db2cca51dcdcfdca3" + "244a0886e32c2af6de7cd4ceef0a9dd0" ], [ "SL.ConcurrentExamples.test21", @@ -292,7 +292,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "198885c1243a61250f2fa2a29668c764" + "c6dc478c8850be3ec75ccb273562a012" ], [ "SL.ConcurrentExamples.test21", @@ -317,7 +317,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "35f85c7fc32c281646bdfe2cd4fef162" + "a8d2e1724c2018d3da7b72769b88df09" ], [ "SL.ConcurrentExamples.test21", @@ -340,7 +340,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "190d4e85d86d40ab65d6e2baea8516b2" + "2259c1e81e64590a271e4d55f02585b6" ], [ "SL.ConcurrentExamples.test21", @@ -349,7 +349,7 @@ 1, [ "@query" ], 0, - "c155d619b782b4e55f55dda3bf7927dc" + "233580a6b6379ca3b9f711f9c9307f61" ], [ "SL.ConcurrentExamples.test21", @@ -370,7 +370,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "4d925e1b2f456c2dadfcc1323a32567f" + "5f549d61dad14681dfc9f2b8c8a22a41" ], [ "SL.ConcurrentExamples.test21", @@ -389,7 +389,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "6e476f41bc0c3202cd5032f0956b0f68" + "80e09a163a3a7a90f19c95ed6bbefbde" ], [ "SL.ConcurrentExamples.test21", @@ -401,7 +401,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "7c119c55ac42178859892e43bd6df3a9" + "569109b7aee6416927a6a2c1432eea63" ], [ "SL.ConcurrentExamples.test22", @@ -424,7 +424,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "e9932707e37d44949090bf41bf922437" + "c940fa020af8a839ef622b52771a837b" ], [ "SL.ConcurrentExamples.test22", @@ -459,7 +459,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_typing" ], 0, - "ba5ac99c434e9208fd50c2eaded99944" + "35daf3e81425ed7e4428acfcc441b069" ], [ "SL.ConcurrentExamples.test22", @@ -484,7 +484,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "baa8b62d2ead912b78f0abe756d08c44" + "01886b43b296864b13f3ee48fccfa4bf" ], [ "SL.ConcurrentExamples.test22", @@ -511,7 +511,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "3c21a463e9c1e4638688376a3b38435c" + "b97e05a5237b3ce5f1ac279a59f1416c" ], [ "SL.ConcurrentExamples.test22", @@ -520,7 +520,7 @@ 1, [ "@query" ], 0, - "043537461eda7583cc21057aeab3ead6" + "d729747db0dc43a73a7fd37b7cf84e9b" ], [ "SL.ConcurrentExamples.test22", @@ -541,7 +541,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "d94280e84f6df8c5a50fec24cf772bd3" + "f22460910385c923db26ecb4d9c24274" ], [ "SL.ConcurrentExamples.test22", @@ -560,7 +560,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "2978bd018b975daa6fd56c88d11143c3" + "bff5170509f8898ec51799beca8fc06b" ], [ "SL.ConcurrentExamples.test22", @@ -572,7 +572,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "a3739e329c7ce22c8970aacaff1f1f53" + "c6d96feea850ba0af0bf417fa3a6e69d" ], [ "SL.ConcurrentExamples.test23", @@ -595,7 +595,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "a39d42984d45e3ea27667c175bd04c7b" + "7ffe32fede89983a69e9afd471223f0d" ], [ "SL.ConcurrentExamples.test23", @@ -630,7 +630,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_typing" ], 0, - "cffb51344c2a7936a3ba5065f5643f3d" + "ea5ef68e88e197636324c395e68ce4c1" ], [ "SL.ConcurrentExamples.test23", @@ -655,7 +655,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "a359ed95b0b62a3676dad4af845a5031" + "9d08feed666fb24bc95385da42bb31e4" ], [ "SL.ConcurrentExamples.test23", @@ -682,7 +682,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "7dcc574d2b29665effe535b0550f3bd0" + "5a74d86572fe66ac2b00cb0f5963bb37" ], [ "SL.ConcurrentExamples.test23", @@ -691,7 +691,7 @@ 1, [ "@query" ], 0, - "f43ab53bf30a7769b8670834debe900c" + "c27734a5888c5a9db253bb29bd9ccb51" ], [ "SL.ConcurrentExamples.test23", @@ -700,7 +700,7 @@ 1, [ "@query" ], 0, - "d6bd04b25e15bd68e99ff49be2d012c9" + "a0bf457861c4db52d7d26b40df663c56" ], [ "SL.ConcurrentExamples.test23", @@ -721,7 +721,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "5b101608c5a7dbe29c857166ec90e475" + "2e40a3fe0f27c0aa1e69cadfb9c72609" ], [ "SL.ConcurrentExamples.test23", @@ -740,7 +740,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "daf71044af247158034704e2a81b38d5" + "5715e934370b77881fcbdfc13d428bfa" ], [ "SL.ConcurrentExamples.test23", @@ -752,7 +752,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "95058b4dee680d7c88aa39c7e49aacdb" + "f14ebfd88b3742f7983abf71d90dd370" ], [ "SL.ConcurrentExamples.incr_both_swap", @@ -764,7 +764,7 @@ "refinement_interpretation_SL.ConcurrentExamples_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "3ec1a52e86a827e996c98b2bb9846483" + "c65abd3e4c31ec7adf52408d60f5151e" ], [ "SL.ConcurrentExamples.incr_both_swap", @@ -773,7 +773,7 @@ 1, [ "@query" ], 0, - "733da80f17ab981e864df5d05614b8e5" + "f3b2945e952a84ac2c8540085438ea4f" ], [ "SL.ConcurrentExamples.incr_both_swap", @@ -792,7 +792,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "d115fc1b20ffcf6d7ab996f3ce4adab2" + "4b9910f20b23e1ce7640ba236e07c924" ], [ "SL.ConcurrentExamples.incr_both_swap", @@ -815,7 +815,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "10e3772e528b3cf12c9bb36058f9c7ba" + "de6b6e3b671ae1ae5a1e7f6b6304c8bb" ], [ "SL.ConcurrentExamples.incr_both_swap", @@ -833,7 +833,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "ae5102e11e9a6b5065b1d4ec26401148" + "c340a86e29065e31aac422099d6c89c8" ], [ "SL.ConcurrentExamples.incr_both_swap", @@ -852,7 +852,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "4f90becc0b2c1ba4555e95598203d799" + "6b6bb2f682d8bacefc75cb310f97af26" ], [ "SL.ConcurrentExamples.acq_step", @@ -865,7 +865,7 @@ "refinement_interpretation_SL.ConcurrentExamples_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "3cbf15002d1a10d15ee9c07570f6f8ea" + "bb869d9d276bd6c913a87ab4b67eaec2" ], [ "SL.ConcurrentExamples.acq_step", @@ -892,7 +892,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_typing" ], 0, - "70d50131e4f681748c8b497739ea3e7c" + "4ff3311de44725721ba1cfd18cdcda72" ], [ "SL.ConcurrentExamples.acq_step", @@ -901,7 +901,7 @@ 1, [ "@query" ], 0, - "15750e6075ee44ec1ba774d735fd7f86" + "940d488c1bbe4ce75ac113b26432b3fc" ], [ "SL.ConcurrentExamples.acq_step", @@ -921,7 +921,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "f8d62a6e7266a0975902b22cba05949e" + "386bb4face0d25fa2432eb3dfdbea699" ], [ "SL.ConcurrentExamples.acq_step", @@ -933,7 +933,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "fe8b3c7355668d1950f437b5b56b7a36" + "e40dcc0fbbf37bd3f006bfde37c5e7ae" ], [ "SL.ConcurrentExamples.test24", @@ -956,7 +956,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "7957c19069938d7a9331f34b9f734ec9" + "cadd9ab5e9b83243e23850633f26a305" ], [ "SL.ConcurrentExamples.test24", @@ -991,7 +991,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_typing" ], 0, - "937b871d50060d944f7d2b3c19bc8844" + "a602d2ccf0a21b3b078604a265dce20e" ], [ "SL.ConcurrentExamples.test24", @@ -1016,7 +1016,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "f226ba7d92720d779bc784b0055546ee" + "e8eb232d4a13d12e8e5217319061112b" ], [ "SL.ConcurrentExamples.test24", @@ -1041,7 +1041,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "070bf970bc088e0542ea92c1781be50b" + "f95be2f0176ca8171b83eaf035234e4e" ], [ "SL.ConcurrentExamples.test24", @@ -1050,7 +1050,7 @@ 1, [ "@query" ], 0, - "4dacbc2cc0929b37b9ca5c0888999309" + "568fbba1035f54596771729f4cb591c1" ], [ "SL.ConcurrentExamples.test24", @@ -1065,7 +1065,7 @@ "projection_inverse_FStar.Algebra.CommMonoid.CM_unit" ], 0, - "2239e8857b7568133e2aabf0f62212e0" + "74d10d13f627a3ea83b581da6cc6eaea" ], [ "SL.ConcurrentExamples.test24", @@ -1074,7 +1074,7 @@ 1, [ "@query" ], 0, - "53df63c632db1c74c196448c6d730b6d" + "86a83f63d68b5f3ff2cd24d1f3134002" ], [ "SL.ConcurrentExamples.test24", @@ -1095,7 +1095,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "e6c26bfb2bc1934d3b31af6c427a63b1" + "30a77ccf29fbe00e8b29d1dce8a4eecd" ], [ "SL.ConcurrentExamples.test24", @@ -1114,7 +1114,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "fdaa8961a77c92c265c93ef689f2cc4a" + "0ccc05d3e4ffc5c196477ee037843811" ], [ "SL.ConcurrentExamples.test24", @@ -1126,7 +1126,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "5d845b4b2056f2a2ec34a7160b1b5e1f" + "ca41e1d49a92a7c1bcfbc7cf8e507728" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.ExamplesAuto.fst.hints b/examples/csl/SL.ExamplesAuto.fst.hints index fd98caa3554..000b8cd1947 100644 --- a/examples/csl/SL.ExamplesAuto.fst.hints +++ b/examples/csl/SL.ExamplesAuto.fst.hints @@ -17,7 +17,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "f3a2f77e8c75049ecc054188cae282e3" + "8b4ddd318eaf4d382cac9edeb4ccae6a" ], [ "SL.ExamplesAuto.swap", @@ -36,7 +36,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "ee0ff814dc3603f6528ebbdbd7bc6c9d" + "495a0a3f825deb48c95ea3e7a46979ff" ], [ "SL.ExamplesAuto.swap", @@ -65,7 +65,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "f8b92ca6ad0a5662ab5125804a7e78da" + "b0bbd6a883ac6d10158b7a65b3cc6865" ], [ "SL.ExamplesAuto.swap", @@ -83,7 +83,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "2c90850062d15e83d967d34ae2550e30" + "edbc2f94556a53bdc2311554abe6c836" ], [ "SL.ExamplesAuto.swap", @@ -102,7 +102,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "64ab0390a7af6bca79998abde82bcc3e" + "4f3b2a2d574dbf33f0abaa9b52a66375" ], [ "SL.ExamplesAuto.rotate", @@ -121,7 +121,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "d01099e40cbca99478bf9cf37df241a4" + "dc1a306afc3926b8932743e583a0cd2b" ], [ "SL.ExamplesAuto.rotate", @@ -140,7 +140,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "9edefca1ecb28653e4eef23eb8932d83" + "5c2af0198892d91c7f89ef9430fe59ca" ], [ "SL.ExamplesAuto.rotate", @@ -160,7 +160,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "14722db3cf424045e75dbf49d8d8c136" + "e3715328c005a6c45716e6ae248b5e02" ], [ "SL.ExamplesAuto.test", @@ -178,7 +178,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "a5c4d638216fc63ef22d813f2f61ddfe" + "e28d6ba7c7df8e0efcf036d99477b143" ], [ "SL.ExamplesAuto.test", @@ -192,7 +192,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_db83beed0426cdd22c659815fb9a6f83" ], 0, - "e67dacd9e0ffbaae96b724fb1e45854e" + "b98c167478eca234724e059d079bd5f3" ], [ "SL.ExamplesAuto.write_read", @@ -210,7 +210,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "abcb62f26e3932083b41e6b4ed2d0832" + "f5a33a6af9440f441bd1e890addd0b79" ], [ "SL.ExamplesAuto.write_read", @@ -228,7 +228,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "7a078ebc2c0134b723f80925d466994a" + "d559c83672c0805595541333691e98d3" ], [ "SL.ExamplesAuto.write_read", @@ -248,7 +248,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "3fec171825a8a6478b08a49395152078" + "9013a22a68a9e9bcd0a891d0be810f6e" ], [ "SL.ExamplesAuto.read_write", @@ -266,7 +266,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "7d744ef79a83ece88bdaf28d66ee3cd5" + "8230c02c2aba73e2d36026c81d773713" ], [ "SL.ExamplesAuto.read_write", @@ -285,7 +285,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "09425b4d8e40a4e6eda4d69ee260a97c" + "5776784f744d4ce2bdc17a63c62a7216" ], [ "SL.ExamplesAuto.read_write", @@ -304,7 +304,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "bbc64f905cdb1b6db779804c21042576" + "e5a48de9be455cc92d19ffd25ae67cf3" ], [ "SL.ExamplesAuto.cond_test", @@ -316,7 +316,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "5f386163cc75d563b59b6f5b887118ee" + "7e424477e80898e5500b42a908e3fcee" ], [ "SL.ExamplesAuto.cond_test", @@ -328,7 +328,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_8359878918c830803afb203cd8a44f99" ], 0, - "c8667e63f1196b2fb523bd26c4571462" + "af2ce2b143367a7abc76c659199962cf" ], [ "SL.ExamplesAuto.cond_test", @@ -341,7 +341,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_de4dc1318c9ad6d244a7472e52c18df1" ], 0, - "a4ce8acffada039697ee2ca17a54cb36" + "01627ecd7032279dad9251ff695d333c" ], [ "SL.ExamplesAuto.cond_test", @@ -353,7 +353,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_8359878918c830803afb203cd8a44f99" ], 0, - "f97cd984b52f9dfd173130119a598bd3" + "097d1dd743ebcf8100b131ecba37a0fd" ], [ "SL.ExamplesAuto.cond_test", @@ -366,7 +366,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_de4dc1318c9ad6d244a7472e52c18df1" ], 0, - "9391fde78e917cb0f8bb176154cb0aa4" + "75c4f0c46eac1222b22ba2d87907e5dd" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -378,7 +378,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "525b6523005c919dd9560bed8e46b512" + "9a53df259192730863512d833ff0a5d7" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -394,7 +394,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "956ab42a393997b369f9a119f97cb716" + "f86957b0fe26cab60bc943411496414b" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -409,7 +409,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "3b6487ebbfbc54c162c77bb23043b863" + "90f69f56238975e8e2ca20270cd7f4f6" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -422,7 +422,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_a5f12cbf43548265004dbd7acdaa10cf" ], 0, - "a79076a4aad5e23a98466029e0c919b6" + "908719a171dd7786b92db186181c34e5" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -434,7 +434,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_65e45a2890915eacaad5ce9413efe12c" ], 0, - "234ae5624c7bcc6fe3c626c01bc7471c" + "f5b5d0c906271cd8fb1da093b3be1036" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.ExamplesLocks.fst.hints b/examples/csl/SL.ExamplesLocks.fst.hints index 90fefe9538f..640a9c60227 100644 --- a/examples/csl/SL.ExamplesLocks.fst.hints +++ b/examples/csl/SL.ExamplesLocks.fst.hints @@ -19,7 +19,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "2197077f29fa28d2a008a4e3f7079b8d" + "52081828310e5ce97d70b4c1b6734902" ], [ "SL.ExamplesLocks.test_acq", @@ -31,7 +31,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "46031a759c9c2faa54ce39255adcf854" + "67fa1ca5be38a5388e19ed4f02622670" ], [ "SL.ExamplesLocks.test_acq_rel", @@ -44,7 +44,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "621538c0131b87fc99de90234b96d47f" + "59cccd6440400d6eacd22fa293b095f7" ], [ "SL.ExamplesLocks.test_acq_rel", @@ -62,7 +62,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "49b7147bfee1a0061cf7e9b805954feb" + "04fa672b630596b0eb8ce1df12aa8bfa" ], [ "SL.ExamplesLocks.test_acq_rel", @@ -71,7 +71,7 @@ 1, [ "@query" ], 0, - "5a9b8c652170d8fe9fca43485afbad08" + "4f3064b6bd1e0effdf3b2c2a97abbbe3" ], [ "SL.ExamplesLocks.test_acq_rel", @@ -83,7 +83,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "d6851ad4d3f8fa706865ee0348a83cb7" + "cb938a0c471fe1874b6a5b2bbc42963b" ], [ "SL.ExamplesLocks.set_and_ret", @@ -96,7 +96,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "dabd10067b5698b3e626fbbdf8fdf789" + "fccea245d7e4f58fe27049516b435e1b" ], [ "SL.ExamplesLocks.set_and_ret", @@ -108,7 +108,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "48017da445de73f2285ef46aced6e5e0" + "781dde34a19b6286e785de60bac971b3" ], [ "SL.ExamplesLocks.set_and_ret", @@ -120,7 +120,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "4fd7ad60c793732b0178cc27f23240bf" + "75313c28d78dd03eba59750aaea7ed70" ], [ "SL.ExamplesLocks.set_and_ret", @@ -132,7 +132,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "691e4279c5bfbbf20a3bc866bd4eb517" + "75772fd97aa1a2faabdc353b4b818e40" ], [ "SL.ExamplesLocks.set_and_ret", @@ -150,7 +150,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "ff3a3398a867120aa79ee7a3490c8979" + "a2a0ccb83167fcaa2d256c548a8f0a2e" ], [ "SL.ExamplesLocks.set_and_ret", @@ -162,7 +162,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "6d66a705dc6ec7e08a5cbc5f5fb65e86" + "a6583a57cc6587ecfef0c2318e422cb3" ], [ "SL.ExamplesLocks.set_and_ret", @@ -174,7 +174,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "042266a7d722eb9a0f3fe24b57fac836" + "43a4c44a9a41fc113ea85c12770497aa" ], [ "SL.ExamplesLocks.set_and_ret", @@ -183,7 +183,7 @@ 1, [ "@query" ], 0, - "cbd1e5c9450edf9ba6a5c8cc90029bf1" + "4ff0cf1a7d5486796f12d5747b26465b" ], [ "SL.ExamplesLocks.set_and_ret", @@ -195,7 +195,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "44b46ed89c1164a477abeaee86b602fd" + "a4073b7cdcbd02fe63b1482a0391c03a" ], [ "SL.ExamplesLocks.set_and_ret", @@ -207,7 +207,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "3dcf38e149e116ce052354fcc83ae7cb" + "3a641d3706fef5c897d307eea8a443e5" ], [ "SL.ExamplesLocks.set_and_ret", @@ -219,7 +219,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "c8c2128da48e9fa4b8252f85693a46e8" + "8e15af5544152944ac30c9da02352ff2" ], [ "SL.ExamplesLocks.set_and_ret", @@ -231,7 +231,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "300951fd6501b9b442a4b22ce0804579" + "dadb21b291e2f355b88b62e4b93b5265" ], [ "SL.ExamplesLocks.set_and_ret", @@ -243,7 +243,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "0955eae66f42311bf7cc05795438ed13" + "5a5b0d4dfeafc9bcae7e147293af8641" ], [ "SL.ExamplesLocks.set_and_ret", @@ -255,7 +255,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "a74103165fc4e8d1c35796f3279b51b3" + "0db7d929166ff5ec97085a9f4ebe38c8" ], [ "SL.ExamplesLocks.set_and_ret", @@ -267,7 +267,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "bfe259a14371aa417abddcd373d0851f" + "ad4dd0bf2e2c0db41f51c62635c76628" ], [ "SL.ExamplesLocks.set_and_ret", @@ -279,7 +279,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "32bc37779321271b8b419667b258e26f" + "8943dbafdeb1b7e278e0fd58c0d54454" ], [ "SL.ExamplesLocks.set_and_ret", @@ -291,7 +291,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "f322ebfcb908969d3d13ab6c20ce2adb" + "542c569e0e516b09fd5a8ff2e90f10b4" ], [ "SL.ExamplesLocks.set_and_ret", @@ -303,7 +303,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "ef1d39ec0d69f24d6be6119e76547d60" + "e36ff1baf58410487bd7b0bfff59ccdc" ], [ "SL.ExamplesLocks.set_and_ret", @@ -315,7 +315,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "1f41b0358195c18ba2f3f51dcee66547" + "d905ee65fe007d2939906a22c819caa4" ], [ "SL.ExamplesLocks.set_and_ret", @@ -327,7 +327,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "5be04cfb7c090ffc2d423595d770de76" + "ac4336a8b2e1cf2b7980cecae1ab3851" ], [ "SL.ExamplesLocks.set_and_ret", @@ -339,7 +339,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "d5d6442161873aa831996184fd70b3ff" + "f7423d6c04955b41cd9d39687273dd5b" ], [ "SL.ExamplesLocks.test06", @@ -357,7 +357,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "914aa438d164227da05a7487dbd31ad6" + "615e0a685bb6d2fb8d09e9f1d11f4642" ], [ "SL.ExamplesLocks.test06", @@ -372,7 +372,7 @@ "projection_inverse_FStar.Algebra.CommMonoid.CM_unit" ], 0, - "9bc31fb276cfebb71dda065e2b83994f" + "eeaa49ec5ae56acdb533d6e9eeb24d12" ], [ "SL.ExamplesLocks.test06", @@ -381,7 +381,7 @@ 1, [ "@query" ], 0, - "337711280caba9cb43dd206facc054e5" + "16ccc981a05a9e4cff8fd9a1d29e786a" ], [ "SL.ExamplesLocks.test06", @@ -393,7 +393,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_8359878918c830803afb203cd8a44f99" ], 0, - "40564a584b3ad626ff388fce7d9344b8" + "2f2f99c3f482086fc013884778d1c243" ], [ "SL.ExamplesLocks.test07", @@ -406,7 +406,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_4b34bc22d8ccfb71814cfc1eec9117e7" ], 0, - "b143b654216ca9314ed05ede433082c0" + "74eeff3d339ae0307ce27c176770ac84" ], [ "SL.ExamplesLocks.test07", @@ -418,7 +418,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "dfeb09d351df1af0517f422fab213f8f" + "aeb07079ce2d0c68dca2d4376772618b" ], [ "SL.ExamplesLocks.test08", @@ -442,7 +442,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "fca42a33707c30f97152121e7255fe6d" + "fa7c9170cc42fa588682f12021d0ac87" ], [ "SL.ExamplesLocks.test08", @@ -454,7 +454,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_8359878918c830803afb203cd8a44f99" ], 0, - "61f44ce0aff5d302d3521ea1ad9bdb90" + "67272b659e3822622e8762f7e960d39d" ], [ "SL.ExamplesLocks.test08", @@ -472,7 +472,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "131fb915f075ce89b58bcbb95ad7e140" + "d70b14dea4db15f67e3b6849dbefa070" ], [ "SL.ExamplesLocks.test09", @@ -492,7 +492,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "ceacf5e7767b90ece6e5b323018e4eb1" + "39953bbcfea9872970eebd03772fcd9e" ], [ "SL.ExamplesLocks.test09", @@ -504,7 +504,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_8359878918c830803afb203cd8a44f99" ], 0, - "78b4dcb75510a1b55517591c0b86b55b" + "cc8ca37c11d5b8c8918dd5c0e95a8dc7" ], [ "SL.ExamplesLocks.test09", @@ -522,7 +522,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "ec55c24470e26fc9a1a8ba58c7e46406" + "ae2ebc323325038c1ac0a37121b1636e" ], [ "SL.ExamplesLocks.test10", @@ -537,7 +537,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "c012652fa2d687464f09b9b660e0c6f3" + "bb6cb524074071dd85aad89e8dbbd32c" ], [ "SL.ExamplesLocks.test10", @@ -546,7 +546,7 @@ 1, [ "@query" ], 0, - "e09d2b3d0e1be7763638eacd3b8638df" + "c68405cb68fe7ff0ced0b2d07764fbdc" ], [ "SL.ExamplesLocks.test10", @@ -558,7 +558,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "06a4268da785b6ab83cdf91b1e365bd8" + "b090d5847bb071244b8c1ce922c1f030" ], [ "SL.ExamplesLocks.test11", @@ -571,7 +571,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "f52be2ab1848e3c25587f256202ffb4c" + "592bc60ecf5143c7697ac046f6460819" ], [ "SL.ExamplesLocks.test11", @@ -580,7 +580,7 @@ 1, [ "@query" ], 0, - "eb05a0f5f010745c106afe34630c064a" + "9e67c2a9bde5a3dfc1a1ef305b26b348" ], [ "SL.ExamplesLocks.test11", @@ -589,7 +589,7 @@ 1, [ "@query" ], 0, - "ed94bc98fa56eed6870e6509570a8fc6" + "06f7e28b7e539042ef99e6a547e1ce83" ], [ "SL.ExamplesLocks.test11", @@ -601,7 +601,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "be0c3ddc51da0c6d2f34687b647c596d" + "965ea19ef0efdd10a493d5d76de14743" ], [ "SL.ExamplesLocks.take_and_incr", @@ -614,7 +614,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "f5949f62b0cb9a6b5c2462e67f858c5c" + "60e3f648dd1d5cf2b08c4a20bb0a9ff2" ], [ "SL.ExamplesLocks.take_and_incr", @@ -643,7 +643,7 @@ "typing_SL.Heap.op_Bar_Greater", "unit_typing" ], 0, - "e1c10487e3f840f609285b696570edf5" + "8f6bbf57b225b979727f6258fd623465" ], [ "SL.ExamplesLocks.take_and_incr", @@ -661,7 +661,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "c1bf8813f4105b31aa99b2f1b7a1263a" + "b12e0b908d56b17f502d9b5ab4aff020" ], [ "SL.ExamplesLocks.take_and_incr", @@ -670,7 +670,7 @@ 1, [ "@query" ], 0, - "7a1ffc85e79a1c6cf7d064c477c148d4" + "cc7842028d9eee6d9a9c2bd5cce0840e" ], [ "SL.ExamplesLocks.take_and_incr", @@ -679,7 +679,7 @@ 1, [ "@query" ], 0, - "35ef08aa9b2624501574b291f8c377b3" + "838eb0944371bde7080cd34d8185a8e7" ], [ "SL.ExamplesLocks.take_and_incr", @@ -691,7 +691,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "37f4a544af4462aaaddaf2dca90aad5d" + "58423b919ffd7160db485babce18d3ce" ], [ "SL.ExamplesLocks.test12", @@ -705,7 +705,7 @@ "unit_inversion" ], 0, - "bd1ba4ce5ae245e8a9e5d5bd73566911" + "263db9f367e8e03457bab6e075bedd63" ], [ "SL.ExamplesLocks.test12", @@ -714,7 +714,7 @@ 1, [ "@query" ], 0, - "734123856182d90f4aa6ada2ae793b47" + "c6158ba17cc247027c7c1dd33011b497" ], [ "SL.ExamplesLocks.test12", @@ -726,7 +726,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "df97eea538e0feb544154e4ebe8de54a" + "34dba27e1dfbd4d926342097be1a0b26" ], [ "SL.ExamplesLocks.test13", @@ -739,7 +739,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "ff47c23710ffd44faf84c8dc4c478bf6" + "ef51f2095dba36333653307cb7f8b230" ], [ "SL.ExamplesLocks.test13", @@ -757,7 +757,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "61e27630e7caa0b68f879512676c83f8" + "cfe70db2d126134383b78056aa7248e8" ], [ "SL.ExamplesLocks.test13", @@ -766,7 +766,7 @@ 1, [ "@query" ], 0, - "791f59cbd3a4899cff730b272d3456fc" + "6bfce31a97132e2165ba85299be3d49f" ], [ "SL.ExamplesLocks.test13", @@ -775,7 +775,7 @@ 1, [ "@query" ], 0, - "c04c2bc1d6e7d21352711b53bde363d0" + "0859fba9c7cad5b05c660c34dcc4a038" ], [ "SL.ExamplesLocks.test13", @@ -787,7 +787,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "b784448ae723e24273ec5d97ad9a6a08" + "f33e06c92794713ba1bbf9a2f5e9b55e" ], [ "SL.ExamplesLocks.test14", @@ -800,7 +800,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "37ac5880f20ce0cc1b9a366ee51745e1" + "40b4f0514cbc01c235da3b3c1b251487" ], [ "SL.ExamplesLocks.test14", @@ -818,7 +818,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "aa57f26afd4d2b44b66499819ac63db6" + "61c73e16ff8ace9cae967ad2929bb0ec" ], [ "SL.ExamplesLocks.test14", @@ -827,7 +827,7 @@ 1, [ "@query" ], 0, - "06d2a588d28e0381ca9bb48ab95f8ff0" + "e4a9ae82dd7fea721afab6a0ac26d061" ], [ "SL.ExamplesLocks.test14", @@ -842,7 +842,7 @@ "projection_inverse_FStar.Algebra.CommMonoid.CM_unit" ], 0, - "72c1b6bcbef33469f34a654dcf059a5f" + "1bfe1d9605d14bcbf6fe1e2d61a14421" ], [ "SL.ExamplesLocks.test14", @@ -851,7 +851,7 @@ 1, [ "@query" ], 0, - "75cb95eb8c4b0ca3d01968da28aa9f25" + "829e69188f1f8f759da044cd6fd941fd" ], [ "SL.ExamplesLocks.test14", @@ -860,7 +860,7 @@ 1, [ "@query" ], 0, - "0e706cc1b3b0b3bb7bfb7445c12aa2f0" + "b340dd2da5986ad97351c7f274bd9db0" ], [ "SL.ExamplesLocks.test14", @@ -872,7 +872,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "e3b3ebc289b03fd5def71e068c083782" + "618d6c7d2dc6b837f6050a1ed441da2b" ], [ "SL.ExamplesLocks.test15", @@ -885,7 +885,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "00737aeef0279d82c37bf09a23a11ccd" + "8ffe904b5c330336d96c10d9ef64670a" ], [ "SL.ExamplesLocks.test15", @@ -903,7 +903,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "26b7be419c23ab1ce3d9df7e3b027739" + "497ad0ad1a79999b816ea097296e23a4" ], [ "SL.ExamplesLocks.test15", @@ -912,7 +912,7 @@ 1, [ "@query" ], 0, - "89f2016f8f60a33f5487f3ef380890e1" + "834d2191040b7509704e190d897300cd" ], [ "SL.ExamplesLocks.test15", @@ -921,7 +921,7 @@ 1, [ "@query" ], 0, - "181ddbc835f0f78e909e9c5afb56c3d3" + "e10cc108be16a9b04ef731446c83442e" ], [ "SL.ExamplesLocks.test15", @@ -936,7 +936,7 @@ "projection_inverse_FStar.Algebra.CommMonoid.CM_unit" ], 0, - "9d2dbf0b3e0c88c799284b9cc8aa817c" + "3942d5f10c58eac47f972de930bb3f86" ], [ "SL.ExamplesLocks.test15", @@ -945,7 +945,7 @@ 1, [ "@query" ], 0, - "b62eedbf1d710fdcc4759fd6f32d6d46" + "faa00ac44fa939805097737519552004" ], [ "SL.ExamplesLocks.test15", @@ -954,7 +954,7 @@ 1, [ "@query" ], 0, - "cf017647341b7f6f6fa78f8353b6a31d" + "78d1169f6a41a61a93f58ac54d927583" ], [ "SL.ExamplesLocks.test15", @@ -966,7 +966,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "916a5cc0d7c9d9fa7aaaf6aead931446" + "991793f61703aada2f7643efd2f03b43" ], [ "SL.ExamplesLocks.test16", @@ -979,7 +979,7 @@ "refinement_interpretation_SL.ExamplesLocks_Tm_refine_80c9652fe96a19b293f5cd63a93f6e93" ], 0, - "77e782ac3072a1f4c5131c9f00ded721" + "9d4f0de9a8be7554e41906eec825f527" ], [ "SL.ExamplesLocks.test16", @@ -988,7 +988,7 @@ 1, [ "@query" ], 0, - "5d03ef998d0edc096ff3cc2a4dd27ede" + "21bd08d6e300bac9e6eef8f1059ad898" ], [ "SL.ExamplesLocks.test16", @@ -1013,7 +1013,7 @@ "typing_SL.Heap.op_Bar_Greater", "unit_typing" ], 0, - "a6097c0132061a48ec9558f552683029" + "83f7643369c6f00a01a09b6e7cde0e71" ], [ "SL.ExamplesLocks.test16", @@ -1031,7 +1031,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "24ea3de65246f9719a6ec728f4950c27" + "02657f01db88a6fcfe22b0b98dcfcdf2" ], [ "SL.ExamplesLocks.test16", @@ -1040,7 +1040,7 @@ 1, [ "@query" ], 0, - "0f35237d6c5ef84424f7ed49612cf665" + "4042e10c5848cae2a9f996cbf00ee941" ], [ "SL.ExamplesLocks.test16", @@ -1055,7 +1055,7 @@ "projection_inverse_FStar.Algebra.CommMonoid.CM_unit" ], 0, - "7240da546481f96c9833fe2939dfc37c" + "92ba7681b7726099e393e5a799bb7f66" ], [ "SL.ExamplesLocks.test16", @@ -1064,7 +1064,7 @@ 1, [ "@query" ], 0, - "5a96ee612ff20996b54fe8c67f4d1692" + "00669266e0dbc8b22d622ecd179aac82" ], [ "SL.ExamplesLocks.test16", @@ -1073,7 +1073,7 @@ 1, [ "@query" ], 0, - "bb22820d18bd2e3f32cde06e9a2ed137" + "ac1c679605dea4dccbea954b8e05971a" ], [ "SL.ExamplesLocks.test16", @@ -1085,7 +1085,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "a1282eff7498971fd916f3bcfbcbbd76" + "37b188fb93dd9520df514eda25efb6aa" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.ExamplesLocks2.fst.hints b/examples/csl/SL.ExamplesLocks2.fst.hints index 4971b3bfd6a..6cf7602e147 100644 --- a/examples/csl/SL.ExamplesLocks2.fst.hints +++ b/examples/csl/SL.ExamplesLocks2.fst.hints @@ -13,7 +13,7 @@ "unit_inversion" ], 0, - "dcbc71c244a77e89e54514e3651bd5f8" + "83300ab75739b7bc77034ae421d6b8f4" ], [ "SL.ExamplesLocks2.test17", @@ -25,7 +25,7 @@ "refinement_interpretation_SL.ExamplesLocks2_Tm_refine_cd225dd77bc8476b2ce0cc839b0de7bb" ], 0, - "86fb0d19ffbbacb50659132ca6eeaf3e" + "199871ab37ac6468fcc5eb33f6227405" ], [ "SL.ExamplesLocks2.test17'", @@ -39,7 +39,7 @@ "unit_inversion" ], 0, - "fbe94cdd14d1fc0a8186fa26e20285f5" + "3fa5c26213e493f0d8ae664b5d9c6425" ], [ "SL.ExamplesLocks2.test17'", @@ -53,7 +53,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "bfd79f582e582e8e928641e481048163" + "c56955b1a549cba7c8de6d0bcaa7f8a1" ], [ "SL.ExamplesLocks2.test18", @@ -67,7 +67,7 @@ "unit_inversion" ], 0, - "cfffb271312571142e91ee4a898cb9ab" + "d868f7fbc13be9ae193c2aa91554d30d" ], [ "SL.ExamplesLocks2.test18", @@ -88,7 +88,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "884333d915e47fee1bba8fa4a936812f" + "f965f030be389f31e0c37438ac165fbd" ], [ "SL.ExamplesLocks2.test18", @@ -107,7 +107,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "29e0875a51ad1e3e9f4c12d5194f1f6b" + "4c05ba6312d41d1d09e50227c4ff4664" ], [ "SL.ExamplesLocks2.test18", @@ -119,7 +119,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "5684b89011fcc2dd831dd0a80ba13eae" + "428a47a86a64724e93eda322b42fde0c" ], [ "SL.ExamplesLocks2.test19", @@ -133,7 +133,7 @@ "unit_inversion" ], 0, - "f58dd96d76f6cbfad1fca144e0868bf4" + "b69631ded6d95264b43bf56c34ea4291" ], [ "SL.ExamplesLocks2.test19", @@ -154,7 +154,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "57ccdfa80281db4cc2ed5b8b64822762" + "bf109b6881c8decc31b5fa295fb5a587" ], [ "SL.ExamplesLocks2.test19", @@ -173,7 +173,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "6d8006feb5dd460e198edc8bd5b09da3" + "31488928e71b03f141050c5dc2cd7df3" ], [ "SL.ExamplesLocks2.test19", @@ -185,7 +185,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "2965b97c2bba6df75efc4dfb1eb1b9b3" + "b461616d9eb00e7e336682a4e67b1e21" ], [ "SL.ExamplesLocks2.test20", @@ -206,7 +206,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "7831405148c9a28abe36f428526c7281" + "39d2ff023773ddaee7a737d4e332abe1" ], [ "SL.ExamplesLocks2.test20", @@ -215,7 +215,7 @@ 1, [ "@query" ], 0, - "ed78acd293392a1d48fc7e66afd1df8c" + "40969ebe1da80c29c4bd1dc7e5b6a677" ], [ "SL.ExamplesLocks2.test20", @@ -236,7 +236,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "8c233ab40d9fcb47bb08912fc040ca64" + "7141d7280d114b6bb66b2f90199b668f" ], [ "SL.ExamplesLocks2.test20", @@ -255,7 +255,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "82f5e484eb8ee0f885aabf20013d3c23" + "0296de453e00e096e04b52c1eff909d0" ], [ "SL.ExamplesLocks2.test20", @@ -267,7 +267,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "f2d6b4cdef3775bc826584e3cfeae9ec" + "29aaa2dab2895bedeeb8bfed4cd79b3e" ], [ "SL.ExamplesLocks2.test21", @@ -292,7 +292,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "a17c493bd9c7aa853fabb8bfda1f92f3" + "184577764297f7f4db5b3dffd13c7011" ], [ "SL.ExamplesLocks2.test21", @@ -317,7 +317,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "a015b3c4a50c8cd129b4b59fddf3db34" + "5271465b5c575a09666a7a37e90a1a73" ], [ "SL.ExamplesLocks2.test21", @@ -340,7 +340,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "3f791d821d38a415de33fd5a621df81a" + "0622d2e4f6992be77b5a2d13f652fe3d" ], [ "SL.ExamplesLocks2.test21", @@ -349,7 +349,7 @@ 1, [ "@query" ], 0, - "7d392ce0a7ce074a76d0731d5dc31c0c" + "61192c841a8c4ce4d374db6ecfbbd882" ], [ "SL.ExamplesLocks2.test21", @@ -370,7 +370,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "cb62bfea2d56ab6884cd5035610941c6" + "6ffe417f8a8d2e00af7512e7fc5032dc" ], [ "SL.ExamplesLocks2.test21", @@ -389,7 +389,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "5f781a638aefbb828bc7be31fce297eb" + "6456bac05111ac5d20f93c09c873727a" ], [ "SL.ExamplesLocks2.test21", @@ -401,7 +401,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "000876f8690a4bf584b73be677e66bbf" + "8f933db4e5e80a820ae5a2b2f243f8f3" ], [ "SL.ExamplesLocks2.test22", @@ -424,7 +424,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "36f25536d1d8057014f8959ce6936db2" + "0b1202a561bb63addba42d2a4e0c75cf" ], [ "SL.ExamplesLocks2.test22", @@ -459,7 +459,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_typing" ], 0, - "eadc1255b31d54516d7a857796c127b0" + "e06cfe262b74199ec7dd6e3bb3c99400" ], [ "SL.ExamplesLocks2.test22", @@ -484,7 +484,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "d1615472d8c601056a2207854f92a468" + "e139a20395c0362b65b16114b3eab935" ], [ "SL.ExamplesLocks2.test22", @@ -511,7 +511,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "8cca312bf02dc42e1761a03cc1364a94" + "0460deaa33b7210c23646b75aac9009b" ], [ "SL.ExamplesLocks2.test22", @@ -520,7 +520,7 @@ 1, [ "@query" ], 0, - "4b2d59088cf948a56e1fb07b6b0ba2f1" + "15cc2744cc8cc2ad742aaae6551369d7" ], [ "SL.ExamplesLocks2.test22", @@ -541,7 +541,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "4e1ecd0f2432f68da7ea1ddf38c2c13d" + "bbe64144634a0244efef361300d1a3a2" ], [ "SL.ExamplesLocks2.test22", @@ -560,7 +560,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "79bc0da138cd924ef978ca77e89d0a9a" + "dce8c005fe500681ce8a98ceebe7045f" ], [ "SL.ExamplesLocks2.test22", @@ -572,7 +572,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "5427c23c894fe6016671529ef8d4e181" + "07357b9218ac330a58ac920527c5db96" ], [ "SL.ExamplesLocks2.test23", @@ -595,7 +595,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_inversion" ], 0, - "26cd72898186f9b65c8648c038db19e6" + "5cc753bd36512ac46347fbc2f2c42137" ], [ "SL.ExamplesLocks2.test23", @@ -630,7 +630,7 @@ "typing_SL.Heap.op_Less_Star_Greater", "unit_typing" ], 0, - "dceade90b5853d84e1d552d36912f968" + "1085dfb1601f6c82fc0bd8b22ef9e518" ], [ "SL.ExamplesLocks2.test23", @@ -655,7 +655,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "c2ac7ab21ddf40b31440aea5c87881b7" + "7dd397b1c4a9013b9f26ba195a316f00" ], [ "SL.ExamplesLocks2.test23", @@ -682,7 +682,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "ff226d8372e09bc0e4c948170a8f2f45" + "5bcf9891c7413d7d43f9f16817e45d3d" ], [ "SL.ExamplesLocks2.test23", @@ -691,7 +691,7 @@ 1, [ "@query" ], 0, - "4d70887decfad10c86572ed79ecd6375" + "7b3bfc62f23d65370821ebbea66bf321" ], [ "SL.ExamplesLocks2.test23", @@ -700,7 +700,7 @@ 1, [ "@query" ], 0, - "01ff041b6e298d56eaf685885d0e59df" + "34f24cf4f2e978b1933d02f401a9aecd" ], [ "SL.ExamplesLocks2.test23", @@ -721,7 +721,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "1222bdf5861c147f11cdae59e5b598c6" + "d5d2f4924f4628bd3d953f163b2c8da7" ], [ "SL.ExamplesLocks2.test23", @@ -740,7 +740,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "6d77d3dabf933617882c9fe2e1d19311" + "db73f1c06761efb432bd1c04bdaeaba3" ], [ "SL.ExamplesLocks2.test23", @@ -752,7 +752,7 @@ "lemma_SL.Heap.lemma_sep_unit_" ], 0, - "27beda4a27a46fb15d9a54920bf20716" + "d8ba147e18f3100e0ba7b31ca1f4e571" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.ExamplesPar.fst.hints b/examples/csl/SL.ExamplesPar.fst.hints index 1b50bd8da2f..0b297171875 100644 --- a/examples/csl/SL.ExamplesPar.fst.hints +++ b/examples/csl/SL.ExamplesPar.fst.hints @@ -13,7 +13,7 @@ "refinement_interpretation_SL.ExamplesPar_Tm_refine_a7ed30f75f7986ddb8ec09f2485210f5" ], 0, - "012d5204617877ef854fe5c6ca4c2d19" + "060122706bb881587dfc5542a5994a9e" ], [ "SL.ExamplesPar.right", @@ -27,7 +27,7 @@ "refinement_interpretation_SL.ExamplesPar_Tm_refine_d498339ca04b7f24aa6c67ad75cf6c85" ], 0, - "7f0d4ca8cbd75ed2b76f6e9204fe6b53" + "570b660309b95f2626eef52fd26d30ee" ], [ "SL.ExamplesPar.par1", @@ -46,7 +46,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "6b885043564054d8079e490910f12a01" + "c694984688debb9a04c9e0c8c7a28585" ], [ "SL.ExamplesPar.par1", @@ -59,7 +59,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "b1537f14977147572c2e25acbe9b256a" + "652eafc96e1426cf2f75bb2a77acc63f" ], [ "SL.ExamplesPar.par1", @@ -88,7 +88,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "5c2abc19a965aa2f6edaa77e9c5b51ed" + "ba4e3374d066eda9438bbb7fcbb9073e" ], [ "SL.ExamplesPar.par2", @@ -107,7 +107,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "2fecf06d1513a3d904509079598d9140" + "344902d4c4d7c30d741e94b6f3f9f646" ], [ "SL.ExamplesPar.par2", @@ -120,7 +120,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "a239f164e636084ec7d9d775ae083d3b" + "f5634d35d831800f9df4ac45197bedc9" ], [ "SL.ExamplesPar.par2", @@ -136,7 +136,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "03249ce456e77b0781ced9428f7f5b0c" + "7495c073bb0ac0be288432e902e93193" ], [ "SL.ExamplesPar.par3", @@ -155,7 +155,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "574d0e870cf0657f790a2db925ffa5aa" + "7ee8ed8ad3fb047cd05b7076a48c5b99" ], [ "SL.ExamplesPar.par3", @@ -168,7 +168,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "2ddf4840ba43b9fa291b8a1403f8ece9" + "36f28ae29fab0a634ae317413ca0f2e1" ], [ "SL.ExamplesPar.par3", @@ -197,7 +197,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "fa698c8c0bd01a7f5fed905b2e3d3ff1" + "7eebe13b0d51857ed2ec4803cd7e3743" ], [ "SL.ExamplesPar.par3'", @@ -216,7 +216,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "e62186e18ab6a0b2f6fc0b3c28bce6dc" + "688cb42ed99414c620350f9a110cd0b3" ], [ "SL.ExamplesPar.par3'", @@ -229,7 +229,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "cc940866240111ce29bb400edb2a2e9d" + "9bce64037a3479ba0be08e45bfc780fe" ], [ "SL.ExamplesPar.par3'", @@ -258,7 +258,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "33af0ec2f859793e99f499668ac75376" + "5d3987f1942dd1c491a38df7e79bd1cd" ], [ "SL.ExamplesPar.ret", @@ -274,12 +274,12 @@ "interpretation_SL.Effect_Tm_abs_ee3b492c1ada998fe8f6b35b3bcd82cf", "interpretation_SL.ExamplesPar_Tm_abs_9564a78966209243bce740a2fa63521c", "interpretation_SL.ExamplesPar_Tm_abs_f8ff6b4e95041d032c0e5a07c9309162", - "l_and-interp", "l_imp-interp", "l_quant_interp__10516", + "l_and-interp", "l_imp-interp", "l_quant_interp__10542", "token_correspondence_SL.Actions.lift_div_st", "token_correspondence_SL.Effect.frame_wp" ], 0, - "5f47a7835935b39004e1d661ecb430d7" + "a70af2906e891ef60835a5c779bbc6c6" ], [ "SL.ExamplesPar.set_to_2", @@ -302,13 +302,13 @@ "interpretation_SL.ExamplesPar_Tm_abs_addc6e66579cf4835b97030a5ec01935", "interpretation_SL.ExamplesPar_Tm_abs_bc9bdaee1e07889148600d86cfa17179", "interpretation_SL.ExamplesPar_Tm_abs_d5a4d9a20136220d0d9c6d3c18df52d5", - "l_imp-interp", "l_quant_interp__10521", "l_quant_interp__10529", - "l_quant_interp__7588", + "l_imp-interp", "l_quant_interp__10547", "l_quant_interp__10555", + "l_quant_interp__7614", "token_correspondence_SL.Actions.lift_div_st", "token_correspondence_SL.Effect.frame_wp", "unit_typing" ], 0, - "8f3f0b8824cb63297342b83bca2ca36d" + "c4a1908bb6ab33726547abeb7b873962" ], [ "SL.ExamplesPar.par_set", @@ -330,7 +330,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "106fbd633b360a247a771e1615af9de3" + "289a11bc89e2406c9f7435088493c836" ], [ "SL.ExamplesPar.par_set", @@ -345,7 +345,7 @@ "projection_inverse_FStar.Algebra.CommMonoid.CM_unit" ], 0, - "893205397e808273aa819f3d8e0b8415" + "514dc35e3081e6132a241110f5e3d16d" ], [ "SL.ExamplesPar.par_set", @@ -357,7 +357,7 @@ "refinement_interpretation_SL.ExamplesPar_Tm_refine_8359878918c830803afb203cd8a44f99" ], 0, - "440e3ddb650f7d2d48f7f9fe2854d25f" + "0dc7126884a8a6b2fc0b7ff811b6b233" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.Heap.fst.hints b/examples/csl/SL.Heap.fst.hints index 301d209f659..c76cda53b23 100644 --- a/examples/csl/SL.Heap.fst.hints +++ b/examples/csl/SL.Heap.fst.hints @@ -1936,7 +1936,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "5993828236ec7f37bb5ef1254c03b96b" + "d310532d2388459a8169891c72900ad2" ], [ "SL.Heap.dom_forall", @@ -1950,7 +1950,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "58f33a7a5a41e6c895489a4ff351da6f" + "399f881c96864cc0786cc369f2f21cc0" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.Heap.fsti.hints b/examples/csl/SL.Heap.fsti.hints index 9b1f10ec7d5..08410909abd 100644 --- a/examples/csl/SL.Heap.fsti.hints +++ b/examples/csl/SL.Heap.fsti.hints @@ -192,7 +192,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "bb001feff19cb49990d3fbca664633fe" + "6d315efdac93fcee073bb1bab4d50326" ], [ "SL.Heap.dom_forall", @@ -208,7 +208,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "8b01cf789cd7a12e6f5a6f622856a302" + "1eb4dad8e941c70c3928ed9faaaa86b0" ] ] ] \ No newline at end of file diff --git a/examples/csl/SL.Tactics.fst.hints b/examples/csl/SL.Tactics.fst.hints index fb0206d8e07..b8cb2648b84 100644 --- a/examples/csl/SL.Tactics.fst.hints +++ b/examples/csl/SL.Tactics.fst.hints @@ -22,7 +22,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "72279b8a9caa27eab56da5b6fc377cc8" + "b97ec9c1dcdcb7718d8ef3037e823527" ], [ "SL.Tactics.lemma_alloc_return", @@ -39,7 +39,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "dc7eebdeff83386a47aa5188dfa6b266" + "413838e8d7cefcfc769536d2e6c5a39e" ], [ "SL.Tactics.lemma_bind", @@ -53,7 +53,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "9be08a0d3e5d4ca4c944fe32ff2a8328" + "ddfec2066153a6dbabb40991fc7d304d" ], [ "SL.Tactics.lemma_eq_implies_intro", @@ -62,7 +62,7 @@ 1, [ "@query" ], 0, - "a78d30e06f8d8daa9117bd812a01a324" + "9ec6dc899cae8b2e9d7996150c26de55" ], [ "SL.Tactics.lemma_eq_implies_intro'", @@ -71,7 +71,7 @@ 1, [ "@query" ], 0, - "9a0e86fd30ed28e0076ebd04b3898a78" + "5d8906eeb62a427c41b2748fe2a0e114" ], [ "SL.Tactics.lemma_addr_not_eq_refl", @@ -86,7 +86,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "a750678568596766fd972e95cb99a9ce" + "45022114873819f4b1f7ad1c05363e10" ], [ "SL.Tactics.lemma_impl_l_cong", @@ -100,7 +100,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "bdd6986f17b0997040b53cd6c10fa3b9" + "e324578776319b00f452d67ee12d915f" ], [ "SL.Tactics.lemma_eq_l_cong", @@ -113,7 +113,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "a48815191acf8b06c69c150fbb51511c" + "4003755e1f757aaa1c00bff7ca56cd12" ], [ "SL.Tactics.lemma_eq_cong", @@ -126,7 +126,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "3b64840e8b7a46e553ffd948398ba233" + "691a5f0af8b6e3fac2119a1b440364e0" ], [ "SL.Tactics.repeat_step_select", @@ -144,7 +144,7 @@ "lemma_FStar.Pervasives.invertOption" ], 0, - "c1d860e288307729b66d83d2e3dab6fb" + "4b90eb8ae0337844bcc0fc440f2bcc5b" ], [ "SL.Tactics.lemma_read_write", @@ -156,7 +156,7 @@ "refinement_interpretation_SL.Tactics_Tm_refine_3bcf4b7474eb7f3eaa30f4c958188cd5" ], 0, - "55263fbe8cca15d42a3d70bd3c5aaa25" + "191af6df67ca7e14d68f990ec6d49bf5" ], [ "SL.Tactics.lemma_addr_not_eq_refl", @@ -171,7 +171,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "602dd5183d8f43970785270ca7e91860" + "441df1d165f0a5180c5fccc2a4d3e0d1" ], [ "SL.Tactics.repeat_step_select", @@ -189,7 +189,7 @@ "lemma_FStar.Pervasives.invertOption" ], 0, - "bea6ea0d463a37a87057562e1705ae4a" + "ca1418e9d541d674f27f6ca9ebf8a3d2" ] ] ] \ No newline at end of file diff --git a/examples/data_structures/ArrayRealized.fst.hints b/examples/data_structures/ArrayRealized.fst.hints index fbbad7c15a2..3a7d8f62e72 100644 --- a/examples/data_structures/ArrayRealized.fst.hints +++ b/examples/data_structures/ArrayRealized.fst.hints @@ -141,7 +141,7 @@ "subterm_ordering_ArrayRealized.Upd" ], 0, - "c3aefd963e4c38d6505b1e1930bd3038" + "dd9653952ec4cb5bfb7ba839260779fd" ], [ "ArrayRealized.__update__", @@ -161,7 +161,7 @@ "subterm_ordering_ArrayRealized.Seq" ], 0, - "5aefc0e065787e216bd1f6c2da579f9c" + "87428ec0e35fb024556da243bce46371" ], [ "ArrayRealized.slice", @@ -348,7 +348,7 @@ "subterm_ordering_ArrayRealized.Upd" ], 0, - "e2c69b2e305af70e21b1218d1eb0d1e5" + "ceb43944710d419e5a639267b3255fb8" ], [ "ArrayRealized.__update__", @@ -368,7 +368,7 @@ "subterm_ordering_ArrayRealized.Seq" ], 0, - "59c02fa29091c63ae9e8ed2596b5440a" + "9a75328e573973c37005b88a45e0641e" ], [ "ArrayRealized.slice", diff --git a/examples/data_structures/BinarySearchTree.fst.hints b/examples/data_structures/BinarySearchTree.fst.hints index 192008454cc..23a105a7ba7 100644 --- a/examples/data_structures/BinarySearchTree.fst.hints +++ b/examples/data_structures/BinarySearchTree.fst.hints @@ -68,7 +68,7 @@ "subterm_ordering_BinarySearchTree.Node" ], 0, - "b12f6655a59a82691e075588a5b7a42b" + "5304d0575e7badabf02f7c868b663ee2" ], [ "BinarySearchTree.all", @@ -80,13 +80,13 @@ "@fuel_correspondence_BinarySearchTree.in_tree.fuel_instrumented", "@fuel_irrelevance_BinarySearchTree.in_tree.fuel_instrumented", "@query", + "BinarySearchTree_pretyping_4fb05f28dfa2fb41ed53b888dfc12a53", "Prims_interpretation_Tm_arrow_9cb3c953faf527c316d427b2ce8bd81b", "Prims_pretyping_ae567c2fb75be05905677af440075565", "Prims_pretyping_f537159ed795b314b4e58c260361ae86", "binder_x_4fb05f28dfa2fb41ed53b888dfc12a53_1", "binder_x_76e2639fdbc6710cc1f69127f0a620f4_0", "bool_inversion", - "bool_typing", "constructor_distinct_BinarySearchTree.Leaf", - "constructor_distinct_BinarySearchTree.Node", + "bool_typing", "constructor_distinct_BinarySearchTree.Node", "disc_equation_BinarySearchTree.Leaf", "disc_equation_BinarySearchTree.Node", "equality_tok_BinarySearchTree.Leaf@tok", @@ -98,14 +98,15 @@ "projection_inverse_BinarySearchTree.Node__1", "projection_inverse_BinarySearchTree.Node__2", "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_BinarySearchTree_Tm_refine_81e4e4ff211597af5b5d1125596270a3", "refinement_interpretation_BinarySearchTree_Tm_refine_8fb9d562aed03e52df412b353233e9df", - "refinement_interpretation_BinarySearchTree_Tm_refine_ba379995ec634955e50ec495c69576d2", "subterm_ordering_BinarySearchTree.Node", "token_correspondence_BinarySearchTree.in_tree.fuel_instrumented", - "typing_BinarySearchTree.all", "typing_BinarySearchTree.in_tree" + "typing_BinarySearchTree.all", "typing_BinarySearchTree.in_tree", + "typing_tok_BinarySearchTree.Leaf@tok" ], 0, - "e16baeaf886f6566315e9e35d0f82856" + "6ff415a7a64940a3ee42bbcaf1959d53" ], [ "BinarySearchTree.is_bst", @@ -121,7 +122,7 @@ "subterm_ordering_BinarySearchTree.Node" ], 0, - "fb52d8dcbdde94cab08fd742310f22b1" + "13d7356b2d7b204fa20f21f9caa670ef" ], [ "BinarySearchTree.search", @@ -168,7 +169,7 @@ "typing_BinarySearchTree_Tm_abs_07d54406df86a0f1fa6b7e73e17b87bd" ], 0, - "36e00b78a7d7e19ffdf5a5aa611c0269" + "1af540dad5a96217b16decedb6eae65f" ], [ "BinarySearchTree.insert", @@ -233,7 +234,7 @@ "typing_tok_BinarySearchTree.Leaf@tok" ], 0, - "cbba89cef98106533ef9d9dbc9ebeac3" + "55f0531500c5be11ee71e9013f7b8513" ], [ "BinarySearchTree.tree", @@ -302,7 +303,7 @@ "subterm_ordering_BinarySearchTree.Node" ], 0, - "1f6c20622d48b7312d040246ebf71718" + "b3c824ef20050cc31fad6408b1c62e49" ], [ "BinarySearchTree.all", @@ -314,15 +315,16 @@ "@fuel_correspondence_BinarySearchTree.in_tree.fuel_instrumented", "@fuel_irrelevance_BinarySearchTree.in_tree.fuel_instrumented", "@query", + "BinarySearchTree_pretyping_4fb05f28dfa2fb41ed53b888dfc12a53", "Prims_interpretation_Tm_arrow_9cb3c953faf527c316d427b2ce8bd81b", "Prims_pretyping_ae567c2fb75be05905677af440075565", "Prims_pretyping_f537159ed795b314b4e58c260361ae86", "binder_x_4fb05f28dfa2fb41ed53b888dfc12a53_1", "binder_x_76e2639fdbc6710cc1f69127f0a620f4_0", "bool_inversion", - "bool_typing", "constructor_distinct_BinarySearchTree.Leaf", - "constructor_distinct_BinarySearchTree.Node", + "bool_typing", "constructor_distinct_BinarySearchTree.Node", "disc_equation_BinarySearchTree.Leaf", "disc_equation_BinarySearchTree.Node", + "equality_tok_BinarySearchTree.Leaf@tok", "equation_with_fuel_BinarySearchTree.in_tree.fuel_instrumented", "fuel_guarded_inversion_BinarySearchTree.tree", "int_inversion", "primitive_Prims.op_AmpAmp", "primitive_Prims.op_BarBar", @@ -331,14 +333,15 @@ "projection_inverse_BinarySearchTree.Node__1", "projection_inverse_BinarySearchTree.Node__2", "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_BinarySearchTree_Tm_refine_81e4e4ff211597af5b5d1125596270a3", "refinement_interpretation_BinarySearchTree_Tm_refine_8fb9d562aed03e52df412b353233e9df", - "refinement_interpretation_BinarySearchTree_Tm_refine_ba379995ec634955e50ec495c69576d2", "subterm_ordering_BinarySearchTree.Node", "token_correspondence_BinarySearchTree.in_tree.fuel_instrumented", - "typing_BinarySearchTree.all", "typing_BinarySearchTree.in_tree" + "typing_BinarySearchTree.all", "typing_BinarySearchTree.in_tree", + "typing_tok_BinarySearchTree.Leaf@tok" ], 0, - "d7ffe6c39f8fdbb667a2cab42fde490c" + "30e5dc8cec9865f6cb1e04b6f305c1ef" ], [ "BinarySearchTree.is_bst", @@ -354,7 +357,7 @@ "subterm_ordering_BinarySearchTree.Node" ], 0, - "bd164229ce058b1cdfe22178ef57eb04" + "9e2e0d14e70a0deb220ae5b211af5761" ], [ "BinarySearchTree.search", @@ -400,7 +403,7 @@ "typing_BinarySearchTree_Tm_abs_07d54406df86a0f1fa6b7e73e17b87bd" ], 0, - "b7303cee914b2899400c905d6b563fd6" + "828f7153b693229569a5dc0dbf6ef236" ], [ "BinarySearchTree.insert", @@ -456,7 +459,7 @@ "typing_tok_BinarySearchTree.Leaf@tok" ], 0, - "980650fab70439a6a2b38a30e4a2c61b" + "6278b9a66fa3ce16e16b4b62eee1f3a4" ] ] ] \ No newline at end of file diff --git a/examples/data_structures/BinarySearchTree0.fst.hints b/examples/data_structures/BinarySearchTree0.fst.hints index 0e278e804ed..d743000fe23 100644 --- a/examples/data_structures/BinarySearchTree0.fst.hints +++ b/examples/data_structures/BinarySearchTree0.fst.hints @@ -68,7 +68,7 @@ "subterm_ordering_BinarySearchTree0.Node" ], 0, - "c6b7860c1e6508ac3787dda9b7a3414b" + "ae0ff0c03b1e75772e27fc7e32a2d2b9" ], [ "BinarySearchTree0.insert", @@ -86,7 +86,7 @@ "subterm_ordering_BinarySearchTree0.Node" ], 0, - "fe31ef8289444eb9568afb4a12124b7c" + "8d79fa01148b40ec8df319703adb9ef2" ], [ "BinarySearchTree0.tree", @@ -155,7 +155,7 @@ "subterm_ordering_BinarySearchTree0.Node" ], 0, - "2f1b9cf9cacc5ba16166dc4da0a8c0c8" + "9ceae8a81b5673163c1db5c4c746541b" ], [ "BinarySearchTree0.insert", @@ -173,7 +173,7 @@ "subterm_ordering_BinarySearchTree0.Node" ], 0, - "18cfe528fea692f0da30f2d42850cf24" + "83e8d1e1ad20e2e677a7b22e26faae14" ] ] ] \ No newline at end of file diff --git a/examples/data_structures/BinarySearchTreeBasic.fst.hints b/examples/data_structures/BinarySearchTreeBasic.fst.hints index 7daad333a11..9f4b5069e36 100644 --- a/examples/data_structures/BinarySearchTreeBasic.fst.hints +++ b/examples/data_structures/BinarySearchTreeBasic.fst.hints @@ -68,7 +68,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "5e95f4ec70b87265946c4190357c5468" + "1d17d8d8b0d438f0a6cf777c00786d1f" ], [ "BinarySearchTreeBasic.all", @@ -80,13 +80,13 @@ "@fuel_correspondence_BinarySearchTreeBasic.in_tree.fuel_instrumented", "@fuel_irrelevance_BinarySearchTreeBasic.in_tree.fuel_instrumented", "@query", + "BinarySearchTreeBasic_pretyping_7e2d337133ee482b75591994ee2d6817", "Prims_interpretation_Tm_arrow_9cb3c953faf527c316d427b2ce8bd81b", "Prims_pretyping_ae567c2fb75be05905677af440075565", "Prims_pretyping_f537159ed795b314b4e58c260361ae86", "binder_x_76e2639fdbc6710cc1f69127f0a620f4_0", "binder_x_7e2d337133ee482b75591994ee2d6817_1", "bool_inversion", - "bool_typing", "constructor_distinct_BinarySearchTreeBasic.Leaf", - "constructor_distinct_BinarySearchTreeBasic.Node", + "bool_typing", "constructor_distinct_BinarySearchTreeBasic.Node", "disc_equation_BinarySearchTreeBasic.Leaf", "disc_equation_BinarySearchTreeBasic.Node", "equality_tok_BinarySearchTreeBasic.Leaf@tok", @@ -98,15 +98,16 @@ "projection_inverse_BinarySearchTreeBasic.Node__2", "projection_inverse_BinarySearchTreeBasic.Node_n", "projection_inverse_BoxBool_proj_0", - "refinement_interpretation_BinarySearchTreeBasic_Tm_refine_86f87430bb88920f175156c281ad66c2", "refinement_interpretation_BinarySearchTreeBasic_Tm_refine_b4ba2096e786a03bd781e044eb85f053", + "refinement_interpretation_BinarySearchTreeBasic_Tm_refine_e8ee330683702b2405d81a17f5fd5420", "subterm_ordering_BinarySearchTreeBasic.Node", "token_correspondence_BinarySearchTreeBasic.in_tree.fuel_instrumented", "typing_BinarySearchTreeBasic.all", - "typing_BinarySearchTreeBasic.in_tree" + "typing_BinarySearchTreeBasic.in_tree", + "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "fe5175dc20aad84cd3cf41b101662944" + "5a79068367b3556f05c137f6ecddbd17" ], [ "BinarySearchTreeBasic.is_bst", @@ -122,7 +123,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "56333dec948cdc6123ba68ae8099f68a" + "c84e912c5ea5b6352987f6c38db76bcc" ], [ "BinarySearchTreeBasic.search", @@ -175,7 +176,7 @@ "typing_BinarySearchTreeBasic.is_bst" ], 0, - "3e8e0761c7da16bfc2092cb95df67529" + "ee58966990f177de69c05c82791593ba" ], [ "BinarySearchTreeBasic.insert", @@ -243,7 +244,7 @@ "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "48a397aec11a980b43780e4016568027" + "43de3573babfec0e38199e460226391d" ], [ "BinarySearchTreeBasic.insert'", @@ -309,7 +310,7 @@ "typing_BinarySearchTreeBasic.is_bst" ], 0, - "92df77e6dc34c5517bd64c3b2a88a87e" + "60a20904ced8d480405953b97471f63f" ], [ "BinarySearchTreeBasic.insert''", @@ -327,7 +328,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "04094cb09ae0fa20e7a52ce7d60f15b8" + "ed46dd298abec29df81f4488c3bcdd26" ], [ "BinarySearchTreeBasic.insert_lemma", @@ -458,7 +459,7 @@ "typing_BinarySearchTreeBasic.uu___is_Node" ], 0, - "89115cbc2424940c39e5de52cf61383c" + "afa85b1feea481e69a8699dad019ae2e" ], [ "BinarySearchTreeBasic.find_max'", @@ -477,7 +478,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "62b0e4e4a311a0c3cd567e25652c5395" + "8683b3141e31c8cae7bc1ba1a2764e95" ], [ "BinarySearchTreeBasic.find_max_lemma", @@ -682,7 +683,7 @@ "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "363f6e1e73e188bd58d4fc7b12637a94" + "cbbc6848de0f9559bfcbd71db735f1d8" ], [ "BinarySearchTreeBasic.delete'", @@ -706,7 +707,7 @@ "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "7f77b2d88fca82b19a0f205c0b017db2" + "322573cd49c79c28e8ce56baf76740ef" ], [ "BinarySearchTreeBasic.delete_lemma", @@ -859,7 +860,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "fb89d6bcd3d9c2bd3c5e9d8643f96017" + "1167a5428f657fafe544566b82072cb3" ], [ "BinarySearchTreeBasic.all", @@ -871,15 +872,16 @@ "@fuel_correspondence_BinarySearchTreeBasic.in_tree.fuel_instrumented", "@fuel_irrelevance_BinarySearchTreeBasic.in_tree.fuel_instrumented", "@query", + "BinarySearchTreeBasic_pretyping_7e2d337133ee482b75591994ee2d6817", "Prims_interpretation_Tm_arrow_9cb3c953faf527c316d427b2ce8bd81b", "Prims_pretyping_ae567c2fb75be05905677af440075565", "Prims_pretyping_f537159ed795b314b4e58c260361ae86", "binder_x_76e2639fdbc6710cc1f69127f0a620f4_0", "binder_x_7e2d337133ee482b75591994ee2d6817_1", "bool_inversion", - "bool_typing", "constructor_distinct_BinarySearchTreeBasic.Leaf", - "constructor_distinct_BinarySearchTreeBasic.Node", + "bool_typing", "constructor_distinct_BinarySearchTreeBasic.Node", "disc_equation_BinarySearchTreeBasic.Leaf", "disc_equation_BinarySearchTreeBasic.Node", + "equality_tok_BinarySearchTreeBasic.Leaf@tok", "equation_with_fuel_BinarySearchTreeBasic.in_tree.fuel_instrumented", "fuel_guarded_inversion_BinarySearchTreeBasic.tree", "int_inversion", "primitive_Prims.op_AmpAmp", "primitive_Prims.op_BarBar", @@ -888,15 +890,16 @@ "projection_inverse_BinarySearchTreeBasic.Node__2", "projection_inverse_BinarySearchTreeBasic.Node_n", "projection_inverse_BoxBool_proj_0", - "refinement_interpretation_BinarySearchTreeBasic_Tm_refine_86f87430bb88920f175156c281ad66c2", "refinement_interpretation_BinarySearchTreeBasic_Tm_refine_b4ba2096e786a03bd781e044eb85f053", + "refinement_interpretation_BinarySearchTreeBasic_Tm_refine_e8ee330683702b2405d81a17f5fd5420", "subterm_ordering_BinarySearchTreeBasic.Node", "token_correspondence_BinarySearchTreeBasic.in_tree.fuel_instrumented", "typing_BinarySearchTreeBasic.all", - "typing_BinarySearchTreeBasic.in_tree" + "typing_BinarySearchTreeBasic.in_tree", + "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "568a9e6566792f506fdcbff936d69383" + "c066df0136ebf91525202cc42fbd6087" ], [ "BinarySearchTreeBasic.is_bst", @@ -912,7 +915,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "1f6239eab63d05aae502f7a4b96d2f45" + "1f818a839765ca7857f5fd563475fbce" ], [ "BinarySearchTreeBasic.search", @@ -964,7 +967,7 @@ "typing_BinarySearchTreeBasic.is_bst" ], 0, - "8a78839f2cac5574a05c99ce3010cc92" + "72c7abd775bf08b827fd1f4b0584f15c" ], [ "BinarySearchTreeBasic.insert", @@ -1023,7 +1026,7 @@ "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "938f8e7266be92736f6f14536d0aa064" + "cc54af2d1f932fbf09f08446ccd25508" ], [ "BinarySearchTreeBasic.insert'", @@ -1080,7 +1083,7 @@ "typing_BinarySearchTreeBasic.is_bst" ], 0, - "6a3d5b3953e8e9be249d437a28ff928d" + "59fcf37f230042c2657f384c5034ed64" ], [ "BinarySearchTreeBasic.insert''", @@ -1098,7 +1101,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "775db9f5affdf81396232c3d48b3b932" + "989e0b15a2ed9f3eedc5b8df4ffbb22c" ], [ "BinarySearchTreeBasic.insert_lemma", @@ -1164,7 +1167,7 @@ "typing_BinarySearchTreeBasic.uu___is_Node" ], 0, - "bb86cb9ddb07ccc47015a19fba9d35fc" + "f804c33e314cc80882ce10325f02d6b4" ], [ "BinarySearchTreeBasic.find_max'", @@ -1183,7 +1186,7 @@ "subterm_ordering_BinarySearchTreeBasic.Node" ], 0, - "f2d4700109b7415c048d70d720db4ce1" + "a34d5ed8417e8a5bc85d9e10e4c8fda9" ], [ "BinarySearchTreeBasic.find_max_lemma", @@ -1278,7 +1281,7 @@ "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "37ef53e1901c6253e67a4763a36a3f96" + "568277a74d0fa5917f984191eb0572fe" ], [ "BinarySearchTreeBasic.delete'", @@ -1302,7 +1305,7 @@ "typing_tok_BinarySearchTreeBasic.Leaf@tok" ], 0, - "e41d7ddbed0b1747dc54bea8809fc303" + "32dbe5e20ad6e1d0b1ab8d36655d247f" ], [ "BinarySearchTreeBasic.delete_lemma", diff --git a/examples/data_structures/BinarySearchTreeFirst.fst.hints b/examples/data_structures/BinarySearchTreeFirst.fst.hints index 81c2da87d34..96ea871c60f 100644 --- a/examples/data_structures/BinarySearchTreeFirst.fst.hints +++ b/examples/data_structures/BinarySearchTreeFirst.fst.hints @@ -127,7 +127,7 @@ "typing_FStar.Pervasives.Native.uu___is_None" ], 0, - "49a7105a5b881110bc5e14182774c655" + "b6ecb302ae27348ba2b21b53b3ff7438" ], [ "BinarySearchTreeFirst.contains", @@ -151,7 +151,7 @@ "subterm_ordering_FStar.Pervasives.Native.Some" ], 0, - "156929a1ca4dd706d1aa94b5af5d31b4" + "6efd3d5908946267a0bcfc4c5fddcd0a" ], [ "BinarySearchTreeFirst.in_order_opt", @@ -174,7 +174,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "cb201a674e6dd9b8e7c867b0d58dd7c7" + "08509bd01425d11b6ce5653396a7fcf0" ], [ "BinarySearchTreeFirst.index_is_max", @@ -319,7 +319,7 @@ "typing_FStar.Pervasives.Native.uu___is_None" ], 0, - "1f84aded2ddbc0b77cbb1d27b0a9ce2d" + "f8fb571b214fd1e8e5c17a8d5f8159f9" ], [ "BinarySearchTreeFirst.contains", @@ -343,7 +343,7 @@ "subterm_ordering_FStar.Pervasives.Native.Some" ], 0, - "51675566a05dde12f6b85687453a0216" + "afef8e9dca31110ef840a60ab8d81859" ], [ "BinarySearchTreeFirst.in_order_opt", @@ -366,7 +366,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "f48b23b411d4c81636de7f8a34cfed92" + "8ffe30162f656c0d4d51cf9bf28a0c37" ], [ "BinarySearchTreeFirst.index_is_max", diff --git a/examples/data_structures/BinaryTrees.fst.hints b/examples/data_structures/BinaryTrees.fst.hints index 3e6236cc601..af54bac06ba 100644 --- a/examples/data_structures/BinaryTrees.fst.hints +++ b/examples/data_structures/BinaryTrees.fst.hints @@ -65,7 +65,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "15269fb365de5e62aed1d03b1d27ad02" + "7db9054693316b14fa75809174dda402" ], [ "BinaryTrees.map", @@ -80,7 +80,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "9ababcb7671edeea131305a71969a138" + "5ee5caff6e386157355d88d725ea4e3e" ], [ "BinaryTrees.map_size", @@ -134,7 +134,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "c6fff6b864a393e0c5c04b2aa8e7fa56" + "c72d55546b60ee59dfbc0befbbe52764" ], [ "BinaryTrees.find_some", @@ -277,7 +277,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "6da233187684cd0220be9db74a013597" + "cc207690853315bed960429e16bd356a" ], [ "BinaryTrees.fold", @@ -293,7 +293,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "e920b405e6855b6730186a5c8f3fdb1b" + "8e0551aa3e3006a6f3036ae7e040ea85" ], [ "BinaryTrees.fold_map", @@ -450,7 +450,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "e4bfe9f0fd6ed9435aefbbd9e97f6c62" + "66b8b627d581816dfa8538a1e6434f4d" ], [ "BinaryTrees.revert_involutive", @@ -582,7 +582,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "c12e89db664d5819697e039ebaba41ea" + "931a10a26eebd8201b86f02ab46dd4e6" ], [ "BinaryTrees.add_root", @@ -604,7 +604,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "9ec6e2e8050e959abf7732e3d553326b" + "13d0eaa99f1b1a3e8344c73b4dab813f" ], [ "BinaryTrees.remove_add_root", @@ -669,7 +669,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "af61725d66dc02c20ac3b58fa121ef52" + "4a421d064548d2a3b468303bd673e65a" ], [ "BinaryTrees.remove", @@ -699,7 +699,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "9abfe5a4591217035a230a4837bf99a5" + "486b69b6b4c22adf6c9eb14e8e0d8748" ], [ "BinaryTrees.count_remove_root", @@ -847,7 +847,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "4421156fc4734c55ad4aa85860a5a201" + "bd7c181539630f121a15183a31bf2d01" ], [ "BinaryTrees.map", @@ -862,7 +862,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "a4760ea11914e6e493ad0e5a6171ffa1" + "b5b7048566dda677b88c1397b32cda33" ], [ "BinaryTrees.map_size", @@ -889,7 +889,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "51aa3fcac0390ca22d14ee205cb2da5f" + "c2f6bdc0b294d3efb8dbd7f7c4355c32" ], [ "BinaryTrees.find_some", @@ -949,7 +949,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "f157fd5e486dc9f885b9f080f9938dac" + "a3735229bdc6c8d135c61d04468ad187" ], [ "BinaryTrees.fold", @@ -965,7 +965,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "30fbda613ec810ddc08b2f9c7fb2a4a0" + "9617dcedb4e676fcb2fca7581be0d745" ], [ "BinaryTrees.fold_map", @@ -1024,7 +1024,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "0c1fa00104af2377cbb1c5e069f5864d" + "68f5dfcb4e579243bf17d24c24fe2571" ], [ "BinaryTrees.revert_involutive", @@ -1069,7 +1069,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "515ea9de6f26e4a860e0e5fc010159b6" + "879c95693af23144dbd9c75d77b5abb5" ], [ "BinaryTrees.add_root", @@ -1091,7 +1091,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "101ee5f4f72c21151805e4035d5ab3de" + "df3909c19d442946d5f73c13fc71d804" ], [ "BinaryTrees.remove_add_root", @@ -1123,7 +1123,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "249fa6634f7b76902ec43a1aa928121a" + "6a9027683450470b8a6f98c97c8ab169" ], [ "BinaryTrees.remove", @@ -1153,7 +1153,7 @@ "subterm_ordering_BinaryTrees.Node" ], 0, - "a43565e97566bbb3a9b964ddcfd120af" + "857db99ef98636fec57149a3bb241090" ], [ "BinaryTrees.count_remove_root", diff --git a/examples/data_structures/BinaryTreesEnumeration.fst.hints b/examples/data_structures/BinaryTreesEnumeration.fst.hints index 5a2ab137116..c026f30cf84 100644 --- a/examples/data_structures/BinaryTreesEnumeration.fst.hints +++ b/examples/data_structures/BinaryTreesEnumeration.fst.hints @@ -25,7 +25,7 @@ "well-founded-ordering-on-nat" ], 0, - "4c6e34bec8263330ef4f1419b8ec82af" + "1f32b037f7a8b530fda1c49720d7e057" ], [ "BinaryTreesEnumeration.pairs_with_sum", @@ -89,7 +89,7 @@ "typing_tok_BinaryTreesEnumeration.Leaf@tok" ], 0, - "c2830566b79b513680b15a0241bdc48b" + "ebadfd19ced5c19d1e59c8b0f3215807" ], [ "BinaryTreesEnumeration.trees_of_size", @@ -130,7 +130,7 @@ "well-founded-ordering-on-nat" ], 0, - "894abf1999ea864e96ad41e58754957a" + "ab7c689be11fbd87228c27451e2423cc" ], [ "BinaryTreesEnumeration.pws'_complete", @@ -173,7 +173,7 @@ "well-founded-ordering-on-nat" ], 0, - "887860ff825c61589bf5b1432e80389b" + "9b34d0c2b9768d1ba5389405abffec8c" ], [ "BinaryTreesEnumeration.pws_complete", @@ -291,7 +291,7 @@ "typing_FStar.Pervasives.Native.snd", "unit_typing" ], 0, - "bfc4011cb233bd10a561cc8d04f6e766" + "a4560acdde581d9e3b7ad709cf858446" ], [ "BinaryTreesEnumeration.flatten_app", @@ -603,7 +603,7 @@ "typing_tok_BinaryTreesEnumeration.Leaf@tok" ], 0, - "e2016aba88073be2e508fe62873850a6" + "4e3076604d99257959ad0fd9c4898fb6" ], [ "BinaryTreesEnumeration.trees_of_size", @@ -644,7 +644,7 @@ "well-founded-ordering-on-nat" ], 0, - "381e3db5231cd1a97ea4cba056ccde5d" + "578766e9686a6f3d2b29b536dafadf0e" ], [ "BinaryTreesEnumeration.pws'_complete", diff --git a/examples/data_structures/MerkleTree.fst.hints b/examples/data_structures/MerkleTree.fst.hints index 9473b6c0ffb..6ab32dc227e 100644 --- a/examples/data_structures/MerkleTree.fst.hints +++ b/examples/data_structures/MerkleTree.fst.hints @@ -247,7 +247,7 @@ "token_correspondence_MerkleTree.len" ], 0, - "24bb930cde319856bbe4561fbd327aab" + "e2a00d3fe78a561124b4a8d1bccc8377" ], [ "MerkleTree.proof", @@ -391,7 +391,7 @@ "typing_MerkleTree.lenp" ], 0, - "5b6130d57d7791e099a704678e35dfc3" + "80846d7c9079a2c13e74fd2b0bf3ef61" ], [ "MerkleTree.prover", @@ -448,7 +448,7 @@ "token_correspondence_MerkleTree.len" ], 0, - "820a31efe4313a7ae9e8710a70e04c17" + "974d0ef052a7264e48f8a8f1b7b3d313" ], [ "MerkleTree.correctness", @@ -596,7 +596,7 @@ "unit_inversion", "unit_typing" ], 0, - "e40890b35b9106c85a4254a5fb7983f5" + "e0e9f31f44ee6bdb4977207f7e0acc39" ], [ "MerkleTree.hash_collision", @@ -772,7 +772,7 @@ "typing_MerkleTree.lenp" ], 0, - "fe486aaedd11fb17e753aadefebd00b7" + "1de0984d05c2fb4289fd3707f6164573" ], [ "MerkleTree.mstring", @@ -1020,7 +1020,7 @@ "token_correspondence_MerkleTree.len" ], 0, - "e3324fcb79ee23b201138eb5c1fabdcc" + "ab859d03ab64f50ba90cf38c6418104c" ], [ "MerkleTree.proof", @@ -1114,7 +1114,7 @@ "typing_MerkleTree.lenp" ], 0, - "4b9dfe679282e571ec796172753146e2" + "4705efa1bb2592143731ae42639b1191" ], [ "MerkleTree.prover", @@ -1159,7 +1159,7 @@ "token_correspondence_MerkleTree.len" ], 0, - "0931d6b23290b90570e454d72998ef59" + "69ab7e9b16246f12769dd4b2fe1fcdd9" ], [ "MerkleTree.correctness", @@ -1282,7 +1282,7 @@ "typing_MerkleTree.lenp", "typing_Prims.__proj__Cons__item__tl" ], 0, - "4bc0c4584c535e8dfe364fee7fe471e9" + "b9c7b9dd8940fb972f46f3aa4b676084" ] ] ] \ No newline at end of file diff --git a/examples/data_structures/RBTree.fst.hints b/examples/data_structures/RBTree.fst.hints index 87d96717217..571001bd6db 100644 --- a/examples/data_structures/RBTree.fst.hints +++ b/examples/data_structures/RBTree.fst.hints @@ -98,7 +98,7 @@ "subterm_ordering_RBTree.T" ], 0, - "5d04607ffc9384768b89cd7ac0445143" + "e47f952c182e1bf3c1035f32f9c82991" ], [ "RBTree.min_elt", @@ -115,7 +115,7 @@ "typing_RBTree.uu___is_T" ], 0, - "b8ff1115afe0b4e48b1b9788b5f3876a" + "cf1c8ee404050ea8a1538b4592b3cf08" ], [ "RBTree.max_elt", @@ -132,7 +132,7 @@ "typing_RBTree.uu___is_T" ], 0, - "38f1c9f7e226359f976dbb81451895af" + "4b6afdc7ac55ee9c016c0823a3e66a26" ], [ "RBTree.r_inv", @@ -162,7 +162,7 @@ "subterm_ordering_RBTree.T", "typing_RBTree.__proj__T__item__col" ], 0, - "e65c8cca123f3722ab3292faab37c4d8" + "96969f85343ef2220e9a206af0e65bd0" ], [ "RBTree.k_inv", @@ -180,7 +180,7 @@ "projection_inverse_RBTree.T_right", "subterm_ordering_RBTree.T" ], 0, - "ee6104b3cd87fa65546b3bb4afbcdf75" + "6b377f72d969f904ef36d72b887877b7" ], [ "RBTree.in_tree", @@ -200,7 +200,7 @@ "subterm_ordering_RBTree.T" ], 0, - "8d06f08abd3966e63fa82ecde867ade7" + "489ddedc082cf7ece128939fa153cc74" ], [ "RBTree.not_c_inv", @@ -436,7 +436,7 @@ "typing_tok_RBTree.E@tok" ], 0, - "2c7762df4b8fbbdeb45dbbd1b0fe2ce5" + "01d63c880e578410ee6fdcdd44bc49ef" ], [ "RBTree.make_black", @@ -633,7 +633,7 @@ "subterm_ordering_RBTree.T" ], 0, - "9d0ed4c955169115facc37a3fce5c0e1" + "f5a80e60c5a5880c9b21f4df0b31317b" ], [ "RBTree.min_elt", @@ -650,7 +650,7 @@ "typing_RBTree.uu___is_T" ], 0, - "25497f2fef5939a52e39e5fdc97d5e43" + "fe2f763fa057114c3a77e246d1950e11" ], [ "RBTree.max_elt", @@ -667,7 +667,7 @@ "typing_RBTree.uu___is_T" ], 0, - "8bb99a407f41deea14422d0d1c972588" + "bd3b7e5babd062e553746c12784b4f74" ], [ "RBTree.r_inv", @@ -697,7 +697,7 @@ "subterm_ordering_RBTree.T", "typing_RBTree.__proj__T__item__col" ], 0, - "b313b3cab36f55edc77996afb1359be2" + "986f8a08ac73ebddd0ed9fa71c73ae4f" ], [ "RBTree.k_inv", @@ -715,7 +715,7 @@ "projection_inverse_RBTree.T_right", "subterm_ordering_RBTree.T" ], 0, - "ae43ac1e6e0e35dd3f5cec7071ddd0f7" + "9126d8d49173efa046f751e68495c3c3" ], [ "RBTree.in_tree", @@ -735,7 +735,7 @@ "subterm_ordering_RBTree.T" ], 0, - "f6462f395e634fc0f96c26d037d7b1b9" + "db211d973aa9a33df9c30cebf35532ae" ], [ "RBTree.not_c_inv", @@ -955,7 +955,7 @@ "typing_tok_RBTree.E@tok" ], 0, - "b78c299d89dbd13217795b72c5dcb12c" + "8b80f58e86de294d56b6328b9ed3b9ab" ], [ "RBTree.make_black", diff --git a/examples/data_structures/Vector.fst.hints b/examples/data_structures/Vector.fst.hints index 5a1b9abc3c9..5d6b20d6dd7 100644 --- a/examples/data_structures/Vector.fst.hints +++ b/examples/data_structures/Vector.fst.hints @@ -129,7 +129,7 @@ "well-founded-ordering-on-nat" ], 0, - "a0ba3b043972c7fe35934eb86942491c" + "ff31816a973c050b2fa90e7ca1ea9019" ], [ "Vector.append", @@ -165,7 +165,7 @@ "well-founded-ordering-on-nat" ], 0, - "7bc4c4e13155c8c7d5aca107abac2bd5" + "6a4d82fb9da4856752fe90cb0c7c42fd" ], [ "Vector.reverse", @@ -186,7 +186,7 @@ "well-founded-ordering-on-nat" ], 0, - "f62aea2250143fc6d97b06dfeaf2704b" + "a6b92c31f3daf6c957bff9e680869520" ], [ "Vector.mapT", @@ -207,7 +207,7 @@ "well-founded-ordering-on-nat" ], 0, - "28efea2cab4cfc176a2ae7c56aaa2713" + "1bfd6704c186adb87f0f9f7daf7c7a24" ], [ "Vector.fold_left", @@ -228,7 +228,7 @@ "well-founded-ordering-on-nat" ], 0, - "272db1bb6f65884cb414ff6891653f0f" + "753544bd662a48ae2a247fc81f108213" ], [ "Vector.fold_right", @@ -248,7 +248,7 @@ "well-founded-ordering-on-nat" ], 0, - "3b4f6f39528639dd10ad6a2907234b0c" + "ad8ff3602da60c7f0aadf48df46afe3e" ], [ "Vector.find", @@ -269,7 +269,7 @@ "well-founded-ordering-on-nat" ], 0, - "fd58d94e83800017abd645e11c5539e2" + "4f331440ef5d6fc0cddbee77034c172b" ], [ "Vector.zip'", @@ -291,7 +291,7 @@ "well-founded-ordering-on-nat" ], 0, - "cf366f520873ef19110704220ce31bc1" + "34a6b87c793d1522e45de810597f22c6" ], [ "Vector.vector", @@ -408,7 +408,7 @@ "well-founded-ordering-on-nat" ], 0, - "7e10f00118c90d9945618103e96aa032" + "066ec2fdc80195e390d089ba35aeeea5" ], [ "Vector.append", @@ -431,7 +431,7 @@ "well-founded-ordering-on-nat" ], 0, - "1023fd38c0ded81a7b9d1461f92dcf10" + "68501856c9940e7c134a24806f9ceba3" ], [ "Vector.reverse", @@ -452,7 +452,7 @@ "well-founded-ordering-on-nat" ], 0, - "c082ffb644ff856e1c296296a90cb7eb" + "73a9d9606539bb665d67ec24b3b044d3" ], [ "Vector.mapT", @@ -473,7 +473,7 @@ "well-founded-ordering-on-nat" ], 0, - "bcef0f403378eb2b9237e9c57b7439b0" + "9c76bce660c4e629c7fb35ff88895ccd" ], [ "Vector.fold_left", @@ -494,7 +494,7 @@ "well-founded-ordering-on-nat" ], 0, - "dd80a640ec31919b96b41a6ddb92a438" + "fe34abdac2128b09294e42f82f90af4d" ], [ "Vector.fold_right", @@ -514,7 +514,7 @@ "well-founded-ordering-on-nat" ], 0, - "e4146a720e09b1d30b17b68fd5e8db7c" + "a5625006f996f54f064b24adc2c23955" ], [ "Vector.find", @@ -535,7 +535,7 @@ "well-founded-ordering-on-nat" ], 0, - "53628e80bc71ad1c61b10fbdf8ec5a9e" + "2209c112ae4097206f92fc273542da2e" ], [ "Vector.zip'", @@ -557,7 +557,7 @@ "well-founded-ordering-on-nat" ], 0, - "5230d95cd39d6a661bd8aaf2815ac5ee" + "1331a8f9755cf8c53a8ee7b58cb217c5" ] ] ] \ No newline at end of file diff --git a/examples/dm4free/FStar.DM4F.Heap.ST.fst.hints b/examples/dm4free/FStar.DM4F.Heap.ST.fst.hints index aca08438bf8..e4c9dcea6ba 100644 --- a/examples/dm4free/FStar.DM4F.Heap.ST.fst.hints +++ b/examples/dm4free/FStar.DM4F.Heap.ST.fst.hints @@ -272,7 +272,7 @@ "well-founded-ordering-on-nat" ], 0, - "c892856ed8951212058a6dbd24b5bdd6" + "67d2d07baaefa3c593da45cc58f89b9b" ], [ "FStar.DM4F.Heap.ST.refine_st", @@ -610,7 +610,7 @@ "well-founded-ordering-on-nat" ], 0, - "00a14bf0319871cb48f8c4d366eb694c" + "5157d4e126b8f9190612865bf4847a63" ], [ "FStar.DM4F.Heap.ST.refine_st", diff --git a/examples/kv_parsing/EnumParsing.fst.hints b/examples/kv_parsing/EnumParsing.fst.hints index 7ed9f847285..ba138c357ac 100644 --- a/examples/kv_parsing/EnumParsing.fst.hints +++ b/examples/kv_parsing/EnumParsing.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq" ], 0, - "0bf1836476dd77be103beb3223df9b5d" + "7678cca2f19728c28f3f2a3953f5b4c5" ], [ "EnumParsing.__proj__OneNum__item__n", @@ -21,7 +21,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_4f83c2c575e4b9df7e99e95590ac6726" ], 0, - "203bf3e88e8d7769cc4346b97711632a" + "c84b2d69c9f8ba1bbc3964e747466cca" ], [ "EnumParsing.__proj__TwoNums__item__n", @@ -35,7 +35,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_f7b177f0e5c9dfa961ddcd32747ed85b" ], 0, - "a76ecf405c3d11e36325e4d60bc0cd0a" + "d873833d1aefea175fc1a4b20c004fd8" ], [ "EnumParsing.__proj__TwoNums__item__m", @@ -49,7 +49,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_f7b177f0e5c9dfa961ddcd32747ed85b" ], 0, - "f4d124d2cf94f79b3cb2d70dcd87bb6f" + "0f90aae0a2254d1089613fe45dd3b1f4" ], [ "EnumParsing.numbers_tag_val", @@ -64,7 +64,7 @@ "fuel_guarded_inversion_EnumParsing.numbers" ], 0, - "e1fd3fbebd432ea8555fab7827455825" + "3ebacffaaa264a8f8f6c09ce97454c39" ], [ "EnumParsing.parse_numbers_tag", @@ -93,7 +93,7 @@ "typing_FStar.UInt32.v", "typing_FStar.UInt8.v" ], 0, - "8b51ef0ff428a03d3bc6115998197230" + "21297ca76e6266c85f346b71882dcbfd" ], [ "EnumParsing.parse_Nothing", @@ -107,7 +107,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "3ad114381c4d304e1601932d263404bb" + "7ebbf34d138a82e4f75d3c989c1c444e" ], [ "EnumParsing.parse_OneNum", @@ -121,7 +121,7 @@ "projection_inverse_EnumParsing.OneNum_n" ], 0, - "69f829f980db00b5708409fa4959438e" + "6f16510bae45989b127b06b9e024ff4e" ], [ "EnumParsing.parse_TwoNums", @@ -136,7 +136,7 @@ "projection_inverse_EnumParsing.TwoNums_n" ], 0, - "e048a44f7e1f3c6b46c8035403ba6e5a" + "1f64d8541af0bb20aba792cdf1b661f5" ], [ "EnumParsing.parser_forget", @@ -157,7 +157,7 @@ "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b" ], 0, - "cdb516bb0b31b1d70444d1c968234e58" + "3a498cd6f18c98bae493161dc5f75310" ], [ "EnumParsing.validate_ok", @@ -176,7 +176,7 @@ "refinement_interpretation_Parsing_Tm_refine_2c4ed52ca61af0afe406eb07485d9cb6" ], 0, - "b8b1c274e10c7819b1ebabdfbb13a430" + "4ebf358b5804256f2d0844780cb7404c" ], [ "EnumParsing.parser_forget_ok", @@ -197,7 +197,7 @@ "projection_inverse_FStar.Pervasives.Native.Some_v" ], 0, - "078f4a5c5d4001184c590b4c492f83af" + "789b7a7476517616d0dc639e835f47dc" ], [ "EnumParsing.make_correct", @@ -211,7 +211,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_e0227620956763aa0703230757ef418a" ], 0, - "fe930b1dd948bc1023773c5b2c53852a" + "c84a18d54282898b603604e5d4582b03" ], [ "EnumParsing.validate_Nothing_pure", @@ -247,7 +247,7 @@ "typing_FStar.Seq.Base.length", "typing_tok_EnumParsing.Nothing@tok" ], 0, - "3f87c95f04b23a5aae6bf65579c6ca48" + "bdcad8dafc80e4a5f5179154a55552f6" ], [ "EnumParsing.validate_OneNum_pure", @@ -308,7 +308,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "51468e28b5b04462889a4ed96b8def50" + "8fc3a525ec52e4a64409cc71974ef272" ], [ "EnumParsing.validate_TwoNums_pure", @@ -390,7 +390,7 @@ "typing_FStar.UInt32.v", "typing_tok_EnumParsing.Nothing@tok" ], 0, - "ea30de02aa318a86a88dc3cf253259ba" + "4a8c1ec009309f277d1018e27350ece2" ], [ "EnumParsing.validate_numbers_data_pure", @@ -419,7 +419,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "848b448a179685c964552acbf414df9d" + "04e426b2e4698ef56a9f7b43f4718651" ], [ "EnumParsing.seq_pure_validate", @@ -462,7 +462,7 @@ "typing_FStar.UInt32.v" ], 0, - "22ae1760f57d01f7befac0208eb9e27a" + "6974a26a1565f76decf64a79e0b12d95" ], [ "EnumParsing.lemma_seq_pure_validate_A2_ok", @@ -532,7 +532,7 @@ "typing_Parsing_Tm_abs_def4c30b0e696cb7641fc338f7922e40" ], 0, - "5affb0968e1cafc1d1c7cb0853c39d16" + "605113c0b2bc0e6d3cecdcc6393f50a0" ], [ "EnumParsing.then_pure_check", @@ -571,7 +571,7 @@ "typing_FStar.UInt32.v" ], 0, - "4145cd0aea82061e586b8acd7686206c" + "5bb59c76d6a37169f78d8ddc2c499a3a" ], [ "EnumParsing.lemma_then_pure_check_ok", @@ -632,7 +632,7 @@ "typing_FStar.UInt32.v" ], 0, - "53d159bf83d2fe14e700be07b8abd849" + "afde63e68bf49cf63547f593ac9606b3" ], [ "EnumParsing.validate_numbers_pure", @@ -660,7 +660,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "2982db07b3b029ba52f4e77a6b684639" + "f078bd25a59af0b6fc5c969c4ca11dd3" ], [ "EnumParsing.parse_numbers_tag_st", @@ -742,7 +742,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "592ab18a49f5a7df967883bf0fa3172f" + "ab02ee4fb08655c1011723c7a164d9cf" ], [ "EnumParsing.parse_numbers_tag_st_nochk", @@ -845,7 +845,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "66f311b68412a83b9e09344edffb77ae" + "a1715eea2d1a98cda4f77e5da474b39d" ], [ "EnumParsing.parse_numbers_tag_st_nochk", @@ -879,7 +879,7 @@ "typing_Slice.as_seq" ], 0, - "6363df882247b46787803f68110d7bfb" + "2eadbb5a567d10cb375fcbdee94ee9cb" ], [ "EnumParsing.check_length", @@ -892,7 +892,7 @@ "proj_equation_Slice.BSlice_len", "projection_inverse_BoxBool_proj_0" ], 0, - "3069bd531de688be7217c0773d1f02bd" + "9766d665ea249e38875423c86e565119" ], [ "EnumParsing.validate_Nothing", @@ -992,7 +992,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "2c3cd5065db50ba638429a8a53f8403a" + "4fba3e6490897b8deaf7df064988d40d" ], [ "EnumParsing.validate_OneNum", @@ -1091,7 +1091,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "84edc5fbdaaf4407bb4b467fb6a8f624" + "2b45f869beb0ffa56f4b173b2f21ba65" ], [ "EnumParsing.validate_TwoNums", @@ -1188,7 +1188,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "336a7bd3d8e13703198f4a578fd82a1a" + "51b9f6d9561addfbb57e060e75a487b3" ], [ "EnumParsing.validate_numbers_data", @@ -1200,7 +1200,7 @@ "equation_Parsing.parser" ], 0, - "02663c03430e8c0c5d4ba81abe4795ed" + "a7bd89e2719bf3774404fd3525946863" ], [ "EnumParsing.coerce_validator", @@ -1262,7 +1262,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "242fe657b314961224d65e9f89d27523" + "3dd18bc4f3e787ecb470289f94fb91d1" ], [ "EnumParsing.and_check", @@ -1406,7 +1406,7 @@ "typing_Slice.as_seq" ], 0, - "531b544a20b496b4c2d1d2390f662c92" + "7e585c14232f946a6908d7b3d966b789" ], [ "EnumParsing.encode_numbers_tag", @@ -1427,7 +1427,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "15b27e8425f9780facedd1d44b174bb8" + "83bbd06c66239c64014a380032c516dd" ], [ "EnumParsing.encode_Nothing", @@ -1436,7 +1436,7 @@ 1, [ "@query" ], 0, - "7e46a4b85eae25cba18cbe5553534e3f" + "8b150b8ba16f31902a666b6bc2d69b49" ], [ "EnumParsing.encode_OneNum", @@ -1445,7 +1445,7 @@ 1, [ "@query", "equation_FStar.UInt8.byte", "equation_Slice.byte" ], 0, - "8b4e8f7482a15cb10451861f3474f0f7" + "86faaf8915fe9846ee936ca0e57cb882" ], [ "EnumParsing.encode_TwoNums", @@ -1463,7 +1463,7 @@ "typing_IntegerParsing.encode_u32" ], 0, - "c9ae0780a92f80c09b2bbff3ed046bb5" + "ed30f9682cb997f33571571e2fe1de62" ], [ "EnumParsing.encode_numbers_data", @@ -1478,7 +1478,7 @@ "fuel_guarded_inversion_EnumParsing.numbers" ], 0, - "ea1b8795f13286840565a8f3d5933582" + "99a27a451053f93ae5181687e9ddc42f" ], [ "EnumParsing.ser_Nothing", @@ -1582,7 +1582,7 @@ "typing_Slice.bslice_split_at" ], 0, - "88240c9fe15f3078522cdd561137fcfb" + "cbf2223d22c14c178de7c980416e40cc" ], [ "EnumParsing.ser_TwoNums", @@ -1615,7 +1615,7 @@ "typing_IntegerParsing.encode_u32" ], 0, - "ad9f82853180a8c6d676d53f456fcda8" + "a63b9d8fddaf0e8b3aa6680a6bf429b4" ], [ "EnumParsing.ser_TwoNums'", @@ -1634,7 +1634,7 @@ "typing_FStar.TSet.empty", "typing_FStar.TSet.set" ], 0, - "5f5dcbae23f01da98550dc0229364853" + "2ea9729d3db4c09707fdfc4095c64433" ], [ "EnumParsing.ser_numbers_data", @@ -1658,7 +1658,7 @@ "projection_inverse_EnumParsing.TwoNums_n" ], 0, - "fcda8870b7373a0b9547a381fcbf2035" + "fba9d3d86d3c00ee2befb75216674152" ], [ "EnumParsing.ser_numbers_data'", @@ -1681,7 +1681,7 @@ "typing_FStar.TSet.empty", "typing_FStar.TSet.set" ], 0, - "ed2f76414ce53e4e866068c97c3eb771" + "8f35ac4f1055f29e864768cb228da558" ], [ "EnumParsing.ser_numbers_data2", @@ -1704,7 +1704,7 @@ "typing_FStar.TSet.empty", "typing_FStar.TSet.set" ], 0, - "bffe8843e81cd2fcb3e64712b08d09ac" + "1e7ac3d747a685e05715cadeb24e0612" ], [ "EnumParsing.ser_numbers", @@ -1740,7 +1740,7 @@ "typing_FStar.TSet.set" ], 0, - "a4ea99f7bd2c1eaf019af12ec9d62b72" + "62fc62a8ee39859d1889327101449502" ], [ "EnumParsing.numbers", @@ -1749,7 +1749,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq" ], 0, - "2aef93d3aaff67364f1b70359bf1509f" + "c38f89ee823ff4f3816f301387efca9c" ], [ "EnumParsing.__proj__OneNum__item__n", @@ -1762,7 +1762,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_4f83c2c575e4b9df7e99e95590ac6726" ], 0, - "190da10d027fc1704ea29b67fe8ee95c" + "0d5effa560ab2b5d1b7d08feaf0c88e3" ], [ "EnumParsing.__proj__TwoNums__item__n", @@ -1776,7 +1776,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_f7b177f0e5c9dfa961ddcd32747ed85b" ], 0, - "854ce7aebc4102115378c449a820e186" + "82e1cc1a7e86f36ab4bd78ac95b7ad12" ], [ "EnumParsing.__proj__TwoNums__item__m", @@ -1790,7 +1790,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_f7b177f0e5c9dfa961ddcd32747ed85b" ], 0, - "739ba624e93fa027c59fd9518f010248" + "16df47c90eb8cd102c4223c1a2581724" ], [ "EnumParsing.numbers_tag_val", @@ -1805,7 +1805,7 @@ "fuel_guarded_inversion_EnumParsing.numbers" ], 0, - "11a0e06abb1ac5727ae87f31263cda0e" + "8c6a8e9d68cf6a92a60958800f9e7054" ], [ "EnumParsing.parse_numbers_tag", @@ -1834,7 +1834,7 @@ "typing_FStar.UInt32.v", "typing_FStar.UInt8.v" ], 0, - "02938fc4afe42d217746e8004f0c8bff" + "93c50a9f8ed1bd3fd444b15925c42759" ], [ "EnumParsing.parse_Nothing", @@ -1848,7 +1848,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "caea04f0ca4c64238afa3d5f894c2790" + "45f442cdfa9d76d9c5397a7d82919159" ], [ "EnumParsing.parse_OneNum", @@ -1862,7 +1862,7 @@ "projection_inverse_EnumParsing.OneNum_n" ], 0, - "b42ce4a7c004a6065686c6af58a3d46f" + "2d631af3ef70b5d8ae045b67d5877439" ], [ "EnumParsing.parse_TwoNums", @@ -1877,7 +1877,7 @@ "projection_inverse_EnumParsing.TwoNums_n" ], 0, - "379e72d463e8e6e2a37a40818f1e0f29" + "52176a5f21197d5b180de123bb10e190" ], [ "EnumParsing.parser_forget", @@ -1898,7 +1898,7 @@ "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b" ], 0, - "50ee7d6d3c5779f8f7b86afb4fa49b8e" + "03f2b22a82968b1f6674020f21523f41" ], [ "EnumParsing.validate_ok", @@ -1917,7 +1917,7 @@ "refinement_interpretation_Parsing_Tm_refine_2c4ed52ca61af0afe406eb07485d9cb6" ], 0, - "01377d934cdd66af7b2f51b377b1bff3" + "5aed99e65edd78419956a6be968b5153" ], [ "EnumParsing.make_correct", @@ -1931,7 +1931,7 @@ "refinement_interpretation_EnumParsing_Tm_refine_e0227620956763aa0703230757ef418a" ], 0, - "7a39dda46c03e5f5f109c064357d175d" + "9d90490d3c06a4b7503942d82f5afb7e" ], [ "EnumParsing.validate_Nothing_pure", @@ -1967,7 +1967,7 @@ "typing_FStar.Seq.Base.length", "typing_tok_EnumParsing.Nothing@tok" ], 0, - "3cf57c220d3bd922c2f169f923d17ef7" + "5204d5edc2134ed837b5194f7353e063" ], [ "EnumParsing.validate_OneNum_pure", @@ -2028,7 +2028,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "34abc80ea97c7700bb2abdca4c6ba38e" + "a0b5600fc49b8eb9e432f3419dc4f377" ], [ "EnumParsing.validate_TwoNums_pure", @@ -2110,7 +2110,7 @@ "typing_FStar.UInt32.v", "typing_tok_EnumParsing.Nothing@tok" ], 0, - "76a7d49862cfb2360307f2f48b43f965" + "0851a9f8eaf2e2c62620c608b8f3fd7e" ], [ "EnumParsing.validate_numbers_data_pure", @@ -2139,7 +2139,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "997be7e4dc3d7e17cf91a9a94990e39a" + "3745c1eab62fc2b278d2eb0da5b9f2ea" ], [ "EnumParsing.seq_pure_validate", @@ -2182,7 +2182,7 @@ "typing_FStar.UInt32.v" ], 0, - "31d1759833494b4ec085165315545c50" + "19207faf75b37b52cb6d9b23c82cead8" ], [ "EnumParsing.then_pure_check", @@ -2221,7 +2221,7 @@ "typing_FStar.UInt32.v" ], 0, - "a428087c338a9d4330a7c646d95e55ac" + "d4dedd5eef4c0e7c0fb66851721c8c83" ], [ "EnumParsing.validate_numbers_pure", @@ -2249,7 +2249,7 @@ "typing_tok_EnumParsing.Nothing@tok" ], 0, - "39fd7cd0933085454b980bf66dcafc1e" + "f8fe06e3260422e684938313c50c468a" ], [ "EnumParsing.parse_numbers_tag_st", @@ -2279,7 +2279,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "fb7a1c592312aa70943213c36a6ee7b6" + "a3a98e560e9f3e7b1f5013ac732a4da0" ], [ "EnumParsing.parse_numbers_tag_st_nochk", @@ -2313,7 +2313,7 @@ "typing_Slice.as_seq" ], 0, - "cd33e736afd894354c1347a09fc9de78" + "c8179b88800fced208951e9ec21d45b7" ], [ "EnumParsing.check_length", @@ -2340,7 +2340,7 @@ "typing_FStar.UInt32.v" ], 0, - "2519b4e9d2fcf9321091cc626e3ecafc" + "a404296b2324646020169591a1b5c943" ], [ "EnumParsing.validate_Nothing", @@ -2366,7 +2366,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "cf5e4d410ca64c7350836b72eea49fe8" + "5f813ded8e7fd310b378175db9323df3" ], [ "EnumParsing.validate_OneNum", @@ -2392,7 +2392,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "dc1176cb6f9ca90addab3d4a6ba33c0f" + "f57cffd3e3adf71cd5725c714d765623" ], [ "EnumParsing.validate_TwoNums", @@ -2418,7 +2418,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "62f803f584c3a6d2e622fafb6f6abf4c" + "f74ca615e014ac1ce0d3f77ef5534f47" ], [ "EnumParsing.validate_numbers_data", @@ -2430,7 +2430,7 @@ "equation_Parsing.parser" ], 0, - "54ce6810cef9e219a946921b7ba083e5" + "923ec017efe870ab4a71ab0720340f99" ], [ "EnumParsing.coerce_validator", @@ -2492,7 +2492,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "f6c9a6d6de7fe17e3d5644d62558ecab" + "b41c8437dcd871e8f2a4582fbfdb0443" ], [ "EnumParsing.and_check", @@ -2635,7 +2635,7 @@ "typing_Slice.as_seq" ], 0, - "a5c927de9aecc5b69e341afca04ca6b4" + "d480b5e616d91533b6220188e50ad438" ], [ "EnumParsing.validate_numbers", @@ -2644,7 +2644,7 @@ 1, [ "@query", "equation_EnumParsing.parse_numbers" ], 0, - "f3db5f80a8da9106a9b3fc8ba08fd63e" + "53de1695144eeefe5f68eac689a1d5b8" ], [ "EnumParsing.encode_numbers_tag", @@ -2665,7 +2665,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "dd15dbe7118a8f2b3fd60f9b88488fd0" + "e2bb7f4dee1c0f11dc8f60d9c228dff2" ], [ "EnumParsing.encode_Nothing", @@ -2674,7 +2674,7 @@ 1, [ "@query" ], 0, - "031201e244dc143737afa8f18b21f5b2" + "0b56e8f5c77837ef2f3805cd0a912870" ], [ "EnumParsing.encode_OneNum", @@ -2683,7 +2683,7 @@ 1, [ "@query", "equation_FStar.UInt8.byte", "equation_Slice.byte" ], 0, - "49248491fa057ef2d57b15dacad633b9" + "a05e19871c09af439c8a4fac14fe6211" ], [ "EnumParsing.encode_TwoNums", @@ -2701,7 +2701,7 @@ "typing_IntegerParsing.encode_u32" ], 0, - "00bf3564e911c319a2c36616c50c1728" + "6d97d5a41eb34f11b9d1cf1f0f395e79" ], [ "EnumParsing.encode_numbers_data", @@ -2716,7 +2716,7 @@ "fuel_guarded_inversion_EnumParsing.numbers" ], 0, - "7680962a6dcabfa3330b429fc735d7a1" + "461d20ded9aff510f70f9b37501d48da" ], [ "EnumParsing.ser_Nothing", @@ -2725,7 +2725,7 @@ 1, [ "@query" ], 0, - "b56c13cb37a5b53f88bb92a69b56768d" + "83fe699b4160ed20496b084ff5da9ec1" ], [ "EnumParsing.ser_TwoNums", @@ -2758,7 +2758,7 @@ "typing_IntegerParsing.encode_u32" ], 0, - "c24cdd4352bc466a126b5752d313724a" + "70aa485c2260522dbf3747d028303a47" ], [ "EnumParsing.ser_TwoNums'", @@ -2777,7 +2777,7 @@ "typing_FStar.TSet.empty", "typing_FStar.TSet.set" ], 0, - "a0d29d70fe071b8c481c189b75f0462d" + "f1d4717ad35e1feba9e3c8666e762a66" ], [ "EnumParsing.ser_numbers_data", @@ -2811,7 +2811,7 @@ "typing_FStar.UInt32.v" ], 0, - "d08f410fd4dca2861e8d905c440ea57d" + "6bdff55436d6da61fd64f4ebf3adb426" ], [ "EnumParsing.ser_numbers_data'", @@ -2834,7 +2834,7 @@ "typing_FStar.TSet.empty", "typing_FStar.TSet.set" ], 0, - "eba4c2891061ce8f916282b74228b6a8" + "b38c4d3f1acda0b115aadb0c37ebd875" ], [ "EnumParsing.ser_numbers_data2", @@ -2857,7 +2857,7 @@ "typing_FStar.TSet.empty", "typing_FStar.TSet.set" ], 0, - "b16751631cf4ea5c4113bfa4b2f5c53d" + "91f8ed98bbd496b460dc119d2c2ff1a5" ], [ "EnumParsing.ser_numbers", @@ -2893,7 +2893,7 @@ "typing_FStar.TSet.set" ], 0, - "9ad4a355e0c496a148c46b921d3804b2" + "a7eb1b4452e13cb2ce37631a4506d70d" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/IntegerParsing.fst.hints b/examples/kv_parsing/IntegerParsing.fst.hints index 58dc7f7dd36..ec05983307b 100644 --- a/examples/kv_parsing/IntegerParsing.fst.hints +++ b/examples/kv_parsing/IntegerParsing.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "8a6b0d5a3bd6dc6cafb2754fbe4df9d1" + "efff3c9ab54a6eeb2045ab8e4ec4b299" ], [ "IntegerParsing.u16_array", @@ -17,7 +17,7 @@ 1, [ "@query" ], 0, - "149dff71b34564119181ebed81604736" + "bf510a6325428ac0db5bd54b4c067365" ], [ "IntegerParsing.u16_array", @@ -33,7 +33,7 @@ "haseqIntegerParsing_Tm_refine_67a0f7da090ddd7cabafb21bf5e2ed60" ], 0, - "086c5eb9771034ba85e5f9a5606b38c1" + "be050a361c6a8e7ff6b2c925bc655cc7" ], [ "IntegerParsing.u16_array", @@ -51,7 +51,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "1798427809eb81e7a2338f717f97318d" + "b00c339a2cdda20d8dd05fefcc44b2a6" ], [ "IntegerParsing.__proj__U16Array__item__a16", @@ -60,7 +60,7 @@ 1, [ "@query" ], 0, - "9c774f42572b294deeb0bc1f1228863a" + "b4b447427d450fdd8ccef637e1ac22af" ], [ "IntegerParsing.__proj__U16Array__item__a16", @@ -72,7 +72,7 @@ "projection_inverse_IntegerParsing.U16Array_len16" ], 0, - "e02345a3d62a228fde1f90dcd4b54f44" + "c4687d23df00a8f43527b91e705e0e1b" ], [ "IntegerParsing.u32_array", @@ -81,7 +81,7 @@ 1, [ "@query" ], 0, - "f80d0efe3cc15b8c462bab436ad1d399" + "aea33ae26f6709609c6e5844cb4157c9" ], [ "IntegerParsing.u32_array", @@ -90,7 +90,7 @@ 1, [ "@query" ], 0, - "42b5faf3427dfddf846b542f9a824ff1" + "80754d3c6d8776d6a9129e6ec671b69a" ], [ "IntegerParsing.u32_array", @@ -106,7 +106,7 @@ "haseqIntegerParsing_Tm_refine_81c227cb3788ac9527a15eab9f2e5b39" ], 0, - "76bda6dc099effe06b919ff37e1d031c" + "f31e45cd6df0dc195576107cf3fd52f0" ], [ "IntegerParsing.u32_array", @@ -124,7 +124,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "75103766bddd91fc5b009dd886151d51" + "98e0d1632e9676981bbfb674cb447fd4" ], [ "IntegerParsing.__proj__U32Array__item__a32", @@ -133,7 +133,7 @@ 1, [ "@query" ], 0, - "2ea4ef77064d01284104e717abd88124" + "647cf4f79d03f08bff38a175750d2c06" ], [ "IntegerParsing.__proj__U32Array__item__a32", @@ -145,7 +145,7 @@ "projection_inverse_IntegerParsing.U32Array_len32" ], 0, - "b4072f8da67d23c4e419a13689a4d6c2" + "2d8cd3d8b5aa298db78dd668619c8f3c" ], [ "IntegerParsing.parse_u8", @@ -157,7 +157,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "5dafbd0e411a7edf4db32ea4129e14d2" + "05934be4da19ae94559f2d6143b2edb9" ], [ "IntegerParsing.parse_u16", @@ -188,7 +188,7 @@ "typing_FStar.Kremlin.Endianness.be_to_n" ], 0, - "780769f8499f1abddad21c7994f44f85" + "15ce38bee34ef17c605903a3e9fcdb7a" ], [ "IntegerParsing.parse_u32", @@ -221,7 +221,7 @@ "typing_FStar.Kremlin.Endianness.be_to_n" ], 0, - "ca1c1ec25d15e88106719e4d17b678ee" + "1f4b9de63904c0af2b3039071cee0dc8" ], [ "IntegerParsing.parse_u16_array", @@ -252,7 +252,7 @@ "typing_FStar.Seq.Base.length", "typing_FStar.UInt16.v" ], 0, - "4e831f5a45a85d1f6fd379ba0ab230b1" + "6430b8b5705a8f752c9a5abc18cdc12f" ], [ "IntegerParsing.parse_u32_array", @@ -284,7 +284,7 @@ "typing_FStar.UInt32.v" ], 0, - "c3e27175b00a51ab634f3569a9b36175" + "1703aaf5898be5a7c14f7ef3a967127d" ], [ "IntegerParsing.u16_array_st", @@ -293,7 +293,7 @@ 1, [ "@query" ], 0, - "451c7f9e7a3af6d0eec2841acf94a850" + "eab5d17d3e98907e896043ef6ab847b8" ], [ "IntegerParsing.__proj__U16ArraySt__item__a16_st", @@ -302,7 +302,7 @@ 1, [ "@query" ], 0, - "9eac52a621a069eb388ac44c6b232eac" + "13c3d24699adf8c2fd6f6b32e2427471" ], [ "IntegerParsing.__proj__U16ArraySt__item__a16_st", @@ -314,7 +314,7 @@ "projection_inverse_IntegerParsing.U16ArraySt_len16_st" ], 0, - "07630b7ae06794dea8fecff761e27b12" + "84406499d3501b566176d90d3168ea75" ], [ "IntegerParsing.__proj__U32ArraySt__item__a32_st", @@ -326,7 +326,7 @@ "projection_inverse_IntegerParsing.U32ArraySt_len32_st" ], 0, - "6d85b544f96828bfee4fc7e6fe8bf5d8" + "800767d22b274007de491327ea1c239c" ], [ "IntegerParsing.as_u16_array", @@ -342,7 +342,7 @@ "typing_IntegerParsing.__proj__U16ArraySt__item__a16_st" ], 0, - "4df7574fcba9267c88fbd74a60706aed" + "35b238dd6932862242abe0150e88ccdb" ], [ "IntegerParsing.as_u32_array", @@ -358,7 +358,7 @@ "typing_IntegerParsing.__proj__U32ArraySt__item__a32_st" ], 0, - "385fd755af5a897b95a981996bd34d03" + "38d2bccebae2f859af6608e634443986" ], [ "IntegerParsing.parse_u8_st_nochk", @@ -426,7 +426,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "c6ad93b38703329120d32cbfd9c496a8" + "c582fb3be1f2a4b17211832525523826" ], [ "IntegerParsing.parse_u8_st_nochk", @@ -458,7 +458,7 @@ "typing_Slice.as_seq" ], 0, - "96c4f1ae58b44f3cc5304e2a2e254601" + "c9e7522fdcf7d7cd768a6e1eda6e6d2d" ], [ "IntegerParsing.parse_u8_st", @@ -582,7 +582,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "78e6a1b2c9f539546a05d37d1ae9ad45" + "480a9bc6baa6920552cbf15c05567aa8" ], [ "IntegerParsing.parse_u8_st", @@ -611,7 +611,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "5dcb2ede54232b7fa02610911124a722" + "55d856272c6b065c9a62df3947c2c423" ], [ "IntegerParsing.parse_u16_st_nochk", @@ -700,7 +700,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "e4b07a9c472a2ecd9c043af71e29cb98" + "38099cc8d570bc7583a581bc61f3781a" ], [ "IntegerParsing.parse_u16_st_nochk", @@ -732,7 +732,7 @@ "typing_Slice.as_seq" ], 0, - "0f0cf92a7fb508d955374d2e6598faf1" + "eaa157fc4013c5eb418318dd5b0e237a" ], [ "IntegerParsing.parse_u16_st", @@ -856,7 +856,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "45b2bdb58f00622c5a32fca6b001be53" + "85f7d059c647a0a136d22b085fcbf2d3" ], [ "IntegerParsing.parse_u16_st", @@ -885,7 +885,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "df5c069ead750a6e937de4f4fb70ca9d" + "b6ac875a1457994d0cd06a5c4ab5f2f7" ], [ "IntegerParsing.parse_u32_st_nochk", @@ -974,7 +974,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "28d540ac74db33cb54ef56afebce9b0e" + "03b9a40618be76c1275d00a6d56e7061" ], [ "IntegerParsing.parse_u32_st_nochk", @@ -1007,7 +1007,7 @@ "typing_Slice.as_seq" ], 0, - "f7fd8075bca8dd3a3a480189edaa90c9" + "ec2f7622caf37e643a247d9ce01ce042" ], [ "IntegerParsing.parse_u32_st", @@ -1128,7 +1128,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "e4328650fa7402e1c20af2bc01bf10ec" + "51aada9e2114fc3d542dc348e0ff06c2" ], [ "IntegerParsing.parse_u32_st", @@ -1158,7 +1158,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "b40293ec11672b29763eafc9ca95c293" + "b8d67498f3025e8b76cf3819bdbe25e3" ], [ "IntegerParsing.parse_u16_array_nochk", @@ -1295,7 +1295,7 @@ "typing_Slice.as_seq" ], 0, - "e16620e9794b2473da0198f03ad5847d" + "c2352d0679fcb3dd7f2cc36021fd3f21" ], [ "IntegerParsing.parse_u16_array_nochk", @@ -1328,7 +1328,7 @@ "typing_Slice.as_seq" ], 0, - "0f72d347f6c58ff20b18765d2b5210a3" + "9b04d69c5c54ed5d73a8229df9e4c952" ], [ "IntegerParsing.parse_u32_array_nochk", @@ -1462,7 +1462,7 @@ "typing_Slice.as_seq" ], 0, - "bc23566459f7e1343cc103fedfd86bd3" + "fb253e722d0767bdda8fefea869555ae" ], [ "IntegerParsing.parse_u32_array_nochk", @@ -1495,7 +1495,7 @@ "typing_Slice.as_seq" ], 0, - "73bec71954bcb1667fd9035c8ce5ca2a" + "edaae78d0c7c918054bda8d9f792a49b" ], [ "IntegerParsing.validate_u16_array_st", @@ -1636,7 +1636,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "081191a83f43190dca9a0f57915559ca" + "18d58ca51029f75aba836352def55410" ], [ "IntegerParsing.validate_u16_array_st", @@ -1662,7 +1662,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "910a87898ec063ff037f05c56964bef3" + "be0c5a6449c1867745005a401e9b0a8e" ], [ "IntegerParsing.u32_array_bound_is", @@ -1693,7 +1693,7 @@ "typing_FStar.UInt32.v" ], 0, - "a16c64f6b3410b668fe958cad8c59fdf" + "bdc138c0b0d2ee51b83772c855cc73a9" ], [ "IntegerParsing.validate_u32_array_st", @@ -1799,7 +1799,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "eb8e2e813e320faeb3ce01a300c213f5" + "4d11d441df0c7b4fde50c136e69e3063" ], [ "IntegerParsing.validate_u32_array_st", @@ -1825,7 +1825,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "ec67f816550d76bc8c3af6e752a4f4d8" + "52e7ea2c6e0493007415f233b7d4b62a" ], [ "IntegerParsing.encode_u8", @@ -1844,7 +1844,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "d0474dffb9a22d2327b67b4df36f527e" + "11db14d8ae7c20e74ba566519158f5e0" ], [ "IntegerParsing.encode_u16", @@ -1861,7 +1861,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "8ed961a6998d5be69726853233aac579" + "ffc097a0dc7b6705a0ecc06103a7fe8f" ], [ "IntegerParsing.encode_u32", @@ -1883,7 +1883,7 @@ "typing_FStar.UInt32.v" ], 0, - "ac680525f493ad49f2f68392fc350194" + "4c43fa8f2897b6710a67ac1f5c3f69f2" ], [ "IntegerParsing.encode_u16_array", @@ -1892,7 +1892,7 @@ 1, [ "@query" ], 0, - "a9890c8d8f39c0ade93678f6c48992a2" + "319e73fa938b67aabacea983fbbcd4d2" ], [ "IntegerParsing.encode_u32_array", @@ -1901,7 +1901,7 @@ 1, [ "@query" ], 0, - "0c53aac593839f9c4deb0abab36e7122" + "50152834f1a3f3a3891eca3aa08cd9b5" ], [ "IntegerParsing.upd_len_1", @@ -1913,7 +1913,7 @@ "refinement_interpretation_IntegerParsing_Tm_refine_0e8e6d303853d84bc6b6f6552f57fff5" ], 0, - "8d6ddaf0f585f7a09760acf00a72c592" + "c5dee8b3579d392c91aa503321148e18" ], [ "IntegerParsing.upd_len_1", @@ -1940,7 +1940,7 @@ "typing_FStar.Seq.Base.create", "typing_FStar.Seq.Base.length" ], 0, - "75dab9d949d6e22fa24e5df8e41e5835" + "f42e4f04132fb8ec9d66b4bbda7b8ad3" ], [ "IntegerParsing.ser_byte", @@ -2037,7 +2037,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "99fc092778e64959a50d7fca11098a4d" + "04a952104ff3c6a9afcd71a5999fec3a" ], [ "IntegerParsing.n_to_be_inv", @@ -2058,7 +2058,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "776e7348ca6fe51c3010ab53c2bfdb8a" + "084aa2bb32397bec66e1e1ba200f2d98" ], [ "IntegerParsing.store_be_inv", @@ -2076,7 +2076,7 @@ "typing_FStar.UInt32.v" ], 0, - "943ea968df53a1c6d02dd9b51b794307" + "75b21ec9eb4b9679610b1f0636fd1b26" ], [ "IntegerParsing.store_be_inv", @@ -2094,7 +2094,7 @@ "typing_FStar.UInt32.v" ], 0, - "29f98504435cd99e46d5e0ed1fa482d5" + "a1173f95ebf10686711bf0938038915f" ], [ "IntegerParsing.store_be_inv", @@ -2112,7 +2112,7 @@ "typing_FStar.UInt32.v" ], 0, - "5215df3bf3b3635b2046e327714ec3a0" + "dfea1e2fbc35d9d4f1d631645eb6c21a" ], [ "IntegerParsing.ser_u16", @@ -2203,7 +2203,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "bac8cc7d5c70dc01cb1183987c34266c" + "77d4fb9e6873ee2b0a75a0d48c84af80" ], [ "IntegerParsing.ser_u32", @@ -2293,7 +2293,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "158d10a13bf1e8ba6e2494a147e8874f" + "223a1453ce93034acc5a4077577ace2a" ], [ "IntegerParsing.enc_u16_array_st", @@ -2306,7 +2306,7 @@ "refinement_interpretation_IntegerParsing_Tm_refine_9834a243ad38517d628f708ee085bc54" ], 0, - "9c910c55a12ea34c84e141a7515fb3cd" + "8a33c5bd074f1800fe7558541fe5cb10" ], [ "IntegerParsing.ser_u16_array", @@ -2328,7 +2328,7 @@ "typing_IntegerParsing.__proj__U16ArraySt__item__a16_st" ], 0, - "4e75abd5f3196985b69e4c262286d9b1" + "f196639c86fada09ac89feae3e397c72" ], [ "IntegerParsing.ser_u16_array", @@ -2368,7 +2368,7 @@ "typing_IntegerParsing.encode_u16" ], 0, - "2fa5fe021db2439ab83680046b77b87e" + "baa8758aa21a6e8f4e17596daab89a06" ], [ "IntegerParsing.enc_u32_array_st", @@ -2381,7 +2381,7 @@ "refinement_interpretation_IntegerParsing_Tm_refine_01b2fceba02f49722cb73362c77b09cb" ], 0, - "30c6c05b1837444e8239dc6e6005e806" + "e5ba16c77a3fd16b31b6d0d3d6639f57" ], [ "IntegerParsing.ser_u32_array", @@ -2403,7 +2403,7 @@ "typing_IntegerParsing.__proj__U32ArraySt__item__a32_st" ], 0, - "bc27885ecbf25942e34b9eacecb5a796" + "02b4cb4f051feb23aae06abe380d951c" ], [ "IntegerParsing.ser_u32_array", @@ -2443,7 +2443,7 @@ "typing_IntegerParsing.encode_u32" ], 0, - "4cc9d935be82e1d53e9c1f9e5aa310fa" + "791b311e6ed2fa935dd4ee13727f52c9" ], [ "IntegerParsing.u16_array", @@ -2452,7 +2452,7 @@ 1, [ "@query" ], 0, - "3078eccad4693c4ce495e3f23592e40a" + "06888808126b054a6c09e3ff67602558" ], [ "IntegerParsing.u16_array", @@ -2461,7 +2461,7 @@ 1, [ "@query" ], 0, - "f073b2cb00358fe42dc14989339249d9" + "d3b11ec07fc2da8a35fecbedad4a093e" ], [ "IntegerParsing.u16_array", @@ -2477,7 +2477,7 @@ "haseqIntegerParsing_Tm_refine_67a0f7da090ddd7cabafb21bf5e2ed60" ], 0, - "9adb61ad53bfd9a444463fb195064bae" + "6ce6622708dc71555d44e7df9fa3d776" ], [ "IntegerParsing.u16_array", @@ -2495,7 +2495,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "3b4a501cf20df6f4480185c311c17d50" + "32c825e3da70ee2bf4cfa79b79ab3d2b" ], [ "IntegerParsing.__proj__U16Array__item__a16", @@ -2504,7 +2504,7 @@ 1, [ "@query" ], 0, - "e08f5add53a4611388997fc88f3cd101" + "aaeb7bd75f0e765b53d4041f423c0e1b" ], [ "IntegerParsing.__proj__U16Array__item__a16", @@ -2516,7 +2516,7 @@ "projection_inverse_IntegerParsing.U16Array_len16" ], 0, - "8ba4e20489446265b35ca9d81aacefa2" + "a60a5456fe02c0c07468830f11ff052a" ], [ "IntegerParsing.u32_array", @@ -2525,7 +2525,7 @@ 1, [ "@query" ], 0, - "26e4033b7802cbc801aa85650d577e06" + "a968f1188fe9ffc8b6f28b4a4ad81875" ], [ "IntegerParsing.u32_array", @@ -2534,7 +2534,7 @@ 1, [ "@query" ], 0, - "97dd024f22fcf4d1b31c37634ae1004a" + "02843c638e0cd7301eba6f19de12ab6e" ], [ "IntegerParsing.u32_array", @@ -2550,7 +2550,7 @@ "haseqIntegerParsing_Tm_refine_81c227cb3788ac9527a15eab9f2e5b39" ], 0, - "c4cbe893aec9bd231d0aa6e3f4451483" + "9b17df02136c2a6b172df701f5bebf5f" ], [ "IntegerParsing.u32_array", @@ -2568,7 +2568,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "6ba1f36935213a75ad16b335482a7706" + "7ab41c73677ca4d28dcaccf786ac1cd2" ], [ "IntegerParsing.__proj__U32Array__item__a32", @@ -2577,7 +2577,7 @@ 1, [ "@query" ], 0, - "144c85106031c24f46fbc730cde5c56c" + "b5e07b69bae9d195f35c8313bd491fb3" ], [ "IntegerParsing.__proj__U32Array__item__a32", @@ -2589,7 +2589,7 @@ "projection_inverse_IntegerParsing.U32Array_len32" ], 0, - "2074f86816753cc1203c6116c6181ff9" + "b64f8aabdaf9b07802fdca35573473cd" ], [ "IntegerParsing.parse_u8", @@ -2601,7 +2601,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "5e97044068137d5d2f718353b2c809aa" + "b09c93c1953fb9d1af904da8bff25e0a" ], [ "IntegerParsing.parse_u16", @@ -2632,7 +2632,7 @@ "typing_FStar.Kremlin.Endianness.be_to_n" ], 0, - "6ad498826d7bcf2546142fa8723aed62" + "c0adf1d865f5348b90720be53f11c5b1" ], [ "IntegerParsing.parse_u32", @@ -2665,7 +2665,7 @@ "typing_FStar.Kremlin.Endianness.be_to_n" ], 0, - "87aa4564a2af3630d44f3b78d1787b36" + "013813275679f426972c1a0ea17595b6" ], [ "IntegerParsing.parse_u16_array", @@ -2696,7 +2696,7 @@ "typing_FStar.Seq.Base.length", "typing_FStar.UInt16.v" ], 0, - "273eb0dead229f7032bf5f6f443efb9a" + "c2f06ff006fbff5c6757ed7829949335" ], [ "IntegerParsing.parse_u32_array", @@ -2728,7 +2728,7 @@ "typing_FStar.UInt32.v" ], 0, - "26f5d6e3f005c695593778814a27f500" + "a03fec5a3ccc14d04314469f48d44541" ], [ "IntegerParsing.u16_array_st", @@ -2737,7 +2737,7 @@ 1, [ "@query" ], 0, - "3983aeed668f2c8e0f494bf95aab97d0" + "31eb702e131afe41d56d07942b2499be" ], [ "IntegerParsing.__proj__U16ArraySt__item__a16_st", @@ -2746,7 +2746,7 @@ 1, [ "@query" ], 0, - "69ff1d024ce58d25e9083506774b96ca" + "681a09dba4cbd50f65b8e23321ac2c22" ], [ "IntegerParsing.__proj__U16ArraySt__item__a16_st", @@ -2758,7 +2758,7 @@ "projection_inverse_IntegerParsing.U16ArraySt_len16_st" ], 0, - "f053bb6a183b0717ba98d84f326e9720" + "bb3825ee1e8b8d55167d67be0e4e4d71" ], [ "IntegerParsing.__proj__U32ArraySt__item__a32_st", @@ -2770,7 +2770,7 @@ "projection_inverse_IntegerParsing.U32ArraySt_len32_st" ], 0, - "b3a6e8f3b1566b062767514c27b821e2" + "039e607a171bc2bffa09bd10bc945c17" ], [ "IntegerParsing.as_u16_array", @@ -2787,7 +2787,7 @@ "typing_IntegerParsing.__proj__U16ArraySt__item__a16_st" ], 0, - "6ae9c5f5b9b6a7f16ca7e7c80b990863" + "6570e6026521df66d375b1f5595b45e7" ], [ "IntegerParsing.as_u32_array", @@ -2804,7 +2804,7 @@ "typing_IntegerParsing.__proj__U32ArraySt__item__a32_st" ], 0, - "6bfa05800129f1e326b6947c78614c98" + "80976cd96764d08d4d88eb946c1f7919" ], [ "IntegerParsing.parse_u8_st_nochk", @@ -2836,7 +2836,7 @@ "typing_Slice.as_seq" ], 0, - "ef67424ff85eef400757281488999083" + "6876b1888b1c59546090cf74f7539b97" ], [ "IntegerParsing.parse_u8_st", @@ -2865,7 +2865,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "9fce977cce89290d39af955e35b3f837" + "eabb99763dae281e03852926c9de5814" ], [ "IntegerParsing.parse_u16_st_nochk", @@ -2897,7 +2897,7 @@ "typing_Slice.as_seq" ], 0, - "11e35932a7de7a17f607a881d9e6b8ef" + "8bf9f0a55f6b5d85d9b57db9e807398f" ], [ "IntegerParsing.parse_u16_st", @@ -2926,7 +2926,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "94a25acf840df5020b41891a12ee8869" + "aac1bed529e1b5516291b01038fd0e8d" ], [ "IntegerParsing.parse_u32_st_nochk", @@ -2959,7 +2959,7 @@ "typing_Slice.as_seq" ], 0, - "59b838659c2308b11a50dce50134b3c5" + "73691dcefa0037cdd5ea43989637044e" ], [ "IntegerParsing.parse_u32_st", @@ -2989,7 +2989,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "ebfbfdb703d93fbd51e859a2bb1f6a50" + "bf1e89527a83d847a75958097b630a76" ], [ "IntegerParsing.parse_u16_array_nochk", @@ -3022,7 +3022,7 @@ "typing_Slice.as_seq" ], 0, - "938def2e6f5cd3703b969a70d10e71ae" + "881c6592678d9c5fe2c2d2787052452f" ], [ "IntegerParsing.parse_u32_array_nochk", @@ -3055,7 +3055,7 @@ "typing_Slice.as_seq" ], 0, - "05b096eacaf1e80b0b4b95af01c60025" + "ff1ce7f8599bbb7a2fe408e5edad5465" ], [ "IntegerParsing.validate_u16_array_st", @@ -3088,7 +3088,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "9d8eab25783cf9431994e52416d7d887" + "2095c5c2394d53fbd9d4f9c50b71e579" ], [ "IntegerParsing.u32_array_bound_is", @@ -3097,7 +3097,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "720f3f5c63cf14b6a2d536b63467dcfb" + "ceba21b779b6befd714b51207cca4475" ], [ "IntegerParsing.validate_u32_array_st", @@ -3130,7 +3130,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "e02fe1253b2baa7605b022df8f2b8bef" + "dd28571561fc1bf519c00a42cd8508a5" ], [ "IntegerParsing.encode_u8", @@ -3149,7 +3149,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "527ef1d09e58d81e02e8670f5ec477ac" + "bbd64b2382034096a494daaaf4580d68" ], [ "IntegerParsing.encode_u16", @@ -3166,7 +3166,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "3f37d9caedcf5c709676247b41eca4ee" + "7a243051be2bb0360e9d554c0c4f0c31" ], [ "IntegerParsing.encode_u32", @@ -3188,7 +3188,7 @@ "typing_FStar.UInt32.v" ], 0, - "0b81991cc6e6eeb2767e435c558b33db" + "43db93675aa04ed116cb8c0e2271425b" ], [ "IntegerParsing.encode_u16_array", @@ -3197,7 +3197,7 @@ 1, [ "@query" ], 0, - "96b10d3228a23ba7281c70c132490501" + "ff3e844c4623a14bab5912a9da9656c9" ], [ "IntegerParsing.encode_u16_array", @@ -3206,7 +3206,7 @@ 1, [ "@query" ], 0, - "dc1d6e115f313854cee67af36a3b10ba" + "762e12e8127a4527b8653cbc4a3cd5ab" ], [ "IntegerParsing.encode_u32_array", @@ -3215,7 +3215,7 @@ 1, [ "@query" ], 0, - "7daf25fc32518263c94869bbb606059d" + "558ff9f5d2d3015fd11745f763dab18d" ], [ "IntegerParsing.encode_u32_array", @@ -3224,7 +3224,7 @@ 1, [ "@query" ], 0, - "f19c3e8ec26f39ee28517ca89c1e3cfa" + "82bfd411187f9f70c8ce091ca0874d04" ], [ "IntegerParsing.upd_len_1", @@ -3236,7 +3236,7 @@ "refinement_interpretation_IntegerParsing_Tm_refine_0e8e6d303853d84bc6b6f6552f57fff5" ], 0, - "5849859947c0b2ec1dcf6f3145af8c3b" + "721d76e0afd0cf750af427d50a1637eb" ], [ "IntegerParsing.ser_byte", @@ -3333,7 +3333,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "aeaaf14b0ef50ba7aa06bec56c26485a" + "e21d26ad1a73b6d653f5102bf2fb3de8" ], [ "IntegerParsing.n_to_be_inv", @@ -3354,7 +3354,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "27a3ea4e27a72e6f48b3ee1c06958f96" + "46faa188ba36138263c5c3d9a97ce8a5" ], [ "IntegerParsing.store_be_inv", @@ -3372,7 +3372,7 @@ "typing_FStar.UInt32.v" ], 0, - "09e78a3fb91cabdc3191c54a6d7e3403" + "8552db233761b6a69d508eed79c54ae9" ], [ "IntegerParsing.ser_u16", @@ -3463,7 +3463,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "8adf20aa52319a353996bf1f93fcb1aa" + "e02c70b4adada530283df2f1baa34c39" ], [ "IntegerParsing.ser_u32", @@ -3553,7 +3553,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "f656b728a689624aa539b9752fad1246" + "13d25ae45698e84d3772a75cfd18a548" ], [ "IntegerParsing.enc_u16_array_st", @@ -3566,7 +3566,7 @@ "refinement_interpretation_IntegerParsing_Tm_refine_9834a243ad38517d628f708ee085bc54" ], 0, - "12894e07a6c59620ba2f0c9cfaaa1fed" + "c8dd650b461b80d540374f423554ea4a" ], [ "IntegerParsing.ser_u16_array", @@ -3606,7 +3606,7 @@ "typing_IntegerParsing.encode_u16" ], 0, - "c6ad84f806f54073a3ba391c3025ae2f" + "1578dc4d1ce55a965347b4e3433dd6c7" ], [ "IntegerParsing.ser_u16_array", @@ -3628,7 +3628,7 @@ "typing_IntegerParsing.__proj__U16ArraySt__item__a16_st" ], 0, - "94a6763490365375613226b1b9825f60" + "70055c43cf93e67d04796f412b96b6eb" ], [ "IntegerParsing.enc_u32_array_st", @@ -3641,7 +3641,7 @@ "refinement_interpretation_IntegerParsing_Tm_refine_01b2fceba02f49722cb73362c77b09cb" ], 0, - "a83ef657745c9d420b5cafc8fb629830" + "5e04dee6622dfffd218e09b31e3a345f" ], [ "IntegerParsing.ser_u32_array", @@ -3681,7 +3681,7 @@ "typing_IntegerParsing.encode_u32" ], 0, - "58affc1770486a6f4d2d5588045169b8" + "4dbba892b9cbced2132f1ae9c6b78a2a" ], [ "IntegerParsing.ser_u32_array", @@ -3703,7 +3703,7 @@ "typing_IntegerParsing.__proj__U32ArraySt__item__a32_st" ], 0, - "7d3ea97c7789bdc2d5a37d833a1d6e78" + "4139108454c8baebe3c6046de7037005" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/KeyValue.fst.hints b/examples/kv_parsing/KeyValue.fst.hints index a421e5933cf..04bb92f8da7 100644 --- a/examples/kv_parsing/KeyValue.fst.hints +++ b/examples/kv_parsing/KeyValue.fst.hints @@ -15,7 +15,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "149a3d95e1431f9460bcdf518cb59bab" + "40b5711aab0e8e9d1c270ad701ba87ba" ], [ "KeyValue.encoded_entry", @@ -24,7 +24,7 @@ 1, [ "@query" ], 0, - "c4ba0bb0f6e8a13123198f83cac16219" + "ec56493ac12ea41f01468c95cecd9ddd" ], [ "KeyValue.encoded_entry", @@ -33,7 +33,7 @@ 1, [ "@query" ], 0, - "2e5cc0015fccb942eb6051454f6bc782" + "43e9866ee6bc2cffe387a892cac8562d" ], [ "KeyValue.encoded_entry", @@ -42,7 +42,7 @@ 1, [ "@query" ], 0, - "ffc5d900ddc7ed5d2e28c3afbba21bb8" + "84716fb738d88c8e0afb84370d3eb40c" ], [ "KeyValue.encoded_entry", @@ -60,7 +60,7 @@ "haseqIntegerParsing_Tm_refine_81c227cb3788ac9527a15eab9f2e5b39" ], 0, - "93de0bfd78ecb47feb51bcb70573ca6a" + "f67e0fe2216a4f200420fcac167c1ca4" ], [ "KeyValue.encoded_entry", @@ -80,7 +80,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "c55adf1ba1d2ade82306e2dd5b75634f" + "7b9b5b1d89f27df5acab9a5db15480d8" ], [ "KeyValue.__proj__EncodedEntry__item__key", @@ -89,7 +89,7 @@ 1, [ "@query" ], 0, - "5b809dae9cc97df1fd8be7adfa403014" + "5a19424de3a898f9f51d21a0a8a81509" ], [ "KeyValue.__proj__EncodedEntry__item__key", @@ -101,7 +101,7 @@ "projection_inverse_KeyValue.EncodedEntry_key_len" ], 0, - "58d7de91d0bfda7c6161b9a8f38055ce" + "afe440e8d42865eb46288d6ee8a05740" ], [ "KeyValue.__proj__EncodedEntry__item__value", @@ -110,7 +110,7 @@ 1, [ "@query" ], 0, - "8906b2dfc2c0df410c3df8fd5cf8b66d" + "59386ac4357b375dfb66c980544adf0e" ], [ "KeyValue.__proj__EncodedEntry__item__value", @@ -122,7 +122,7 @@ "projection_inverse_KeyValue.EncodedEntry_val_len" ], 0, - "091cb3214d7ee334bf8103a4fcfa77f7" + "dc410a70d0108f79363fd19d81294adb" ], [ "KeyValue.store", @@ -131,7 +131,7 @@ 1, [ "@query" ], 0, - "8347ae15324ac2a701527ec1327aeb7d" + "86d00fc31adba4af227ef25eab911341" ], [ "KeyValue.store", @@ -140,7 +140,7 @@ 1, [ "@query" ], 0, - "ebdcb0915a481834f2dcd59fe5d346d9" + "b1ce046ff125da0770635f3743500206" ], [ "KeyValue.store", @@ -155,7 +155,7 @@ "kinding_KeyValue.encoded_entry@tok" ], 0, - "09bbd45cf121c3372656cafefa06cd56" + "b2683a2e86b1579b751b702241de0d1a" ], [ "KeyValue.store", @@ -170,7 +170,7 @@ "kinding_KeyValue.encoded_entry@tok" ], 0, - "3f860a97bb95c79666b7baddf4b969af" + "df7c50a596173f486131c3b6018de688" ], [ "KeyValue.__proj__Store__item__entries", @@ -179,7 +179,7 @@ 1, [ "@query" ], 0, - "f6b9c066985ee6497e684c95ae6b644e" + "42f6aba57fed8ccc3d9688f02c54af2b" ], [ "KeyValue.__proj__Store__item__entries", @@ -191,7 +191,7 @@ "projection_inverse_KeyValue.Store_num_entries" ], 0, - "1f5e4bc4ac51c5fabf2e46bb84d509ae" + "4ff4681c12c2624d76659979dd75bcd1" ], [ "KeyValue.as_entry", @@ -203,7 +203,7 @@ "equation_KeyValue.entry_live", "equation_Slice.byte" ], 0, - "82f2d618341997fe6ca265b3c6738474" + "1e83539c66a57bb12d2dba35f4732363" ], [ "KeyValue.entry", @@ -219,7 +219,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "ac0af25f55a7bbefc0840e7655cb45d2" + "20b6c4ff2e6c19743e0fbdfa2cdfa8e6" ], [ "KeyValue.encoded_entry", @@ -228,7 +228,7 @@ 1, [ "@query" ], 0, - "e1d1fef07885de27e946381d92e46145" + "d2453519b2112a0cb855add8c11f9f97" ], [ "KeyValue.encoded_entry", @@ -237,7 +237,7 @@ 1, [ "@query" ], 0, - "b66b73ad3ff5d983823284d47f062f9a" + "7b101f040f134424a83c11054afd1499" ], [ "KeyValue.encoded_entry", @@ -246,7 +246,7 @@ 1, [ "@query" ], 0, - "e2443bc477358a4447eb33fcdc3e9543" + "39782f01387961cb4a2fe61097f15836" ], [ "KeyValue.encoded_entry", @@ -264,7 +264,7 @@ "haseqIntegerParsing_Tm_refine_81c227cb3788ac9527a15eab9f2e5b39" ], 0, - "f25ff65e114f6ffec09c655e52f6ed70" + "123e4e9a6f92147a1253e81fad7509de" ], [ "KeyValue.encoded_entry", @@ -284,7 +284,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "ed5380b9ea81b4f7b72f1a40a84f5965" + "41eee407ce7690c68c8c89e620f89a9c" ], [ "KeyValue.__proj__EncodedEntry__item__key", @@ -293,7 +293,7 @@ 1, [ "@query" ], 0, - "4fa2e663255004f1473b011519abd03d" + "9a5caf1e9f1d1a53e0a72f0912092478" ], [ "KeyValue.__proj__EncodedEntry__item__key", @@ -305,7 +305,7 @@ "projection_inverse_KeyValue.EncodedEntry_key_len" ], 0, - "06fc47ce829ea11979e822d44c94668f" + "c095a5c8bbf5ff5c763a07228dfe4cc5" ], [ "KeyValue.__proj__EncodedEntry__item__value", @@ -314,7 +314,7 @@ 1, [ "@query" ], 0, - "4632fbf83275bb1520a4e60d3b5989f3" + "f2e43bab6d8da5284d0a411bd82bb91e" ], [ "KeyValue.__proj__EncodedEntry__item__value", @@ -326,7 +326,7 @@ "projection_inverse_KeyValue.EncodedEntry_val_len" ], 0, - "d55269879a8080a50d29eef7e6c94f4c" + "eeb71d328d50b04a330ad7459b82baf4" ], [ "KeyValue.store", @@ -335,7 +335,7 @@ 1, [ "@query" ], 0, - "3da8b14b51d4a5caa200a6221895d02e" + "91500d6d617757ea32c69c240eeb803c" ], [ "KeyValue.store", @@ -344,7 +344,7 @@ 1, [ "@query" ], 0, - "24d85caf62389bc8e7905e430c073568" + "cb1c14ebd880ac7856e71bcc7dc33135" ], [ "KeyValue.store", @@ -359,7 +359,7 @@ "kinding_KeyValue.encoded_entry@tok" ], 0, - "c9d6727dbb9e09f084079ca5871d3513" + "5be589eeead964c45a4d342e6e5ca530" ], [ "KeyValue.store", @@ -374,7 +374,7 @@ "kinding_KeyValue.encoded_entry@tok" ], 0, - "c18ecdaed854ce6f2cfdff631080c817" + "fd64dc3eec64377fde82aa7d5f824f02" ], [ "KeyValue.__proj__Store__item__entries", @@ -383,7 +383,7 @@ 1, [ "@query" ], 0, - "ece20b11d999ae6c05157c65f1d81800" + "a642a1c09316de9bbcd14a4eb8ccf394" ], [ "KeyValue.__proj__Store__item__entries", @@ -395,7 +395,7 @@ "projection_inverse_KeyValue.Store_num_entries" ], 0, - "b669e246810a69a9505b3cfe17da698a" + "416c6af64cc8715f899e47e6b520ee7b" ], [ "KeyValue.as_entry", @@ -409,7 +409,7 @@ "fuel_guarded_inversion_KeyValue.entry_st" ], 0, - "45bccd2bc92e88bf4cba1dc1d3e43987" + "7fa1467a395bf5b0833bc19d72dcd334" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/Parsing.fst.hints b/examples/kv_parsing/Parsing.fst.hints index 0ef24eee304..6c0d4a8ab1a 100644 --- a/examples/kv_parsing/Parsing.fst.hints +++ b/examples/kv_parsing/Parsing.fst.hints @@ -34,7 +34,7 @@ "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b" ], 0, - "c6ba29856118b8d992fea41f7b918263" + "ce14ba3d89a5c732963d754ea28c23d2" ], [ "Parsing.parse_ret", @@ -55,7 +55,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "b1988d2a62d890615e146f1c9b399a0c" + "6c33992ae0d928e8d2e671df54061f82" ], [ "Parsing.parsing_done", @@ -67,7 +67,7 @@ "primitive_Prims.op_Equality", "projection_inverse_BoxBool_proj_0" ], 0, - "d118e04c2e3ca40cf0c6492b63be7fb2" + "6053045435bcded24d3b0cf52d087d70" ], [ "Parsing.parse_result", @@ -76,7 +76,7 @@ 1, [ "@query" ], 0, - "1d896713c9f4e5d49ae27b080111cf5b" + "a2bc59b004b96789de18494855eb7b69" ], [ "Parsing.parse_many", @@ -105,7 +105,7 @@ "typing_FStar.List.Tot.Base.length", "well-founded-ordering-on-nat" ], 0, - "6e0003504b9db6a9d85ae3e82e53a66b" + "c9b88bd3a7e08a4c94fb7994ee57927a" ], [ "Parsing.parser_st", @@ -134,7 +134,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "6f6a58d17573b0282fecf76e301dbbbb" + "9c64921f9dea6d04d6ed0e2c65d1b51b" ], [ "Parsing.parser_st_nochk", @@ -167,7 +167,7 @@ "typing_Slice.as_seq" ], 0, - "e3e78b94a3f77416c9c0c9d46c7d8313" + "90968849ccc546511824b646c954b29b" ], [ "Parsing.validation_checks_parse", @@ -176,7 +176,7 @@ 1, [ "@query" ], 0, - "259a2e6af7a00f7c407ff538cb5bf741" + "2b33d4b3314abe0d04d07707592c0a26" ], [ "Parsing.stateful_validator", @@ -202,7 +202,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "0f189f95e98e56affcfb8470b2ddab51" + "c0c8aa60a4dddb857874b68e3d0f3e55" ], [ "Parsing.then_check", @@ -361,7 +361,7 @@ "typing_Slice.as_seq", "typing_Slice.u32_add_overflows" ], 0, - "624a809ef120c80b8d0e7819b7ad24aa" + "26ac68d77e7a38cefe243b783f46f118" ], [ "Parsing.validate_done_st", @@ -444,7 +444,7 @@ "unit_typing" ], 0, - "e2c83841c6d0c23dc39d6e4b8d73ca6d" + "fd7fa444d363a126b52318dc37d24d78" ], [ "Parsing.validate_done_st", @@ -470,7 +470,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "78ffd9d88093620ea532f706e2403e56" + "db08641271bd57e466be9e23730432b7" ], [ "Parsing.validate_fail", @@ -517,7 +517,7 @@ "typing_FStar.Set.mem" ], 0, - "5686a6cee2590dec7134dff143388393" + "076bedee839c554a173c69ba406d305c" ], [ "Parsing.validate_fail", @@ -543,7 +543,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "eb593df701481559bff524f235b2f520" + "bfb28bd2967ee60c307bf8e4599d5199" ], [ "Parsing.and_then_offset", @@ -595,7 +595,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "4f8a13897abe4e5740bf51fa284d63cf" + "5cb41fa8b348585f33d5ae80afda3c78" ], [ "Parsing.parse_many_parse_one", @@ -604,7 +604,7 @@ 1, [ "@query" ], 0, - "51600945e03ab37a4253cdd71132b15a" + "e8dbb842b12385fa21f0a678c0cf5eb5" ], [ "Parsing.parse_many_parse_one", @@ -663,7 +663,7 @@ "typing_Parsing_Tm_abs_def4c30b0e696cb7641fc338f7922e40" ], 0, - "ab864282dac791e720834afd478b4a4a" + "78e1c4e5be465789b631de793059adb8" ], [ "Parsing.validate_n_more", @@ -719,7 +719,7 @@ "unit_typing" ], 0, - "a969a901672ff1fc3cb38f59623a5490" + "b33398c3802c6fc249564e23b3c33d35" ], [ "Parsing.validate_n_more", @@ -776,7 +776,7 @@ "typing_Slice.__proj__BSlice__item__len", "typing_Slice.as_seq" ], 0, - "7f9c51fe59199e5049a81f4cceeb50ff" + "6d4cb7c353bd8adec51fe5e9162414aa" ], [ "Parsing.validate_one_more", @@ -836,7 +836,7 @@ "typing_Slice.as_seq", "unit_typing" ], 0, - "1456ba4b9b0dbef08ee68fd1306375f7" + "62a73dbb208f71fa343145df058d9a47" ], [ "Parsing.validate_one_more", @@ -929,7 +929,7 @@ "typing_Slice.as_seq" ], 0, - "a769195a2f1f8e4dbc69dceced6d6afe" + "e056d7f7bd90f3500fc05a998cd390b2" ], [ "Parsing.for_readonly", @@ -948,7 +948,7 @@ "typing_FStar.UInt32.v" ], 0, - "15a8620e5d465d8993db1b1b62545378" + "da05776a5dc9d30e7368dc2a685bc5fc" ], [ "Parsing.for_readonly", @@ -1071,7 +1071,7 @@ "typing_FStar.UInt32.v", "unit_typing" ], 0, - "aa298c93cc89f14fd0ab6aa534643d41" + "5aaca1f50a07e33d2187040d71853a6a" ], [ "Parsing.for_readonly", @@ -1187,7 +1187,7 @@ "typing_FStar.UInt32.v" ], 0, - "dd052414556a5cacdfd3f11f936c77aa" + "5a5e2b2eb3c16423f22451eccc654329" ], [ "Parsing.validate_many_st", @@ -1204,7 +1204,7 @@ "typing_FStar.UInt32.v" ], 0, - "609b4a0d8464a854232ab854b9372c91" + "5b103adf6536bb870274b34162259b87" ], [ "Parsing.validate_many_st", @@ -1345,7 +1345,7 @@ "typing_Slice.as_seq" ], 0, - "3c039c8eccdf059117949d545d7b7ca2" + "7aebf066f3f4f93343272065876125bb" ], [ "Parsing.and_then", @@ -1380,7 +1380,7 @@ "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b" ], 0, - "82d4bbd4c25dcc22bc6d55d7576b7df5" + "d186640863874115e2797d551ac40fe9" ], [ "Parsing.parse_ret", @@ -1401,7 +1401,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "760693f79795b4ec3625d80a44c48de6" + "7efe4dd4f22afb2719aa016c87d10868" ], [ "Parsing.parsing_done", @@ -1413,7 +1413,7 @@ "primitive_Prims.op_Equality", "projection_inverse_BoxBool_proj_0" ], 0, - "25ef47e8e38d08d884c8c7ad6b852618" + "aaaae0b426a0e017081dab02fe7a8748" ], [ "Parsing.parse_result", @@ -1422,7 +1422,7 @@ 1, [ "@query" ], 0, - "2cb74390ac1f6e56a2de6843431a18c1" + "0cfce9d5d74e596a02b1d801ac98085f" ], [ "Parsing.parse_many", @@ -1454,7 +1454,7 @@ "well-founded-ordering-on-nat" ], 0, - "a143d295fbf71245e0eb60e747b9bea2" + "570b11aa426f53e486435de816bdac5c" ], [ "Parsing.parser_st", @@ -1483,7 +1483,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "e9835499731265d9e6e5462ee955b6ce" + "943a22a78e69e4acc8624fd247622eb6" ], [ "Parsing.parser_st_nochk", @@ -1516,7 +1516,7 @@ "typing_Slice.as_seq" ], 0, - "752fa9b6dc2e1caa6c1e88810f0496c6" + "378982aeeb7496588620233640ee49e1" ], [ "Parsing.validation_checks_parse", @@ -1525,7 +1525,7 @@ 1, [ "@query" ], 0, - "080b7d63490e2cc47e759516bc50d1af" + "205ff16093a5706e46455a74666dfc53" ], [ "Parsing.stateful_validator", @@ -1551,7 +1551,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "19716b284a556c3777c450c1b967dd1d" + "a4812097e1bcb575e53ec674bb0cca2e" ], [ "Parsing.then_check", @@ -1710,7 +1710,7 @@ "typing_Slice.as_seq", "typing_Slice.u32_add_overflows" ], 0, - "d586f02e71b0fdaad3b62a8ba281e6ba" + "7196e731e07b583a8fa9547a0d035034" ], [ "Parsing.validate_done_st", @@ -1743,7 +1743,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "ffc02e564f0db056e3df930d9a437e21" + "ce63e36fdcee2d3def59351995838d83" ], [ "Parsing.validate_fail", @@ -1776,7 +1776,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "130b69ffe0c17462c36c186eb5cdd3a9" + "f5a32d9c1e1090857d1cd511775e92f9" ], [ "Parsing.and_then_offset", @@ -1785,7 +1785,7 @@ 1, [ "@query" ], 0, - "ce6d82db28a8bbbcb2998ae4fbd84cdb" + "8f664b87e9d0072a06dab71805e3ffa7" ], [ "Parsing.parse_many_parse_one", @@ -1794,7 +1794,7 @@ 1, [ "@query" ], 0, - "3699671e839214a92aec881ddca14dcc" + "131cc4e449b2a6b88e52de9b026a9755" ], [ "Parsing.validate_n_more", @@ -1850,7 +1850,7 @@ "unit_typing" ], 0, - "f0caedaefb3484f4ee5b16e01b73a8b3" + "f066d206f7d149bf675867b13c6e1fec" ], [ "Parsing.validate_one_more", @@ -1910,7 +1910,7 @@ "typing_Slice.as_seq", "unit_typing" ], 0, - "c3bf4d979f399ba5d3b49766a3e2b65a" + "95e5599329d1079d98df309e9ef60fa2" ], [ "Parsing.for_readonly", @@ -1929,7 +1929,7 @@ "typing_FStar.UInt32.v" ], 0, - "f0604eb16c25152061e876e839ab1ab4" + "d9d58764f174ef4f6aa784b2f34613eb" ], [ "Parsing.validate_many_st", @@ -2070,7 +2070,7 @@ "typing_Slice.as_seq" ], 0, - "4ab853efb4d273cc6f505f09b2991b6b" + "9a23252847229c8beabcf13aeff668c2" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/PureEncoder.fst.hints b/examples/kv_parsing/PureEncoder.fst.hints index 17f48e894fd..6a6351d1d34 100644 --- a/examples/kv_parsing/PureEncoder.fst.hints +++ b/examples/kv_parsing/PureEncoder.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "equation_FStar.UInt8.byte", "equation_Slice.byte" ], 0, - "8afb09304dbdc46ad385298796e2d585" + "c7e4dacfe0c683c134a5ec5f5f59c9d1" ], [ "PureEncoder.encode_store", @@ -30,7 +30,7 @@ "typing_KeyValue.__proj__Store__item__num_entries" ], 0, - "08e68435edaf9365534f87e62885fa4f" + "01357ddadb3777417c2a401a339ca286" ], [ "PureEncoder.encode_entry", @@ -39,7 +39,7 @@ 1, [ "@query", "equation_FStar.UInt8.byte", "equation_Slice.byte" ], 0, - "5a0f43adb2a2e5245c0b04fd40e71503" + "6419f7f8c9ed1cefac98d68da6686b25" ], [ "PureEncoder.encode_store", @@ -61,7 +61,7 @@ "typing_KeyValue.__proj__Store__item__num_entries" ], 0, - "fce9cdad271600f870b97b7d121ae649" + "82eb0e349d9ceefd422756452ca00879" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/PureParser.fst.hints b/examples/kv_parsing/PureParser.fst.hints index 0add1056ecc..2678c4fd2a7 100644 --- a/examples/kv_parsing/PureParser.fst.hints +++ b/examples/kv_parsing/PureParser.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "equation_FStar.UInt8.byte", "equation_Slice.byte" ], 0, - "b72a6cda9348a92ca6b6e8b34e3f4afb" + "8a7ec80a54ec5f7c56d8f641c9ee86b6" ], [ "PureParser.parse_abstract_store", @@ -25,7 +25,7 @@ "typing_FStar.UInt32.v" ], 0, - "3e327c09ccea27af26eac760e0067024" + "bf7d958a052acbb9e6a94b773f19e1cb" ], [ "PureParser.parse_entries", @@ -42,7 +42,7 @@ "typing_FStar.UInt32.v" ], 0, - "9792d1dde807353aed22ca08e79dfa10" + "0b4419c7972a8cf5dfbb6f28e5f3c0cc" ], [ "PureParser.parse_entry", @@ -51,7 +51,7 @@ 1, [ "@query", "equation_FStar.UInt8.byte", "equation_Slice.byte" ], 0, - "2db993c9be928d2ef58be21d80bf0004" + "3965e6008e141cdefa6d807c2fd5cefc" ], [ "PureParser.parse_abstract_store", @@ -68,7 +68,7 @@ "typing_FStar.UInt32.v" ], 0, - "d33bf59b14a0f62fdec05a922b6b0c3d" + "872e39614aa1e5365a9c31976316aa08" ], [ "PureParser.parse_entries", @@ -85,7 +85,7 @@ "typing_FStar.UInt32.v" ], 0, - "b1216510183b51ff1d3f062d679a13b3" + "c370e164bb311a869b80e1127dfc360e" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/PureValidator.fst.hints b/examples/kv_parsing/PureValidator.fst.hints index 5070d5f6d5f..c6cd0b13d21 100644 --- a/examples/kv_parsing/PureValidator.fst.hints +++ b/examples/kv_parsing/PureValidator.fst.hints @@ -34,7 +34,7 @@ "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b" ], 0, - "d4aa6e57ff7a8c1ffd0123af62f5ac68" + "3c256134c2efefc00920aa49291dea28" ], [ "PureValidator.skip_bytes", @@ -47,7 +47,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "f10d8085db6ad71e81fe29fea0ee1425" + "97d0b245e38e9811ea9f0496b0cda2b8" ], [ "PureValidator.parser_validation_checks_parse", @@ -56,7 +56,7 @@ 1, [ "@query" ], 0, - "e7437f7d4582f27769372e8688dea9ca" + "1773f3e2a332901ea00a82f1ada31c95" ], [ "PureValidator.validate_u16_array", @@ -105,7 +105,7 @@ "token_correspondence_IntegerParsing.parse_u16", "unit_typing" ], 0, - "1c8dbfb1dd9a223b6bf2a72b5e8e4154" + "83a05f067609fe54ec19bb76c7706f7e" ], [ "PureValidator.validate_u32_array", @@ -159,7 +159,7 @@ "typing_FStar.UInt32.v", "unit_typing" ], 0, - "9ba21cfc9312567b872b4c17cfcc104d" + "1183ad43a0501d808f96e7d1e1f3d0b7" ], [ "PureValidator.validate_accept", @@ -180,7 +180,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "edc8133ccc36f328f0d98fee452acf82" + "e16a4880b2919beb0d9c3e539e74a3c9" ], [ "PureValidator.validate_many'", @@ -198,7 +198,7 @@ "well-founded-ordering-on-nat" ], 0, - "f50c1726962f324790d0eb44af99875e" + "dc4fb00241e76f6d3ef46f9d9437f101" ], [ "PureValidator.intro_validator_checks", @@ -207,7 +207,7 @@ 1, [ "@query", "equation_PureValidator.validator_checks" ], 0, - "bd03256805aa235a75d8f888fc4403bc" + "ea1e1c98b2f6b010e858d5cc9b835225" ], [ "PureValidator.validate_many'_ok", @@ -279,7 +279,7 @@ "well-founded-ordering-on-nat" ], 0, - "5f8c166477cfa255148efdc9396033a8" + "9d264c21388d09bdfc11c2a9cccec336" ], [ "PureValidator.validate_many", @@ -288,7 +288,7 @@ 1, [ "@query" ], 0, - "7d7e66bb80f874e8f83e9428bd912eef" + "785c8ef559017fe3c5659795376ec265" ], [ "PureValidator.validate_done", @@ -300,7 +300,7 @@ "primitive_Prims.op_Equality", "projection_inverse_BoxBool_proj_0" ], 0, - "606061b4df72c7f6328885eeef847ca6" + "618f62b616cb95244c8eea933b67826f" ], [ "PureValidator.validate_done", @@ -325,7 +325,7 @@ "token_correspondence_Parsing.parsing_done", "unit_typing" ], 0, - "b873a6778f93952d25366fc19aab81f9" + "73c0feb50510b5fc5a8e70cc47710ea0" ], [ "PureValidator.seq", @@ -360,7 +360,7 @@ "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b" ], 0, - "8de2b6b23abca0725eed83a0fdac60b1" + "db862359abeb0abcff466cfa45597310" ], [ "PureValidator.skip_bytes", @@ -373,7 +373,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "6b6b7f96f91167e115a49b14a9b06de3" + "208a20438568ef0c19ce073b86aaf32e" ], [ "PureValidator.parser_validation_checks_parse", @@ -382,7 +382,7 @@ 1, [ "@query" ], 0, - "b8565ff03cfc9bcea192835b2e9baa62" + "c0a6b6c95a02be60d8b4f0ec6877bbb0" ], [ "PureValidator.validate_u16_array", @@ -431,7 +431,7 @@ "token_correspondence_IntegerParsing.parse_u16", "unit_typing" ], 0, - "0e88e903a60400f4c7b58a83eaf7e3f0" + "39633b177a9cf637902c249d40741b24" ], [ "PureValidator.validate_u32_array", @@ -485,7 +485,7 @@ "typing_FStar.UInt32.v", "unit_typing" ], 0, - "60506bd227edd75d25b487c9dcbb690e" + "a5b54290f1a41f7cfbc56334adccb915" ], [ "PureValidator.validate_accept", @@ -506,7 +506,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "d8678b2bbe8b0a154ca3055776cf5ca5" + "41a97d3b1eb9c1109f19366ba23784a5" ], [ "PureValidator.validate_many'", @@ -524,7 +524,7 @@ "well-founded-ordering-on-nat" ], 0, - "5c5b951db98d25fc54aa322ad953a55f" + "27cad72e3276a190879051c16a375b85" ], [ "PureValidator.validate_many", @@ -533,7 +533,7 @@ 1, [ "@query" ], 0, - "9faf3c77c7b6102fc67b117409be3550" + "2fa76855cdfbcad237876187ff4fdf66" ], [ "PureValidator.validate_done", @@ -545,7 +545,7 @@ "primitive_Prims.op_Equality", "projection_inverse_BoxBool_proj_0" ], 0, - "7b9c44cc0e8ab03d206650788800b476" + "b88669afdc317e14217f4e884396e2d5" ], [ "PureValidator.validate_done", @@ -570,7 +570,7 @@ "token_correspondence_Parsing.parsing_done", "unit_typing" ], 0, - "7b900c41811818d604d41b92b65b2213" + "f64dcc1a1cc56bfd212f2704db0e57b8" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/Serializer.fst.hints b/examples/kv_parsing/Serializer.fst.hints index 1a274acb5e1..aec7e0cb995 100644 --- a/examples/kv_parsing/Serializer.fst.hints +++ b/examples/kv_parsing/Serializer.fst.hints @@ -27,7 +27,7 @@ "typing_KeyValue.__proj__EntrySt__item__val_st" ], 0, - "8b58ed25aec835ba599327c5e1e3702e" + "bbdc752ba248f563f188aaff6b0bd0c5" ], [ "Serializer.ser_entry", @@ -67,7 +67,7 @@ "typing_Serializer.entry_st_bufs" ], 0, - "95599f1119cef39e2c90080b20928ba9" + "e18f8b1624ceafe211b3a8c3faf67642" ], [ "Serializer.adjacent_entries_disjoint", @@ -83,7 +83,7 @@ "typing_FStar.Buffer.__proj__MkBuffer__item__max_length" ], 0, - "d41754aa29da5da91183fe09efd51b9e" + "4f39d20ee177e96ed36052c2f5c825de" ], [ "Serializer.writer_inv", @@ -110,7 +110,7 @@ "typing_Serializer.__proj__Mkwriter__item__num_entries_written" ], 0, - "c8edd1900c5ab90655da0bf2cb3120e3" + "245900f012c056ec0f75f611347d9218" ], [ "Serializer.adjacent_advance", @@ -172,7 +172,7 @@ "typing_Slice.truncated_slice" ], 0, - "789611ac19a799a35894100653fe4037" + "8674ab26da3bfcbdec9b8f4a58551656" ], [ "Serializer.adjacent_truncate", @@ -224,7 +224,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "0bbc5d6581ce9bfaeb78059829d749e9" + "9c3009b4c1149b7ab8d41c79fdea5225" ], [ "Serializer.adjacent_0len", @@ -241,7 +241,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "c6f22f007e446892458f57cd7a483cb6" + "e3684746890cf7f44eee88ecf0641066" ], [ "Serializer.adjacent_0len", @@ -298,7 +298,7 @@ "typing_Slice.truncated_slice" ], 0, - "f091c81fc9911da94c54fbc94d44ab45" + "1b5f184b3a24081aa5fb4f22d38a74df" ], [ "Serializer.writer_init", @@ -401,7 +401,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "ce157da75923f7c925868a18b9129dfa" + "107cd30ffb7048ebb59349f5ac937638" ], [ "Serializer.writer_reinit", @@ -410,7 +410,7 @@ 1, [ "@query" ], 0, - "e590c20cb777e2b03b50a4ad4b9e33fe" + "e2c88d3e4a7277628fb2caa4c6e3defd" ], [ "Serializer.writer_reinit", @@ -502,7 +502,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "389c1fb724e3080e630d172bbe9b6eb4" + "a6b6970586cf352c9f64f87419d1a77f" ], [ "Serializer.join_slices", @@ -568,7 +568,7 @@ "typing_Slice.u32_add_overflows" ], 0, - "cafe3f2bc22eea9478ac3914f1c3c0c6" + "1c095b64e91c3d84047caa1ce34acfb7" ], [ "Serializer.enc_one_more", @@ -577,7 +577,7 @@ 1, [ "@query" ], 0, - "d8506a484a527215f9c0ebcb6dfee6a9" + "8a1b4c956a35d86571fefdaf0ce6986d" ], [ "Serializer.enc_one_more", @@ -617,7 +617,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "15e053cb70695be129c46ca80425bda8" + "add4580aad5f98d2a47cc469b90f6db3" ], [ "Serializer.max_entries_to_write", @@ -637,7 +637,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "acb4d5e4cfbb11f61cb90bbd3ecf5a01" + "1f7c6bb18e4844212d6df9d228b9b2e5" ], [ "Serializer.lt_max_entries", @@ -654,7 +654,7 @@ "refinement_interpretation_Serializer_Tm_refine_cbf5a4e73eb6850050f387d18311bd92" ], 0, - "3cb8b9fc0002ff4240f46e5d4ad7b1fb" + "cdb02c98e324cc59aa91f17ffdd06bcb" ], [ "Serializer.join_adjacent_stable", @@ -683,7 +683,7 @@ "typing_Serializer.join_slices", "unit_typing" ], 0, - "245d4ffe643f25e4773513685d4fb12b" + "7490ffe8cbf5d7f50f4e1900701ef4ab" ], [ "Serializer.writer_append", @@ -692,7 +692,7 @@ 1, [ "@query" ], 0, - "896519d59475867dcd8bfc8c8ce93068" + "78bd4ea69267cc73c844fbf4ef12e8ed" ], [ "Serializer.writer_append", @@ -887,7 +887,7 @@ "typing_Slice.buffer_split_at", "typing_Slice.u32_add_overflows" ], 0, - "b29a1b7e202411ea3d07752d9a90afbd" + "81eb66b7132e5fdd8b8ef2757f6104bf" ], [ "Serializer.join_is_concat", @@ -901,7 +901,7 @@ "typing_FStar.Buffer.__proj__MkBuffer__item__max_length" ], 0, - "31c71d5f07699da728fa5314776be7bd" + "3cda86ee6732bfd0d4b7c3e2085e4a1d" ], [ "Serializer.join_is_concat", @@ -951,7 +951,7 @@ "typing_FStar.UInt32.add", "typing_FStar.UInt32.v" ], 0, - "e7e59a0f5146d15d000654fcb86a87eb" + "b91dd3962dd23d670a656f776be90c0b" ], [ "Serializer.writer_store_buf", @@ -1005,7 +1005,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "e77f89b9b02c14bd8cd40dba31069084" + "2476745560eaeff882d63667547ea651" ], [ "Serializer.writer_finish", @@ -1107,7 +1107,7 @@ "typing_Slice.buffer_split_at" ], 0, - "ff2d5b4f80753b79437751a0a4543b41" + "f2ae2cee028d68165de427e7f3e35d52" ], [ "Serializer.writer_finish", @@ -1231,7 +1231,7 @@ "typing_Slice.bslice_split_at" ], 0, - "55aa304e31c2c5e7dd6edb87fb544a6b" + "102d6dd80c05134a621cb7372fdf6e70" ], [ "Serializer.enc_entry_st", @@ -1259,7 +1259,7 @@ "typing_KeyValue.__proj__EntrySt__item__val_st" ], 0, - "38ec8cde817a4a3934858f1535538a46" + "6361ff0c978e0a27512878dee03b7d1d" ], [ "Serializer.ser_entry", @@ -1299,7 +1299,7 @@ "typing_Serializer.entry_st_bufs" ], 0, - "ecc905f50e6113a5b30b2c8a825b56e7" + "f2d2abbe7332dc3130c1ee91e1de2a25" ], [ "Serializer.ser_entry", @@ -1334,7 +1334,7 @@ "typing_Serializer.entry_st_bufs" ], 0, - "4dbfecea5671f794d144133b44fad2fa" + "49b97d61cb31eed22c7381d58e80118d" ], [ "Serializer.writer_inv", @@ -1361,7 +1361,7 @@ "typing_Serializer.__proj__Mkwriter__item__num_entries_written" ], 0, - "265455382d3a25c092e2d641d501d0cf" + "37f5080f2ea77c2275dec566c2cef3a0" ], [ "Serializer.adjacent_0len", @@ -1378,7 +1378,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "ef521f219a0bfc96e114457b70aae2c7" + "5cb3e8338dc19256f0b4079b49c01ab4" ], [ "Serializer.writer_init", @@ -1387,7 +1387,7 @@ 1, [ "@query" ], 0, - "18b356ed84e7747b1ce9102e27988a65" + "8dacb5683496f1584b9e9da22c15d451" ], [ "Serializer.writer_reinit", @@ -1396,7 +1396,7 @@ 1, [ "@query" ], 0, - "0a2043339d028970da8182e6cc77eb73" + "f0358544dcc42b97f500a83408de010a" ], [ "Serializer.join_slices", @@ -1464,7 +1464,7 @@ "typing_Slice.u32_add_overflows" ], 0, - "6c929e4cede6a9ed35f983a0d348f72e" + "5c866e969afbf688436d35de7bb36fe3" ], [ "Serializer.join_slices", @@ -1480,7 +1480,7 @@ "refinement_interpretation_Serializer_Tm_refine_6189a2d1a8309b48981e73407c0aa96c" ], 0, - "f31c5b73afb80f082b1ae08455e35292" + "2860dfe2fef585f59be2ec49027b6556" ], [ "Serializer.enc_one_more", @@ -1489,7 +1489,7 @@ 1, [ "@query" ], 0, - "720efe3a855042a0c1bb3de1ff8394a9" + "2ff66e8358b14b168eaff009414b261f" ], [ "Serializer.max_entries_to_write", @@ -1508,7 +1508,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "b44e1e73583f10b740d02e4e55bd8187" + "4816c3463000b907f93dcd84c3e0160c" ], [ "Serializer.join_adjacent_stable", @@ -1521,7 +1521,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "b3e641d5710e6d4e84b85a2a010fac6f" + "fd12b08297c8428ace35b4c80cda1ad0" ], [ "Serializer.writer_append", @@ -1530,7 +1530,7 @@ 1, [ "@query" ], 0, - "2f2883e99348107426c77303692aa299" + "bca54b72092107706d0d7553641d2847" ], [ "Serializer.join_is_concat", @@ -1544,7 +1544,7 @@ "typing_FStar.Buffer.__proj__MkBuffer__item__max_length" ], 0, - "fdb8b19b743b4d45bcf9439fd36567cc" + "7aaac1958eefe072e80360020dbccea3" ], [ "Serializer.writer_store_buf", @@ -1598,7 +1598,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "641e4dcb0583cf2fb16fa4ca61cda42b" + "17c11bccfb19dcc420bccb1931380732" ], [ "Serializer.writer_finish", @@ -1607,7 +1607,7 @@ 1, [ "@query" ], 0, - "fe69486f18f58c368d4363879bc10a73" + "1abfcb00bc565ed39ac5b0630823cf30" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/Serializing.fst.hints b/examples/kv_parsing/Serializing.fst.hints index ce567cc86e4..77eb9284090 100644 --- a/examples/kv_parsing/Serializing.fst.hints +++ b/examples/kv_parsing/Serializing.fst.hints @@ -27,7 +27,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.length" ], 0, - "2e7a6f7b7e495036d2a282b847dd7319" + "1e0a9aed007a4f0cb319023a39049ef0" ], [ "Serializing.serialized", @@ -596,7 +596,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.length" ], 0, - "743511420ecdad10adea82ef059dc581" + "a9860a80cfd7490f9d360315acb02fea" ], [ "Serializing.serialized", diff --git a/examples/kv_parsing/ValidatedAccess.fst.hints b/examples/kv_parsing/ValidatedAccess.fst.hints index 07a69320390..0aa9a892ba4 100644 --- a/examples/kv_parsing/ValidatedAccess.fst.hints +++ b/examples/kv_parsing/ValidatedAccess.fst.hints @@ -22,7 +22,7 @@ "typing_FStar.UInt32.v" ], 0, - "8a0a6ae2f182f171866fb870d27d7ecc" + "8c886160a7a186444b1caa26cf9e358d" ], [ "ValidatedAccess.for_readonly2", @@ -148,7 +148,7 @@ "typing_FStar.UInt32.v", "unit_typing" ], 0, - "c7ba2fd17d9cb3d7da426195c6b4f1e4" + "bf2b4a2a43fd94ecdc51f4bc77b3c556" ], [ "ValidatedAccess.for_readonly2", @@ -268,7 +268,7 @@ "typing_FStar.UInt32.v" ], 0, - "062e17e66ffe14db848d560b02af3506" + "90f6050ffe938cf1e0644842448784e0" ], [ "ValidatedAccess.lookup_in_entries", @@ -288,7 +288,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "c6732d006ed142ad73af268c176e9714" + "555635f8435c1c5051a4de882273a9d2" ], [ "ValidatedAccess.lookup_in_entries_st", @@ -318,7 +318,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "d4496b89807abb482a1fd23d96ba73a4" + "b2045881504ea8950858cf962ea49d38" ], [ "ValidatedAccess.lookup_st", @@ -348,7 +348,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "66616e001b5a42625ef063c48f466c97" + "32ecfca804ad795cc77d4791151d07ba" ], [ "ValidatedAccess.lookup_st", @@ -473,7 +473,7 @@ "typing_Slice.as_seq" ], 0, - "fd5da9dd699837ab38abb31b041db990" + "c707677526c5d980eb40a1b54bc176d7" ], [ "ValidatedAccess.for_readonly2", @@ -496,7 +496,7 @@ "typing_FStar.UInt32.v" ], 0, - "8739c8c34ab8aa25d1bbb56c7fb6b18e" + "ee877869fac33d586f835295afd41d4e" ], [ "ValidatedAccess.lookup_in_entries", @@ -516,7 +516,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "b1f88e05e4fc99fcd9317483927d7693" + "ffb46e46f91e11f2960ee547e2032986" ], [ "ValidatedAccess.lookup_in_entries_st", @@ -550,7 +550,7 @@ "typing_Slice.as_seq" ], 0, - "18e34174d645bb9b7a59b5c9f1bf5cf0" + "44aaf393044458fad2c83ffe6f7888e3" ], [ "ValidatedAccess.lookup_st", @@ -591,7 +591,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "14d280388142652cd9dbf08219b4ffa9" + "77abbb5c57ba7e10d2a9180a0625edf9" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/ValidatedParser.fst.hints b/examples/kv_parsing/ValidatedParser.fst.hints index a10ecabbf8f..c977658d1a2 100644 --- a/examples/kv_parsing/ValidatedParser.fst.hints +++ b/examples/kv_parsing/ValidatedParser.fst.hints @@ -14,7 +14,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "4932d7df5211987c9cf9583568aed582" + "cbde2f4b8101ae47d2db04e45ccf88ea" ], [ "ValidatedParser.fold_left_store_n", @@ -44,7 +44,7 @@ "typing_FStar.List.Tot.Base.length", "well-founded-ordering-on-nat" ], 0, - "934ca925d73030b0795e3108701b93f7" + "c1463deb3b722cbc0d49c51899b4ddea" ], [ "ValidatedParser.fold_left_store_n_spec", @@ -66,7 +66,7 @@ "typing_KeyValue.__proj__Store__item__num_entries" ], 0, - "1fa9c3d68fd6bd665f6495503ca2dc4c" + "61957285d95b6157d716c537d59e1cf4" ], [ "ValidatedParser.fold_left_store_n_spec", @@ -118,7 +118,7 @@ "well-founded-ordering-on-nat" ], 0, - "5541e234f1d07e679621e8ea3b29fdad" + "20871eff2d83f27c9628a7c8b2ae9830" ], [ "ValidatedParser.fold_left_entries_st", @@ -138,7 +138,7 @@ "proj_equation_FStar.Monotonic.HyperStack.HS_h" ], 0, - "29295016d37b520aff775fd1e35783f5" + "3e980bad19980aa3bbdbeef57aaeebe8" ], [ "ValidatedParser.fold_left_buffer", @@ -188,7 +188,7 @@ "typing_FStar.UInt32.v", "well-founded-ordering-on-nat" ], 0, - "bc828c25b79bdca5834cd52330c33cc8" + "2422ea1c0dbbfe9570d37b27a5b1ff7f" ], [ "ValidatedParser.parse_num_entries_valid", @@ -239,7 +239,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "595c53eaf85058dac365d737b23b5c5a" + "c52246a890167dc8cddb9ae039fbbd8b" ], [ "ValidatedParser.parse_num_entries_valid", @@ -283,7 +283,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "14dee8d9fffd8b57dd2be1b77549f6a9" + "924191644aea7e28225263db28c312cb" ], [ "ValidatedParser.parse_entry_st_nochk", @@ -465,7 +465,7 @@ "typing_Slice.as_seq" ], 0, - "c4c5d08b2d7c7f9678b288c2c0a6f567" + "518700cb4a9f017a4020bc58fefe5f02" ], [ "ValidatedParser.parse_entry_st_nochk", @@ -500,7 +500,7 @@ "typing_Slice.as_seq" ], 0, - "f91da6fa725c13461eaadf4b6a8b083b" + "6f4d8cb7e8904d61c9098583859ca6c9" ], [ "ValidatedParser.parse_many_next", @@ -564,7 +564,7 @@ "typing_FStar.Pervasives.Native.__proj__Some__item__v" ], 0, - "be120fc713c70865adea06d37ebd52b9" + "e3d92ac4a71d6894d179fdf16342fae0" ], [ "ValidatedParser.parse_one_entry", @@ -616,7 +616,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "ed1c79112e1fbc1157632fdb43ac0d8f" + "50f08c45f6951a441927652f1da7c336" ], [ "ValidatedParser.parse_one_entry", @@ -709,7 +709,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "83756c9e359dfcb0744f37702885aced" + "99dc8410141d9cd1f351d61a1d47f3e1" ], [ "ValidatedParser.fold_left_store_n_unfold1", @@ -736,7 +736,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "6511aa925938cf92b1d6f5764c3404d8" + "527435beea0cc66e0ed82a6c9689b426" ], [ "ValidatedParser.fold_left_store_n_unfold1", @@ -753,7 +753,7 @@ "refinement_interpretation_ValidatedParser_Tm_refine_30c4f26016c0e8363d23289de00ee4f6" ], 0, - "72b46fcba4fc13298eda4433e107a534" + "8da8f924cd2d13bdb019381891605341" ], [ "ValidatedParser.fold_left_buffer_n_mut_st", @@ -804,7 +804,7 @@ "typing_Slice.__proj__BSlice__item__p", "unit_typing" ], 0, - "a1809578621cf1429cab8e3037100c23" + "0d3711e05971966ff194d8f17d27fa1c" ], [ "ValidatedParser.fold_left_buffer_n_mut_st", @@ -817,7 +817,7 @@ "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87" ], 0, - "4f6f6a5376226fc3c47446ca5f7ce967" + "8fa9b64df202bb8f9c1336bab2665a70" ], [ "ValidatedParser.fold_left_buffer_n_st", @@ -844,7 +844,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "21354f51e04a845dae8b51dc770a9254" + "103e3d70b197b86d8cb6258b07cad758" ], [ "ValidatedParser.fold_left_buffer_n_st", @@ -1022,7 +1022,7 @@ "typing_Slice.as_seq" ], 0, - "70ad3a0faad98107d760db466d658b41" + "f4b9bfbe761b81fa04900c76a72481ef" ], [ "ValidatedParser.fold_left_buffer_n_st", @@ -1197,7 +1197,7 @@ "typing_Slice.as_seq" ], 0, - "2871d932757ecb81c7ec6ec569504146" + "49f9497489e02e6ec70656fc9f25be05" ], [ "ValidatedParser.fold_left_buffer_st", @@ -1223,7 +1223,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "df48ff2e6a7ad5b30da5a28736cee338" + "aff71c97feaa80869171d6c0bcfb5aec" ], [ "ValidatedParser.fold_left_buffer_st", @@ -1340,7 +1340,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.advance_slice" ], 0, - "089c478a54cc07ae0212070a3ddedab1" + "ffcabce4ea39317d9538380da28edcb1" ], [ "ValidatedParser.fold_left_buffer_st", @@ -1457,7 +1457,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.advance_slice" ], 0, - "21e7cdc6007468bad46e570a063d0ad7" + "c036eb00c1185c9918970131441cd8c6" ], [ "ValidatedParser.fold_left_n_count", @@ -1483,7 +1483,7 @@ "typing_FStar.List.Tot.Base.length", "typing_FStar.UInt32.v" ], 0, - "7c210018ce742f507255641ee6e2d1c9" + "c429e93428d5a8ed7e5cbce987e8ea43" ], [ "ValidatedParser.fold_left_n_count", @@ -1530,7 +1530,7 @@ "typing_FStar.UInt32.v" ], 0, - "a0d2de4e36748654a8507472a59eeb14" + "c3a63c0e3fd7f2961ea9ac4b1d5657d3" ], [ "ValidatedParser.fold_left_count", @@ -1559,7 +1559,7 @@ "typing_KeyValue.__proj__Store__item__num_entries" ], 0, - "398d38fb51ae0ba34ff0c0a73f07d9df" + "c2d44dce87711c6b3c2a788846a2bc5e" ], [ "ValidatedParser.count_entries_example", @@ -1585,7 +1585,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "6651313c1ddb2d4eedee3adc9befffb4" + "9fa9f3d21a52b8ed40beeb3d9f06e067" ], [ "ValidatedParser.count_entries_example", @@ -1661,7 +1661,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "b1740b3f27bc9502fbb42947f8544eae" + "14431891d03d72daff25232ea9b6e2d9" ], [ "ValidatedParser.fold_left_store_aux", @@ -1676,7 +1676,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "cb99890c6033d627a8cc3c7c3f623c3c" + "a776324e2f1c039d8e90d609edebe1d4" ], [ "ValidatedParser.fold_left_store_n", @@ -1706,7 +1706,7 @@ "typing_FStar.List.Tot.Base.length", "well-founded-ordering-on-nat" ], 0, - "5dcb0f799c1fceffcfeb21c5eaf64294" + "166e28034498272f5bf7946637372ac3" ], [ "ValidatedParser.fold_left_store_n_spec", @@ -1758,7 +1758,7 @@ "well-founded-ordering-on-nat" ], 0, - "eb98f3a2f8c0425c87a2856189ee9725" + "87275bb38893c841dc2075181d50fe6d" ], [ "ValidatedParser.fold_left_buffer", @@ -1808,7 +1808,7 @@ "typing_FStar.UInt32.v", "well-founded-ordering-on-nat" ], 0, - "92b0de39844057e86cc1df22ac06210b" + "3b5af6275ce316ce560dff9afdc87277" ], [ "ValidatedParser.parse_num_entries_valid", @@ -1859,7 +1859,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "e1e77e8856b82e3294229ce5eff2c3ff" + "92821946fd754da0046510d0f2af6d92" ], [ "ValidatedParser.parse_entry_st_nochk", @@ -1894,7 +1894,7 @@ "typing_Slice.as_seq" ], 0, - "1f4b8ce8ec618f454afd9bfe6b7bf98e" + "76f68aaee630f1c2d90d5cf3a9405ada" ], [ "ValidatedParser.parse_many_next", @@ -1939,7 +1939,7 @@ "token_correspondence_Parsing.parse_many", "unit_typing" ], 0, - "7f17483069ca497b807462f219cdef7b" + "4a3b5c5d3a3270bc8acc8c643622e0b1" ], [ "ValidatedParser.parse_one_entry", @@ -1991,7 +1991,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "81cc20f008a7e8d00cf055935cc5b899" + "59142d38ea4db654425ccd5349e92242" ], [ "ValidatedParser.fold_left_store_n_unfold1", @@ -2018,7 +2018,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "719025cd72886fea30e548b574574c4e" + "6abe090b411abd71a63619cbb2c780f4" ], [ "ValidatedParser.fold_left_buffer_n_mut_st", @@ -2069,7 +2069,7 @@ "typing_Slice.__proj__BSlice__item__p", "unit_typing" ], 0, - "e45430511b82c722a02356db4affd62f" + "3e39f95f3943320ebea208b6a059e0aa" ], [ "ValidatedParser.fold_left_buffer_n_st", @@ -2096,7 +2096,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "9a54e6cddb8ddd3e4527f0d7d473feb9" + "03e1ad8e8f015ec5d8f34abec2a8a315" ], [ "ValidatedParser.fold_left_buffer_st", @@ -2123,7 +2123,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "92ba9cf7a3fd5efa08efb5bcaf9b2c9d" + "b80bf7c3757f08030f132c624a937983" ], [ "ValidatedParser.fold_left_n_count", @@ -2149,7 +2149,7 @@ "typing_FStar.List.Tot.Base.length", "typing_FStar.UInt32.v" ], 0, - "57bcbdbe1e2e20af72927cc39bc5938d" + "e5bc963b12dac7cf47f04b5b38aa8729" ], [ "ValidatedParser.count_entries_example", @@ -2180,7 +2180,7 @@ "typing_Slice.as_seq" ], 0, - "7b7fb6a424c820253143371716a6f1ae" + "e7f16ccba83e641b95c355ea5fcfe695" ], [ "ValidatedParser.count_entries_example'", @@ -2289,7 +2289,7 @@ "typing_Slice.__proj__BSlice__item__p", "typing_Slice.as_seq" ], 0, - "9debcd38879207a3654418040a19f970" + "bdc1b77652ca518ea6358069b4a39d41" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/Validator.fst.hints b/examples/kv_parsing/Validator.fst.hints index c851bcdeb52..4c02e8eed55 100644 --- a/examples/kv_parsing/Validator.fst.hints +++ b/examples/kv_parsing/Validator.fst.hints @@ -34,7 +34,7 @@ "typing_Validator_Tm_abs_97608c9ed219c04a162143d32175364e" ], 0, - "eeb860edf66d31ae8b033a19ec9fa53c" + "5218abab110d1b68de6a8798610c43bf" ], [ "Validator.validate_entry_st", @@ -60,7 +60,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "07913c01978d4ddf97ccf76a7ef187c1" + "2f17b73bdb7f3ded379f0b4894132281" ], [ "Validator.validate_entries_st", @@ -160,7 +160,7 @@ "unit_typing" ], 0, - "b0bb2d3c5b80d4bd12d0127e0a589ebc" + "9d247cdc4d75a90b4e55bf88b5a3a7b2" ], [ "Validator.validate_store_st", @@ -315,7 +315,7 @@ "typing_Slice.u32_add_overflows", "unit_typing" ], 0, - "52da54be480c1a1329c1c49f0e9ed910" + "faeeab084d7575a707c82945b8d22cc3" ], [ "Validator.validate_store_st", @@ -341,7 +341,7 @@ "typing_FStar.UInt32.v", "typing_Slice.__proj__BSlice__item__len" ], 0, - "89e82620eb3656acd30b6022d995136d" + "1e632bcdec199f0f4b5e09f525085572" ], [ "Validator.validate_entry_st", @@ -374,7 +374,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "ad15b3c0388ec2211ab38bad06a3c28d" + "ea0e5d09cf3cd29a717e5c1b646d5d05" ], [ "Validator.validate_entries_st", @@ -474,7 +474,7 @@ "unit_typing" ], 0, - "46c6ad1df6c8a8976d9ba8dfb1aaf3b7" + "b13f73304d7fabe05c8625008d7f5827" ], [ "Validator.validate_store_st", @@ -507,7 +507,7 @@ "typing_Slice.__proj__BSlice__item__p" ], 0, - "3998729f9c39aab68565ca53584e9340" + "7d815667dc33104f1deb0b79e23602ba" ] ] ] \ No newline at end of file diff --git a/examples/kv_parsing/VectorParsing.fst.hints b/examples/kv_parsing/VectorParsing.fst.hints index c023cb28c0d..885e86e68a8 100644 --- a/examples/kv_parsing/VectorParsing.fst.hints +++ b/examples/kv_parsing/VectorParsing.fst.hints @@ -30,7 +30,7 @@ "typing_FStar.UInt32.v" ], 0, - "beecdca50e85b83ed49ffc7c3755114d" + "78a1ab7c5d2177285e2415298c581a81" ], [ "VectorParsing.parse_elem_progress", @@ -46,7 +46,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option" ], 0, - "efc5caa2e530ab503b237b2c74a5475b" + "07e6cf897b4ccb2b9d70a03cb01b0dff" ], [ "VectorParsing.parse_elem_progress", @@ -91,7 +91,7 @@ "typing_FStar.UInt32.v", "typing_VectorParsing.enc_elem" ], 0, - "8b7147d5033f89dae9400bba95b93c3b" + "31fd9c0f4545579bbd6fbffb8e79a19b" ], [ "VectorParsing.parse_elem_enc_length", @@ -107,7 +107,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option" ], 0, - "5554e20e4848aaca1ff36c3c30efa942" + "13459be5e30d5f144419e200b885acc7" ], [ "VectorParsing.parse_elem_enc_length", @@ -151,7 +151,7 @@ "typing_FStar.UInt32.v" ], 0, - "85ca5cabfa81bb5f32bceeec916d42f7" + "83d6980f70feb2630d5149141997f923" ], [ "VectorParsing.vector_length", @@ -167,7 +167,7 @@ "typing_VectorParsing.enc_elem" ], 0, - "20bfeecfba6fe602ecdd6a1ecfd76641" + "123c5d87964ac18c8f242878db32195c" ], [ "VectorParsing.parse_vector_length_pre", @@ -234,7 +234,7 @@ "well-founded-ordering-on-nat" ], 0, - "25782b9a391d9c81f453ceb0fe9c2f0f" + "f6a315cb8733e4f6d12f453cb1f04ec2" ], [ "VectorParsing.parse_vector_length_pre", @@ -294,7 +294,7 @@ "typing_VectorParsing.vector_length", "well-founded-ordering-on-nat" ], 0, - "8764bb8096eab8c1e1fc04f1fe8bce46" + "58199c50b2a621bb61a91ca3476dfe58" ], [ "VectorParsing.parse_vector_length_pre_extend", @@ -333,7 +333,7 @@ "typing_FStar.UInt16.v", "typing_FStar.UInt32.v", "unit_typing" ], 0, - "3b2aa57de89ccf86c17316e2bdfefa63" + "03325410e910513d157c0a7499487f92" ], [ "VectorParsing.parse_vector_length", @@ -361,7 +361,7 @@ "typing_FStar.UInt16.v" ], 0, - "b51d9d053d90726c43257af0e6725be4" + "82ffcb17ed290776279ffaa9c3dff53b" ], [ "VectorParsing.parse_vector_length", @@ -389,7 +389,7 @@ "typing_FStar.UInt16.v" ], 0, - "f688372b0045c9e7ad39c591f0a0c516" + "bc16f8f932ac013889f870068bbff03d" ], [ "VectorParsing.parse_vector_length_0", @@ -447,7 +447,7 @@ "typing_Prims.pow2" ], 0, - "26abb859938ad670865dee7fc80beed5" + "b760426aa752a0a481049589f7c590f2" ], [ "VectorParsing.parse_vector_length_consumes_len", @@ -463,7 +463,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option" ], 0, - "ec6312a27f1a077cc8473044329a0958" + "23d981ca5cc905fdb361b80bc537939c" ], [ "VectorParsing.parse_vector_length_consumes_len", @@ -490,7 +490,7 @@ "typing_VectorParsing_Tm_abs_35e00340110bed3b45665770431bd2a7" ], 0, - "871e9907fa212e1d9f3a47338d5a0fcb" + "b15c29817f999fc9e0c510aaa14341e4" ], [ "VectorParsing.parse_vector", @@ -499,7 +499,7 @@ 1, [ "@query" ], 0, - "99410a1423a7d521dab4de41287acc27" + "d256cd12e3c62e1f928c7ac779658449" ], [ "VectorParsing.encode_vector_data", @@ -532,7 +532,7 @@ "subterm_ordering_Prims.Cons", "typing_VectorParsing.enc_elem" ], 0, - "a0a3d1cd7afa146afca5b9b10f8dfc62" + "e110be2fafdaabdf12c601039c1b3a40" ], [ "VectorParsing.encode_vector", @@ -553,7 +553,7 @@ "refinement_interpretation_VectorParsing_Tm_refine_cea800c3dcd3d2cc262663da42897ef4" ], 0, - "4546360fa3cc413c50460a0fd536747b" + "f6975baaafa9fc803ff7c6180ed93f92" ], [ "VectorParsing.do_while_readonly", @@ -666,7 +666,7 @@ "typing_FStar.UInt32.v" ], 0, - "efaf8c2773140769abea1bd82509991c" + "8f59931a513cec41df08e991ce8c1103" ], [ "VectorParsing.u16_bound", @@ -688,7 +688,7 @@ "typing_FStar.UInt16.v" ], 0, - "4fe21c54862cf8d13b651dfaf05c4bdc" + "d61ea272c34f5986bec53476b3042c7f" ], [ "VectorParsing.validate_vector_data", @@ -697,7 +697,7 @@ 1, [ "@query" ], 0, - "4a07369df45366164d6dcba78394f489" + "01f5c3a2972bfd0b83ff08d0fef63321" ], [ "VectorParsing.validate_vector_data", @@ -880,7 +880,7 @@ "typing_VectorParsing_Tm_abs_35e00340110bed3b45665770431bd2a7" ], 0, - "7c5a8a4d726aadcd3935f687040727e2" + "1dbd1a12d055a2abca974abefcef3bd2" ], [ "VectorParsing.parse_elem_enc", @@ -911,7 +911,7 @@ "typing_FStar.UInt32.v" ], 0, - "1853d204c25545885bced81762346403" + "f29bce7984eb4f18b6ca8b9b1c22aa3a" ], [ "VectorParsing.parse_elem_progress", @@ -927,7 +927,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option" ], 0, - "5792a6cd7e681502abf4e77341e4d94b" + "17589baf799298ba3ee978481188c7bc" ], [ "VectorParsing.parse_elem_enc_length", @@ -943,7 +943,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option" ], 0, - "2995d80f92e9a14eb763820ad521a9c8" + "bc06368317a1ba5bf2e5c1dd8f4b9ded" ], [ "VectorParsing.vector_length", @@ -959,7 +959,7 @@ "typing_VectorParsing.enc_elem" ], 0, - "88ba34153a7c607e003d9e32768fa0c0" + "71a133cc2b061d5d33f21b8a52c715f6" ], [ "VectorParsing.parse_vector_length_pre", @@ -1019,7 +1019,7 @@ "typing_VectorParsing.vector_length", "well-founded-ordering-on-nat" ], 0, - "c6f0312b0d16d58bd93743c27f0adf2e" + "2afada17708dca8e052244fed6afcf3a" ], [ "VectorParsing.parse_vector_length_pre_extend", @@ -1058,7 +1058,7 @@ "typing_FStar.UInt16.v", "typing_FStar.UInt32.v", "unit_typing" ], 0, - "11853bc46444577f22ed73f10be7ce93" + "1504c60475bdb2e398a83afced0bb6de" ], [ "VectorParsing.parse_vector_length", @@ -1087,7 +1087,7 @@ "typing_FStar.UInt16.v" ], 0, - "bca121ca93b74086a01214e405ef03e4" + "3c7e116d65f18a704bc12ae50f29f1a4" ], [ "VectorParsing.parse_vector_length", @@ -1096,7 +1096,7 @@ 1, [ "@query" ], 0, - "56baf574e5c0de6a62aad34f80c5a0a0" + "f1e6d372338af4e9ae6c04b21491d9fd" ], [ "VectorParsing.parse_vector_length_0", @@ -1125,7 +1125,7 @@ "typing_FStar.Seq.Base.length", "typing_Prims.pow2" ], 0, - "943acecd2c281063f3d07042deb3231d" + "9a16eeb7e5118c97e160d1e6a2efd185" ], [ "VectorParsing.parse_vector_length_consumes_len", @@ -1141,7 +1141,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option" ], 0, - "b265ce1841ff7326f10a8e93ca5d8197" + "36f4bd7eaba2faa8db4996d7c0d3e8c8" ], [ "VectorParsing.parse_vector", @@ -1150,7 +1150,7 @@ 1, [ "@query" ], 0, - "8148121cd3a71a43304e94366453e942" + "098b0fa0de3baf375705372cb0f47fb5" ], [ "VectorParsing.encode_vector_data", @@ -1183,7 +1183,7 @@ "subterm_ordering_Prims.Cons", "typing_VectorParsing.enc_elem" ], 0, - "feb3f33d33b29ae949e88198850bfe92" + "2ff405f5bcbc35ec9835bb03c8f6e4d3" ], [ "VectorParsing.encode_vector", @@ -1204,7 +1204,7 @@ "refinement_interpretation_VectorParsing_Tm_refine_cea800c3dcd3d2cc262663da42897ef4" ], 0, - "1f0d8dd566b9e13fbd17982f217f7f54" + "fe8a97ed3cb0c2099fa97b88af730caf" ], [ "VectorParsing.validate_vector_data", @@ -1387,7 +1387,7 @@ "typing_VectorParsing_Tm_abs_35e00340110bed3b45665770431bd2a7" ], 0, - "781aac81840e4371046d5dc4a3064f18" + "495873d872a379463b04feebe4a08a3b" ], [ "VectorParsing.validate_vector_data", @@ -1558,7 +1558,7 @@ "typing_VectorParsing_Tm_abs_35e00340110bed3b45665770431bd2a7" ], 0, - "7d7c4c043b635d85a48670dc7bb164f8" + "58aa6b8ca8e659d4ea324dc6e9d336cd" ] ] ] \ No newline at end of file diff --git a/examples/low-mitls-experiments/HSL.fst.hints b/examples/low-mitls-experiments/HSL.fst.hints index d37900f3390..b35e8e26d94 100755 --- a/examples/low-mitls-experiments/HSL.fst.hints +++ b/examples/low-mitls-experiments/HSL.fst.hints @@ -1,5 +1,5 @@ [ - "nkNt'ྷ6,< 6", + "E\u0014knw\u0001I}y\"", [ [ "HSL.__proj__Mk_state__item__buf", @@ -11,7 +11,7 @@ "projection_inverse_HSL.Mk_state_len" ], 0, - "7c40ed27ba332cd59bd916277c69ea46" + "a47110020df6f0116a0a60c0a247536c" ], [ "HSL.null_terminator_invariant_helper", @@ -46,7 +46,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "bdd4c511093f8c4cf500282f1ab74582" + "a3221b8e9ca13bfbfd8064eb0ce0f0f9" ], [ "HSL.null_terminator_invariant", @@ -63,7 +63,7 @@ "refinement_interpretation_HSL_Tm_refine_aefed7d75105bc0157d4fd7d934bf79f" ], 0, - "3e584605011ea5cca4ac8c760f6eb837" + "5ba340f24005de470fce94145e55eee9" ], [ "HSL.msgs_list_invariant_helper", @@ -102,7 +102,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "07c8b0ad316c6750d92a41443eafc985" + "14229dcbd89c70f191934c8e63deec87" ], [ "HSL.msgs_list_invariant", @@ -120,7 +120,7 @@ "refinement_interpretation_HSL_Tm_refine_aefed7d75105bc0157d4fd7d934bf79f" ], 0, - "63b3e27479737e6a46af414c8772c620" + "8e3e23cda5698bb86a42c21c1637a2d5" ], [ "HSL.hsl_invariant_predicate", @@ -129,7 +129,7 @@ 1, [ "@query" ], 0, - "9926fb50dc2a5924a75cdb54da7c9f01" + "cc3761dd252dcf3834c9cff3489bf9ab" ], [ "HSL.lemma_hsl_invariant_elim", @@ -138,7 +138,7 @@ 1, [ "@query", "equation_HSL.hsl_invariant" ], 0, - "7804fda7cf9fa073b299211f5bfef216" + "3ae01abd8eff46a380858383993e953c" ], [ "HSL.hsl_footprint", @@ -162,7 +162,7 @@ "true_interp" ], 0, - "87cc0cc788175c517f87e69ff1bdbc1d" + "6974ac7ca00c0213ea5faec52711f975" ], [ "HSL.lemma_frame_hsl_invariant", @@ -264,7 +264,7 @@ "typing_LowStar.Monotonic.Buffer.mgsub", "unit_typing" ], 0, - "747995f9d4a0108bb086a9c2efa60a39" + "1c4a5f39289fedf6df351de0431af231" ], [ "HSL.hsl_create", @@ -277,9 +277,10 @@ "@query", "FStar.Monotonic.HyperStack_pretyping_cd115f719b336f9a8366e4b68a41d001", "Prims_pretyping_ae567c2fb75be05905677af440075565", - "Prims_pretyping_f537159ed795b314b4e58c260361ae86", "b2t_def", - "bool_inversion", "bool_typing", "constructor_distinct_Prims.Nil", - "data_typing_intro_Prims.Nil@tok", + "Prims_pretyping_f537159ed795b314b4e58c260361ae86", + "assumption_Prims.HasEq_int", "b2t_def", "bool_inversion", + "bool_typing", "constructor_distinct_Prims.Nil", + "data_elim_HSL.Mk_state", "data_typing_intro_Prims.Nil@tok", "equation_FStar.Heap.trivial_preorder", "equation_FStar.HyperStack.ST.equal_stack_domains", "equation_FStar.HyperStack.ST.is_eternal_region", @@ -292,6 +293,7 @@ "equation_FStar.Monotonic.HyperStack.as_addr", "equation_FStar.Monotonic.HyperStack.contains", "equation_FStar.Monotonic.HyperStack.is_eternal_color", + "equation_FStar.Monotonic.HyperStack.is_eternal_region", "equation_FStar.Monotonic.HyperStack.is_stack_region", "equation_FStar.Monotonic.HyperStack.is_wf_with_ctr_and_tip", "equation_FStar.Monotonic.HyperStack.live_region", @@ -307,8 +309,9 @@ "equation_HSL.hsl_get_buf", "equation_HSL.hsl_get_len", "equation_HSL.hsl_get_msgs", "equation_HSL.hsl_get_p0", "equation_HSL.hsl_get_p1", "equation_HSL.hsl_invariant", - "equation_HSL.u32", "equation_LowStar.Monotonic.Buffer.length", - "equation_Prims.eqtype", "equation_Prims.nat", + "equation_HSL.u32", "equation_LowStar.Monotonic.Buffer.fresh_loc", + "equation_LowStar.Monotonic.Buffer.length", "equation_Prims.eqtype", + "equation_Prims.nat", "equation_with_fuel_FStar.List.Tot.Base.mem.fuel_instrumented", "function_token_typing_FStar.Monotonic.Heap.heap", "function_token_typing_FStar.Monotonic.HyperHeap.rid", @@ -317,6 +320,8 @@ "function_token_typing_FStar.UInt32.t", "function_token_typing_LowStar.Monotonic.Buffer.address_liveness_insensitive_locs", "function_token_typing_LowStar.Monotonic.Buffer.loc_none", + "function_token_typing_Prims.nat", + "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", "int_inversion", "int_typing", "kinding_FStar.Pervasives.Native.tuple2@tok", "kinding_Prims.list@tok", @@ -328,17 +333,28 @@ "lemma_FStar.Monotonic.Heap.lemma_sel_upd2", "lemma_FStar.Monotonic.Heap.lemma_unused_upd_modifies", "lemma_FStar.Monotonic.Heap.lemma_upd_contains", + "lemma_FStar.Monotonic.Heap.lemma_upd_contains_different_addr", "lemma_FStar.Monotonic.Heap.lemma_upd_unused", "lemma_FStar.Monotonic.HyperHeap.lemma_root_has_color_zero", "lemma_FStar.Monotonic.HyperStack.lemma_mk_mem__projectors", "lemma_FStar.Set.lemma_equal_elim", "lemma_FStar.UInt32.uv_inv", "lemma_FStar.UInt32.vu_inv", + "lemma_LowStar.Monotonic.Buffer.live_loc_not_unused_in", + "lemma_LowStar.Monotonic.Buffer.loc_disjoint_sym_", + "lemma_LowStar.Monotonic.Buffer.loc_includes_addresses_addresses_2", + "lemma_LowStar.Monotonic.Buffer.loc_includes_addresses_buffer_", "lemma_LowStar.Monotonic.Buffer.loc_includes_none", + "lemma_LowStar.Monotonic.Buffer.loc_includes_trans_backwards", "lemma_LowStar.Monotonic.Buffer.loc_union_loc_none_r", "lemma_LowStar.Monotonic.Buffer.modifies_inert_intro", "lemma_LowStar.Monotonic.Buffer.modifies_inert_liveness_insensitive_buffer_weak", + "lemma_LowStar.Monotonic.Buffer.modifies_inert_loc_unused_in", "lemma_LowStar.Monotonic.Buffer.modifies_ralloc_post", "lemma_LowStar.Monotonic.Buffer.modifies_trans", + "lemma_LowStar.Monotonic.Buffer.mreference_live_loc_not_unused_in", + "lemma_LowStar.Monotonic.Buffer.ralloc_post_fresh_loc", + "lemma_LowStar.Monotonic.Buffer.unused_in_loc_unused_in", + "lemma_LowStar.Monotonic.Buffer.unused_in_not_unused_in_disjoint_2", "primitive_Prims.op_AmpAmp", "primitive_Prims.op_GreaterThan", "primitive_Prims.op_LessThanOrEqual", "primitive_Prims.op_Subtraction", "proj_equation_HSL.Mk_state_buf", @@ -361,33 +377,41 @@ "refinement_interpretation_FStar.UInt32_Tm_refine_6c25b42778726de94cd4dac42edb4860", "refinement_interpretation_FStar.UInt32_Tm_refine_6c5b5bfca8736b34d6f700f752d1df10", "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", - "refinement_interpretation_HSL_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55", "refinement_interpretation_HSL_Tm_refine_601254ebe274211073b2024a11d02039", "refinement_interpretation_HSL_Tm_refine_c1c6870886a55f37f8da073b7f666e03", "refinement_interpretation_HSL_Tm_refine_c91c357d8b481b71bcfe70f0ece722d9", "refinement_interpretation_HSL_Tm_refine_f37754acdd4e0bc4b2335c40890a7b93", + "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_5162887c6054b4734f59cfb79dd5cf2f", + "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f", "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", + "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b", "typing_FStar.Heap.trivial_preorder", "typing_FStar.Map.contains", "typing_FStar.Map.domain", "typing_FStar.Map.sel", - "typing_FStar.Map.upd", "typing_FStar.Monotonic.Heap.contains", - "typing_FStar.Monotonic.Heap.upd", + "typing_FStar.Map.upd", "typing_FStar.Monotonic.Heap.addr_of", + "typing_FStar.Monotonic.Heap.contains", + "typing_FStar.Monotonic.Heap.sel", "typing_FStar.Monotonic.Heap.upd", "typing_FStar.Monotonic.HyperStack.as_ref", "typing_FStar.Monotonic.HyperStack.contains", "typing_FStar.Monotonic.HyperStack.get_hmap", "typing_FStar.Monotonic.HyperStack.get_rid_ctr", "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.Monotonic.HyperStack.sel", + "typing_FStar.Set.singleton", "typing_FStar.StrongExcludedMiddle.strong_excluded_middle", - "typing_FStar.UInt32.lte", "typing_FStar.UInt32.sub", - "typing_FStar.UInt32.uint_to_t", "typing_FStar.UInt32.v", - "typing_HSL.__proj__Mk_state__item__buf", "typing_HSL.hsl_get_msgs", - "typing_HSL.hsl_get_p0", "typing_HSL.hsl_get_p1", + "typing_FStar.UInt32.sub", "typing_FStar.UInt32.uint_to_t", + "typing_FStar.UInt32.v", "typing_HSL.__proj__Mk_state__item__buf", "typing_LowStar.Buffer.trivial_preorder", + "typing_LowStar.Monotonic.Buffer.as_addr", "typing_LowStar.Monotonic.Buffer.g_is_null", - "typing_LowStar.Monotonic.Buffer.len" + "typing_LowStar.Monotonic.Buffer.len", + "typing_LowStar.Monotonic.Buffer.loc_addresses", + "typing_LowStar.Monotonic.Buffer.loc_buffer", + "typing_LowStar.Monotonic.Buffer.loc_not_unused_in", + "typing_LowStar.Monotonic.Buffer.loc_union", + "typing_LowStar.Monotonic.Buffer.loc_unused_in" ], 0, - "e140c0083f3877176951466db8a5f85d" + "8ac30edb7990e05b06f049686a82b9cb" ], [ "HSL.aux_process", @@ -462,7 +486,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "29e48958fb545203fbcdd16ca7b4239e" + "4aeee72f98a4f6aac1d2a94ff5d6eb2a" ], [ "HSL.hsl_process", @@ -615,7 +639,7 @@ "typing_LowStar.Monotonic.Buffer.mgsub" ], 0, - "9899575c87fc3194b187d9ee7901da2a" + "f2a0f75536d3ed233caba21d61abc3de" ], [ "HSL.null_terminator_invariant_helper", @@ -650,7 +674,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "41468860aab387b415ee674a62bc5134" + "f033faf94fad703998b708265e45f1aa" ], [ "HSL.null_terminator_invariant", @@ -667,7 +691,7 @@ "refinement_interpretation_HSL_Tm_refine_aefed7d75105bc0157d4fd7d934bf79f" ], 0, - "68650fda5ce3c948c4dbe9258605d4e0" + "70cca90f1e8cb4a38fd538164ec5c287" ], [ "HSL.null_terminator_invariant", @@ -682,7 +706,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "5d2d157a0517d02b41744c0f91010b8e" + "9b778ed5da3f9355aaebb39b4d2dedd8" ], [ "HSL.msgs_list_invariant_helper", @@ -721,7 +745,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "c28abd3a5a2775798e5da7fe6ade89c4" + "258c1cd5c00b316ce364741dee5e0c5b" ], [ "HSL.msgs_list_invariant", @@ -739,7 +763,7 @@ "refinement_interpretation_HSL_Tm_refine_aefed7d75105bc0157d4fd7d934bf79f" ], 0, - "39886c9ebb7bf34a7285f18a8e79d17f" + "d20ee0120b876621e8731c7b02610c97" ], [ "HSL.msgs_list_invariant", @@ -754,7 +778,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "425bb96f91e6e0590891dfbbfb18ed95" + "92dc1e52c8ed23d6ebda2a21418a7d2b" ], [ "HSL.hsl_invariant_predicate", @@ -763,7 +787,7 @@ 1, [ "@query" ], 0, - "7711a3ce54fcbf4a3d6bd8adaae6f043" + "f3ee818f7c33f7f5c2ac07cad4c3d758" ], [ "HSL.hsl_footprint", @@ -787,7 +811,7 @@ "true_interp" ], 0, - "08f56038024a9795b17716283c633d5b" + "5e7518d3c729cdb06af2bc3a051b1813" ], [ "HSL.lemma_frame_hsl_invariant", @@ -800,7 +824,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "e90e1146f418ae5a58d6682d21c62602" + "a7f422c4223672ee0909241bfb3c4c91" ], [ "HSL.aux_process", @@ -845,7 +869,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "5981351c95d83c224ffbb9c39a7a7df3" + "c7d509e4f86304a668fbebe1d52bebe5" ] ] ] \ No newline at end of file diff --git a/examples/lowparse/LowParse.Bytes32.fst.hints b/examples/lowparse/LowParse.Bytes32.fst.hints index b7652dcd24f..b26cea3597e 100644 --- a/examples/lowparse/LowParse.Bytes32.fst.hints +++ b/examples/lowparse/LowParse.Bytes32.fst.hints @@ -25,7 +25,7 @@ "typing_FStar.Bytes.len", "typing_FStar.UInt32.v" ], 0, - "e5bfc08df976d1b008190396af0bc907" + "d591d934ff9be9795322dfcdf522ff3e" ], [ "LowParse.Bytes32.b32append", @@ -55,7 +55,7 @@ "typing_FStar.Seq.Base.length", "typing_FStar.UInt32.v" ], 0, - "d58702470f779a08cdb7af4d3e0e1266" + "aed3fdacc2ed4a6700e2c3b5ed8cebee" ], [ "LowParse.Bytes32.b32_index_reveal", @@ -83,7 +83,7 @@ "typing_FStar.UInt32.uint_to_t", "typing_FStar.UInt32.v" ], 0, - "d9001f1d66ec9ef33ccc9e14dea0e005" + "d92d3b164e15be09f29323cd34637ff1" ], [ "LowParse.Bytes32.b32_reveal_create", @@ -120,7 +120,7 @@ "typing_FStar.UInt32.v" ], 0, - "b1d74f6b21bf4c0555ede36d4698e087" + "9a96701005a9f5e62f0e96c2c7a972b1" ], [ "LowParse.Bytes32.reveal_empty", @@ -146,7 +146,7 @@ "typing_FStar.Bytes.reveal", "typing_FStar.Seq.Base.empty" ], 0, - "20b1b4c2f2004607dc3a98f87a7bb890" + "326edd59489edcf26f3cbfff9a2cef96" ], [ "LowParse.Bytes32.b32slice", @@ -172,7 +172,7 @@ "typing_FStar.Bytes.len", "typing_FStar.UInt32.v" ], 0, - "15c97b21ce8e34f0b32c76323d370c9f" + "68f5e2b5fd18772df5352fa2e8f0a00c" ], [ "LowParse.Bytes32.b32slice", @@ -193,7 +193,7 @@ "typing_FStar.UInt32.v" ], 0, - "9de0756086ec7e7e0cdf2a6ef1bf4616" + "ad03e4f80c40e34469df600445f52b32" ], [ "LowParse.Bytes32.b32append", @@ -226,7 +226,7 @@ "typing_FStar.Seq.Base.length", "typing_FStar.UInt32.v" ], 0, - "76dcb9f8af1b81a4e17af01002616f57" + "757230e91ae6c0f76fd61aecc7fd93ba" ], [ "LowParse.Bytes32.b32_index_reveal", @@ -235,7 +235,7 @@ 1, [ "@query", "lemma_FStar.Bytes.length_reveal" ], 0, - "d19a740ed5edd56c692371c4f712cff5" + "cf97a88fd79090cdcc6a81c62752cf07" ], [ "LowParse.Bytes32.b32_reveal_create", @@ -249,7 +249,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "698bc6154a4abc57c84f19a1c988995d" + "163af38e6c999f91ce3eb7182d4d3875" ] ] ] \ No newline at end of file diff --git a/examples/lowparse/LowParse.SLow.Base.fst.hints b/examples/lowparse/LowParse.SLow.Base.fst.hints index fe5a035ae73..24328530e86 100644 --- a/examples/lowparse/LowParse.SLow.Base.fst.hints +++ b/examples/lowparse/LowParse.SLow.Base.fst.hints @@ -21,7 +21,7 @@ "typing_LowParse.Spec.Base.consumed_length" ], 0, - "afe558a1784e83a8bb7ed3a083213721" + "20d298ef518de07361166039e8678fd9" ], [ "LowParse.SLow.Base.make_parser32", @@ -30,7 +30,7 @@ 1, [ "@query" ], 0, - "bdd291ce1572dc7b2d2b45611ea4cd9f" + "c955836fa7eb4b12de802cca10806deb" ], [ "LowParse.SLow.Base.coerce_parser32", @@ -42,7 +42,7 @@ "refinement_interpretation_LowParse.Spec.Base_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "7d3c7863cff74e007132d3d64d348f77" + "fdb0dec79798da955372d6cb732ec685" ], [ "LowParse.SLow.Base.validator_correct", @@ -64,7 +64,7 @@ "typing_LowParse.Spec.Base.consumed_length" ], 0, - "c8534834f81f694de50a90d2ebe12947" + "75bb57c7171cc01cf7d1425d03e8a090" ], [ "LowParse.SLow.Base.serializer32_then_parser32", @@ -112,7 +112,7 @@ "typing_FStar.Bytes.len", "typing_FStar.UInt32.v" ], 0, - "2ca3ceb7a2fae7b486119962509a184c" + "6668726304347dd8096a3e1b6276643a" ], [ "LowParse.SLow.Base.parser32_then_serializer32", @@ -174,7 +174,7 @@ "typing_LowParse.Spec.Base.parse", "unit_typing" ], 0, - "4bc47d848faaac1f8437e440156e8a90" + "fe9f359a63749fd09d5cc1e125271d51" ], [ "LowParse.SLow.Base.parser32_then_serializer32'", @@ -249,7 +249,7 @@ "typing_LowParse.Spec.Base.parse" ], 0, - "23a1c9b6d60ea2aaa4ee04aefdd314ad" + "7898dda1fffb9c1dcfe02b1a1a3e3f89" ], [ "LowParse.SLow.Base.parser32_injective", @@ -309,7 +309,7 @@ "typing_LowParse.Spec.Base.parse" ], 0, - "92d348bc62704d93a2103e4c5cc3d001" + "7b196acc2c8edb24332862d8b3888984" ], [ "LowParse.SLow.Base.serializer32_injective", @@ -335,7 +335,7 @@ "refinement_interpretation_LowParse.Spec.Base_Tm_refine_9fc4b705eaf2fe68d9cc8785e7df72bf" ], 0, - "6d79102f1c64c71a606dba2fbbb2732c" + "877a5c420dbeefcf9e7c6019dbe353f4" ], [ "LowParse.SLow.Base.parse32_size", @@ -368,7 +368,7 @@ "typing_FStar.Bytes.reveal" ], 0, - "c0270be23c48e1dce9d4d9f8a876ec77" + "5aa0275c0a3b2d3431338fca38e516e9" ], [ "LowParse.SLow.Base.parse32_total", @@ -401,7 +401,7 @@ "typing_FStar.Bytes.reveal" ], 0, - "ae317082ecca06e7580d66809e101fb1" + "a43b17f828548676234f0d3d4b16bc56" ], [ "LowParse.SLow.Base.u32_max", @@ -427,7 +427,7 @@ "typing_FStar.UInt32.v" ], 0, - "b2dc4572ecbc03e91c7a1a29281731d2" + "11f9cb2417d4369260636ec30796d82f" ], [ "LowParse.SLow.Base.add_overflow", @@ -455,7 +455,7 @@ "typing_FStar.UInt32.v", "typing_LowParse.SLow.Base.u32_max" ], 0, - "05f07f66bda766b3e7d4d363fcc3ca6a" + "67d7a0dbf4497851939b958d0d64fb5b" ], [ "LowParse.SLow.Base.size32_postcond", @@ -464,7 +464,7 @@ 1, [ "@query" ], 0, - "8df58f3c39ff28a0f5b0d084a927fa52" + "5c67a6e74dc1bbe7e803d3f01c699eda" ], [ "LowParse.SLow.Base.size32_constant_precond", @@ -473,7 +473,7 @@ 1, [ "@query" ], 0, - "9affca61af8224f28945f72515098eba" + "12d2f9c31013da7e6a4e6ed24983b3e1" ], [ "LowParse.SLow.Base.size32_constant", @@ -521,7 +521,7 @@ "typing_LowParse.Spec.Base.serialize" ], 0, - "faf1dc6111811daf921ed3fd882e1d38" + "e4b54021a548b18342083b90fd2b3d99" ], [ "LowParse.SLow.Base.parser32_correct", @@ -543,7 +543,7 @@ "typing_LowParse.Spec.Base.consumed_length" ], 0, - "722a0a0f85227626926e0439ddf62c90" + "5c3ee1f13edfdb30eb3f56ceba39917d" ], [ "LowParse.SLow.Base.make_parser32", @@ -552,7 +552,7 @@ 1, [ "@query" ], 0, - "10de43072a08093dc7c3ec6d562d5b73" + "15a2a32103e9c97089e09d8b6cbcd5f5" ], [ "LowParse.SLow.Base.coerce_parser32", @@ -564,7 +564,7 @@ "refinement_interpretation_LowParse.Spec.Base_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "f5f0fdbe6c7d10795e72ef73c87bf2bf" + "7366084fdd078034f3213a128791a716" ], [ "LowParse.SLow.Base.coerce_parser32", @@ -576,7 +576,7 @@ "refinement_interpretation_LowParse.Spec.Base_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "536d6df6c77dc79b8438814e7ed52642" + "5fa495c840b6ec89490d3bd41b997f3c" ], [ "LowParse.SLow.Base.validator_correct", @@ -598,7 +598,7 @@ "typing_LowParse.Spec.Base.consumed_length" ], 0, - "e73fdc586a17914a6299adeb3e8a02aa" + "628e0b6679f4fc1ad4f11a201477b67d" ], [ "LowParse.SLow.Base.parser32_then_serializer32", @@ -621,7 +621,7 @@ "typing_FStar.UInt32.v" ], 0, - "087da51947e010dfcf85bab06abf9c11" + "20e9e7fd65b05fb7ea4b0868677cc793" ], [ "LowParse.SLow.Base.parser32_then_serializer32'", @@ -637,7 +637,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "a3598cd328076f2a1c77351a17263d4c" + "ea5a437602bd904dcfffce94ce6e5993" ], [ "LowParse.SLow.Base.parser32_injective", @@ -661,7 +661,7 @@ "typing_FStar.UInt32.v", "unit_typing" ], 0, - "f76388720735c3124715c51e67978e17" + "3c5a63085770af962cef8595cb066038" ], [ "LowParse.SLow.Base.serializer32_injective", @@ -670,7 +670,7 @@ 1, [ "@query" ], 0, - "a32e032a347a67dd767e79cff281f23c" + "ccd0b3bdc87d61a6e7e038b56b9a2c43" ], [ "LowParse.SLow.Base.parse32_size", @@ -682,7 +682,7 @@ "equation_Prims.nat", "projection_inverse_BoxBool_proj_0" ], 0, - "5257325039d2811e24d1dc31dbf3e8a8" + "6190ab805a3128073d9ef04b5c1c1569" ], [ "LowParse.SLow.Base.u32_max", @@ -708,7 +708,7 @@ "typing_FStar.UInt32.v" ], 0, - "435bd7f5cf79e0589fdc2e46840384ce" + "2ec2a6e6dcef7cb051fa392871031b6e" ], [ "LowParse.SLow.Base.add_overflow", @@ -736,7 +736,7 @@ "typing_FStar.UInt32.v", "typing_LowParse.SLow.Base.u32_max" ], 0, - "39888b5d19ebce46d9a21d0561c569ce" + "e864ca70aa824e069aa72ac53cbd4c5c" ], [ "LowParse.SLow.Base.size32_postcond", @@ -745,7 +745,7 @@ 1, [ "@query" ], 0, - "ad851eed4cbc48449423d4db15c315ce" + "c12da9f4c1d372546e9eb338c133e865" ], [ "LowParse.SLow.Base.size32_constant_precond", @@ -754,7 +754,7 @@ 1, [ "@query" ], 0, - "72388239efc46b61165cac1f9c47132c" + "e285ae1e5e846d5bb2c5609128f31829" ], [ "LowParse.SLow.Base.size32_constant", @@ -802,7 +802,7 @@ "typing_LowParse.Spec.Base.serialize" ], 0, - "2b1140b2ee7f0758c68b903037b105d2" + "af8c4fb16dbc4069cd6fe3ea0fe9d178" ] ] ] \ No newline at end of file diff --git a/examples/lowparse/LowParse.SLow.Combinators.fst.hints b/examples/lowparse/LowParse.SLow.Combinators.fst.hints index 2bbce23d1a2..d3410764f2e 100644 --- a/examples/lowparse/LowParse.SLow.Combinators.fst.hints +++ b/examples/lowparse/LowParse.SLow.Combinators.fst.hints @@ -32,7 +32,7 @@ "typing_FStar.Bytes.len", "typing_FStar.UInt32.v" ], 0, - "a2e48004d0b1d081dae0cc221b76eeca" + "8a0f78865ff7489379b4b33c9965d42e" ], [ "LowParse.SLow.Combinators.parse32_and_then", @@ -146,7 +146,7 @@ "typing_LowParse.Spec.Combinators.and_then_bare", "unit_typing" ], 0, - "e5c1696bc03a230d639b951a6046fb89" + "0d5c0c0d6e1437f774918a026bcbb576" ], [ "LowParse.SLow.Combinators.parse32_nondep_then", @@ -154,7 +154,9 @@ 2, 1, [ - "@MaxIFuel_assumption", "@query", + "@MaxFuel_assumption", "@MaxIFuel_assumption", + "@fuel_correspondence_Prims.pow2.fuel_instrumented", + "@fuel_irrelevance_Prims.pow2.fuel_instrumented", "@query", "FStar.Pervasives.Native_pretyping_b53dbd183c526bc5d0f20d7b966ae125", "LowParse.SLow.Base_interpretation_Tm_arrow_5c70a976cd24289e06fb8048f00682b5", "LowParse.Spec.Combinators_interpretation_Tm_arrow_3e6aa714d1f2c3178c395f779a2d91c7", @@ -171,16 +173,15 @@ "data_elim_FStar.Pervasives.Native.Some", "disc_equation_FStar.Pervasives.Native.None", "disc_equation_FStar.Pervasives.Native.Some", "eq2-interp", - "equation_FStar.UInt.fits", "equation_FStar.UInt.lte", - "equation_FStar.UInt.max_int", "equation_FStar.UInt.min_int", - "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", - "equation_FStar.UInt32.lte", "equation_FStar.UInt32.n", - "equation_FStar.UInt32.n_minus_one", "equation_LowParse.Bytes.byte", - "equation_LowParse.Bytes.bytes", + "equation_FStar.Bytes.lbytes", "equation_FStar.UInt.fits", + "equation_FStar.UInt.lte", "equation_FStar.UInt.max_int", + "equation_FStar.UInt.min_int", "equation_FStar.UInt.size", + "equation_FStar.UInt.uint_t", "equation_FStar.UInt32.lte", + "equation_FStar.UInt32.n", "equation_FStar.UInt32.n_minus_one", + "equation_LowParse.Bytes.byte", "equation_LowParse.Bytes.bytes", "equation_LowParse.SLow.Base.bytes32", "equation_LowParse.SLow.Base.parser32_correct", "equation_LowParse.SLow.Base.u32_max", - "equation_LowParse.Spec.Base.bare_parser", "equation_LowParse.Spec.Base.consumed_length", "equation_LowParse.Spec.Base.is_total_constant_size_parser", "equation_LowParse.Spec.Base.parse", @@ -191,6 +192,7 @@ "equation_LowParse.Spec.Base.strong_parser_kind", "equation_LowParse.Spec.Combinators.and_then", "equation_LowParse.Spec.Combinators.and_then_bare", + "equation_LowParse.Spec.Combinators.and_then_kind", "equation_LowParse.Spec.Combinators.nondep_then", "equation_LowParse.Spec.Combinators.parse_empty", "equation_LowParse.Spec.Combinators.parse_ret_kind", @@ -199,6 +201,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.tuple2", "fuel_guarded_inversion_LowParse.Spec.Base.parser_kind_", "fuel_guarded_inversion_Prims.equals", + "function_token_typing_FStar.Bytes.empty_bytes", "function_token_typing_FStar.UInt32.n", "function_token_typing_FStar.UInt32.n_minus_one", "function_token_typing_FStar.UInt32.t", @@ -216,6 +219,7 @@ "lemma_FStar.Bytes.length_reveal", "lemma_FStar.Pervasives.invertOption", "lemma_FStar.Seq.Base.lemma_len_slice", + "lemma_FStar.UInt.pow2_values", "lemma_FStar.UInt32.vu_inv", "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", "primitive_Prims.op_LessThan", "primitive_Prims.op_LessThanOrEqual", "primitive_Prims.op_Subtraction", @@ -235,6 +239,7 @@ "projection_inverse_LowParse.Spec.Base.Mkparser_kind__parser_kind_low", "projection_inverse_LowParse.Spec.Base.Mkparser_kind__parser_kind_metadata", "projection_inverse_LowParse.Spec.Base.Mkparser_kind_metadata_t_parser_kind_metadata_total", + "refinement_interpretation_FStar.Bytes_Tm_refine_b0383769854f2b8d05d9f8fb03a8cbd4", "refinement_interpretation_FStar.Pervasives.Native_Tm_refine_4d5241eb6fe198666a8101195bbd4a2a", "refinement_interpretation_FStar.Seq.Base_Tm_refine_aebc5aa9049e78f605051015a3436e68", "refinement_interpretation_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b", @@ -252,16 +257,15 @@ "typing_FStar.Bytes.len", "typing_FStar.Bytes.reveal", "typing_FStar.Pervasives.Native.__proj__Some__item__v", "typing_FStar.Seq.Base.length", "typing_FStar.Seq.Base.slice", - "typing_FStar.UInt32.v", "typing_LowParse.SLow.Base.u32_max", - "typing_LowParse.Spec.Base.consumed_length", + "typing_FStar.UInt32.v", "typing_LowParse.Spec.Base.consumed_length", "typing_LowParse.Spec.Base.parse", "typing_LowParse.Spec.Combinators.and_then_bare", - "typing_LowParse.Spec.Combinators_Tm_abs_4e8e6588059dcad2a8065b9aa7d0c70d", + "typing_LowParse.Spec.Combinators.nondep_then", "typing_LowParse.Spec.Combinators_Tm_abs_90c48bde0bc5df4667ae567fdeb3dca2", "unit_typing" ], 0, - "d869b8ec6faed3a8551389e27f278237" + "821657e085d66f41ea620e2d115757f7" ], [ "LowParse.SLow.Combinators.serialize32_kind_precond", @@ -270,7 +274,7 @@ 1, [ "@query" ], 0, - "87c58edfbc7b80c5727782cb2abe3434" + "6b202bed768916eb41d393eadaec8976" ], [ "LowParse.SLow.Combinators.serialize32_nondep_then", @@ -351,7 +355,7 @@ "typing_FStar.UInt.fits", "unit_inversion", "unit_typing" ], 0, - "45e3f722d21539ff701e3fd4a12aa691" + "e7cce29d33254d64309b242defb1dd87" ], [ "LowParse.SLow.Combinators.parse32_strengthen", @@ -430,7 +434,7 @@ "typing_LowParse.Spec.Base.parse", "unit_typing" ], 0, - "bda3e80abc06061e976205020ea573ad" + "2cd610197643b1dbc3b71d43ab50089d" ], [ "LowParse.SLow.Combinators.parse32_synth", @@ -520,7 +524,7 @@ "typing_LowParse.Spec.Combinators.parse_synth", "unit_typing" ], 0, - "3378d03488d86ddccee3de49a9f9485d" + "c5b0aaacbcc6653d55c34fb9a0769616" ], [ "LowParse.SLow.Combinators.serialize32_synth", @@ -545,7 +549,7 @@ "refinement_interpretation_LowParse.Spec.Combinators_Tm_refine_771453e5024aef25c5affda17b912259" ], 0, - "71fd36aa25819e25d54e8a980c112732" + "f3067adaf661ce2969e90eaa8579324e" ], [ "LowParse.SLow.Combinators.parse32_filter", @@ -655,7 +659,7 @@ "typing_LowParse.Spec.Combinators.and_then_bare", "unit_typing" ], 0, - "1b05e68ee77b1cd164400de558058077" + "d5ef364450a5f487d5c828de48517d8d" ], [ "LowParse.SLow.Combinators.serialize32_filter", @@ -712,7 +716,7 @@ "typing_LowParse.Spec.Combinators.serialize_filter" ], 0, - "8225a4554daf4a6aab5a88ac9e0a07f0" + "e768c2faf616b4c0b87f7008601c10c1" ], [ "LowParse.SLow.Combinators.make_constant_size_parser32", @@ -771,7 +775,7 @@ "typing_FStar.UInt32.v" ], 0, - "cdb2a9fa7f8d949ed1ab283861928ae6" + "f9ad3fc3c12e86e56920291179b12211" ], [ "LowParse.SLow.Combinators.make_constant_size_parser32", @@ -830,7 +834,7 @@ "typing_FStar.UInt32.v" ], 0, - "2a551e14ab030cee62a9ccbc25dee228" + "416ee76fa91c3a80d4a690a24264a8f4" ], [ "LowParse.SLow.Combinators.make_total_constant_size_parser32", @@ -911,7 +915,7 @@ "typing_LowParse.Spec.Combinators_Tm_abs_18d69f26728d2f40351341008fd21e4e" ], 0, - "88a6082b0619f1a6340ea2f3dcf5d2a8" + "27382380579d5bd0574b92be7b5a1546" ], [ "LowParse.SLow.Combinators.make_total_constant_size_parser32", @@ -992,7 +996,7 @@ "typing_LowParse.Spec.Combinators_Tm_abs_18d69f26728d2f40351341008fd21e4e" ], 0, - "2e746db1c493532464fb21f52601d1f0" + "30fc48af9220cc809f5a952c97328abf" ], [ "LowParse.SLow.Combinators.size32_nondep_then", @@ -1074,7 +1078,7 @@ "typing_LowParse.SLow.Base.u32_max", "unit_typing" ], 0, - "2b0760f765894fb064f6972bf1ba8148" + "4a00513b4bd52efa077f54a5d4d8330b" ], [ "LowParse.SLow.Combinators.size32_filter", @@ -1090,7 +1094,7 @@ "equation_LowParse.Spec.Combinators.serialize_filter_" ], 0, - "5b691dc0fc2316bcadde5d2724eed1f3" + "55358addb45f052a5c8fd547c79cba30" ], [ "LowParse.SLow.Combinators.size32_synth", @@ -1115,7 +1119,7 @@ "refinement_interpretation_LowParse.Spec.Combinators_Tm_refine_771453e5024aef25c5affda17b912259" ], 0, - "2ad78e0a34350a344c55254b05bbfc61" + "fec833dd27ddc371afea426f0734c40a" ], [ "LowParse.SLow.Combinators.parse32_ret", @@ -1148,7 +1152,7 @@ "typing_FStar.Bytes.len", "typing_FStar.UInt32.v" ], 0, - "5a5e45a2fc012d71ffff4fb1355c7637" + "876114e203910a822977509c273b1eb9" ], [ "LowParse.SLow.Combinators.parse32_ret", @@ -1234,7 +1238,7 @@ "unit_typing" ], 0, - "52d80ef24fe08105486595be7b902ef6" + "34c07ea1004389af51677dfbcad246de" ], [ "LowParse.SLow.Combinators.parse32_and_then", @@ -1348,7 +1352,7 @@ "typing_LowParse.Spec.Combinators.and_then_bare", "unit_typing" ], 0, - "e7b22331bd9e6cd2e677bbf89e44d396" + "644d4322b83b7a33b07e96916624c2d9" ], [ "LowParse.SLow.Combinators.parse32_and_then", @@ -1360,7 +1364,7 @@ "refinement_interpretation_LowParse.SLow.Combinators_Tm_refine_61debf8ac78ef71c0a578e2b599ea757" ], 0, - "6f05de25edafcb117f00e82c0abe4984" + "7daa13897881dd6daf18e3b4cf83de74" ], [ "LowParse.SLow.Combinators.parse32_nondep_then", @@ -1368,7 +1372,9 @@ 2, 1, [ - "@MaxIFuel_assumption", "@query", + "@MaxFuel_assumption", "@MaxIFuel_assumption", + "@fuel_correspondence_Prims.pow2.fuel_instrumented", + "@fuel_irrelevance_Prims.pow2.fuel_instrumented", "@query", "FStar.Pervasives.Native_pretyping_b53dbd183c526bc5d0f20d7b966ae125", "LowParse.SLow.Base_interpretation_Tm_arrow_5c70a976cd24289e06fb8048f00682b5", "LowParse.Spec.Combinators_interpretation_Tm_arrow_3e6aa714d1f2c3178c395f779a2d91c7", @@ -1385,16 +1391,15 @@ "data_elim_FStar.Pervasives.Native.Some", "disc_equation_FStar.Pervasives.Native.None", "disc_equation_FStar.Pervasives.Native.Some", "eq2-interp", - "equation_FStar.UInt.fits", "equation_FStar.UInt.lte", - "equation_FStar.UInt.max_int", "equation_FStar.UInt.min_int", - "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", - "equation_FStar.UInt32.lte", "equation_FStar.UInt32.n", - "equation_FStar.UInt32.n_minus_one", "equation_LowParse.Bytes.byte", - "equation_LowParse.Bytes.bytes", + "equation_FStar.Bytes.lbytes", "equation_FStar.UInt.fits", + "equation_FStar.UInt.lte", "equation_FStar.UInt.max_int", + "equation_FStar.UInt.min_int", "equation_FStar.UInt.size", + "equation_FStar.UInt.uint_t", "equation_FStar.UInt32.lte", + "equation_FStar.UInt32.n", "equation_FStar.UInt32.n_minus_one", + "equation_LowParse.Bytes.byte", "equation_LowParse.Bytes.bytes", "equation_LowParse.SLow.Base.bytes32", "equation_LowParse.SLow.Base.parser32_correct", "equation_LowParse.SLow.Base.u32_max", - "equation_LowParse.Spec.Base.bare_parser", "equation_LowParse.Spec.Base.consumed_length", "equation_LowParse.Spec.Base.is_total_constant_size_parser", "equation_LowParse.Spec.Base.parse", @@ -1405,6 +1410,7 @@ "equation_LowParse.Spec.Base.strong_parser_kind", "equation_LowParse.Spec.Combinators.and_then", "equation_LowParse.Spec.Combinators.and_then_bare", + "equation_LowParse.Spec.Combinators.and_then_kind", "equation_LowParse.Spec.Combinators.nondep_then", "equation_LowParse.Spec.Combinators.parse_empty", "equation_LowParse.Spec.Combinators.parse_ret_kind", @@ -1413,6 +1419,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.tuple2", "fuel_guarded_inversion_LowParse.Spec.Base.parser_kind_", "fuel_guarded_inversion_Prims.equals", + "function_token_typing_FStar.Bytes.empty_bytes", "function_token_typing_FStar.UInt32.n", "function_token_typing_FStar.UInt32.n_minus_one", "function_token_typing_FStar.UInt32.t", @@ -1430,6 +1437,7 @@ "lemma_FStar.Bytes.length_reveal", "lemma_FStar.Pervasives.invertOption", "lemma_FStar.Seq.Base.lemma_len_slice", + "lemma_FStar.UInt.pow2_values", "lemma_FStar.UInt32.vu_inv", "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", "primitive_Prims.op_LessThan", "primitive_Prims.op_LessThanOrEqual", "primitive_Prims.op_Subtraction", @@ -1449,6 +1457,7 @@ "projection_inverse_LowParse.Spec.Base.Mkparser_kind__parser_kind_low", "projection_inverse_LowParse.Spec.Base.Mkparser_kind__parser_kind_metadata", "projection_inverse_LowParse.Spec.Base.Mkparser_kind_metadata_t_parser_kind_metadata_total", + "refinement_interpretation_FStar.Bytes_Tm_refine_b0383769854f2b8d05d9f8fb03a8cbd4", "refinement_interpretation_FStar.Pervasives.Native_Tm_refine_4d5241eb6fe198666a8101195bbd4a2a", "refinement_interpretation_FStar.Seq.Base_Tm_refine_aebc5aa9049e78f605051015a3436e68", "refinement_interpretation_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b", @@ -1466,16 +1475,15 @@ "typing_FStar.Bytes.len", "typing_FStar.Bytes.reveal", "typing_FStar.Pervasives.Native.__proj__Some__item__v", "typing_FStar.Seq.Base.length", "typing_FStar.Seq.Base.slice", - "typing_FStar.UInt32.v", "typing_LowParse.SLow.Base.u32_max", - "typing_LowParse.Spec.Base.consumed_length", + "typing_FStar.UInt32.v", "typing_LowParse.Spec.Base.consumed_length", "typing_LowParse.Spec.Base.parse", "typing_LowParse.Spec.Combinators.and_then_bare", - "typing_LowParse.Spec.Combinators_Tm_abs_4e8e6588059dcad2a8065b9aa7d0c70d", + "typing_LowParse.Spec.Combinators.nondep_then", "typing_LowParse.Spec.Combinators_Tm_abs_90c48bde0bc5df4667ae567fdeb3dca2", "unit_typing" ], 0, - "e6ebd1fb41c12404b96f1ebfd0ce3659" + "87638018e5cf00c52fd2c86994badec8" ], [ "LowParse.SLow.Combinators.serialize32_kind_precond", @@ -1484,7 +1492,7 @@ 1, [ "@query" ], 0, - "8ef43d3613df7cc5d9e5e68072d90d31" + "755a883cb9aeefd88e1061a7179b749f" ], [ "LowParse.SLow.Combinators.serialize32_nondep_then", @@ -1565,7 +1573,7 @@ "typing_FStar.UInt.fits", "unit_inversion", "unit_typing" ], 0, - "0f488d8c5519a9ba6597d9f90189b6ae" + "f3d260d6d9ee22a69afaa21ee65bdcb3" ], [ "LowParse.SLow.Combinators.parse32_strengthen", @@ -1644,7 +1652,7 @@ "typing_LowParse.Spec.Base.parse", "unit_typing" ], 0, - "6cbfd1528165c57e48071bd8a6470603" + "c5bd6c4f74fbb31d30194f6df41452b8" ], [ "LowParse.SLow.Combinators.parse32_synth", @@ -1734,7 +1742,7 @@ "typing_LowParse.Spec.Combinators.parse_synth", "unit_typing" ], 0, - "8d06ff0b5d6f766331a45ce6f5a69569" + "b88c01af994da77b137fb220302d461b" ], [ "LowParse.SLow.Combinators.parse32_synth", @@ -1746,7 +1754,7 @@ "refinement_interpretation_LowParse.SLow.Combinators_Tm_refine_d80f4f7d17573d0ef7f44270bf22754e" ], 0, - "4764a6a64c8a23e82fe62cb8a13ff59b" + "35d409dad592f2018d6f96f1a020b043" ], [ "LowParse.SLow.Combinators.serialize32_synth", @@ -1771,7 +1779,7 @@ "refinement_interpretation_LowParse.Spec.Combinators_Tm_refine_771453e5024aef25c5affda17b912259" ], 0, - "a8786ccabf2ceb58dd60550b141fed98" + "ca5f9f719e1b96d2d65bf3e57cfa7680" ], [ "LowParse.SLow.Combinators.serialize32_synth", @@ -1783,7 +1791,7 @@ "refinement_interpretation_LowParse.Spec.Combinators_Tm_refine_771453e5024aef25c5affda17b912259" ], 0, - "58f8d919fb6933689231ad9407983965" + "f908e8840c96ab3bbde2a1582cfdbbca" ], [ "LowParse.SLow.Combinators.parse32_filter", @@ -1895,7 +1903,7 @@ "unit_typing" ], 0, - "470e42a0a7381c90832080a20a9770cb" + "25aceb8b6964ec1e3fc0b52d56eb5efa" ], [ "LowParse.SLow.Combinators.serialize32_filter", @@ -1908,7 +1916,7 @@ "equation_LowParse.Spec.Combinators.serialize_filter_" ], 0, - "835fd1c2bfe38a3a972496fcc523985e" + "c406d89062e05fb383b6e1819c98a9dc" ], [ "LowParse.SLow.Combinators.make_constant_size_parser32", @@ -1925,7 +1933,7 @@ "unit_typing" ], 0, - "a0254c74cfc4b369194eff52d107fce5" + "6c52a7d099d5fa117674c4881e4cb0d5" ], [ "LowParse.SLow.Combinators.make_constant_size_parser32", @@ -1984,7 +1992,7 @@ "typing_FStar.UInt32.v" ], 0, - "9d02d49e1215d496e0fb2807568980d5" + "2a82c80eaf6bc4f76076bf55de7cf7d8" ], [ "LowParse.SLow.Combinators.make_constant_size_parser32", @@ -2001,7 +2009,7 @@ "unit_typing" ], 0, - "61d34df052ced4a317d8949b24579b87" + "cf4a8ebbe4e6040a17755f856bddb9fb" ], [ "LowParse.SLow.Combinators.make_total_constant_size_parser32", @@ -2018,7 +2026,7 @@ "unit_typing" ], 0, - "26a48b3624a0abd19663529ba25a6e0b" + "bd35de5fc2f1114366c26791e4fa9af6" ], [ "LowParse.SLow.Combinators.make_total_constant_size_parser32", @@ -2099,7 +2107,7 @@ "typing_LowParse.Spec.Combinators_Tm_abs_18d69f26728d2f40351341008fd21e4e" ], 0, - "fd06eaab2dec7cc690de14406351f564" + "685146b9b431be7ab1dab56d089ebf01" ], [ "LowParse.SLow.Combinators.make_total_constant_size_parser32", @@ -2116,7 +2124,7 @@ "unit_typing" ], 0, - "1054d5018d8c964345fc29488792208a" + "889b6f78753b9f221a8a9fdbd2e9a78d" ], [ "LowParse.SLow.Combinators.size32_nondep_then", @@ -2198,7 +2206,7 @@ "typing_LowParse.SLow.Base.u32_max", "unit_typing" ], 0, - "808c957848fd5ec2b253205aa3b37f7e" + "ad82d88a489c360e369a9a5282a61ecd" ], [ "LowParse.SLow.Combinators.size32_filter", @@ -2214,7 +2222,7 @@ "equation_LowParse.Spec.Combinators.serialize_filter_" ], 0, - "7c71cb6f607a1b1cf54588e376966045" + "3509e2c7c4eb6fefb0c29c469083634d" ], [ "LowParse.SLow.Combinators.size32_synth", @@ -2239,7 +2247,7 @@ "refinement_interpretation_LowParse.Spec.Combinators_Tm_refine_771453e5024aef25c5affda17b912259" ], 0, - "e2a59d57836fdabe979d52cf42a1fa0c" + "49e75f98797d1f34202196f78374958b" ], [ "LowParse.SLow.Combinators.size32_synth", @@ -2251,7 +2259,7 @@ "refinement_interpretation_LowParse.Spec.Combinators_Tm_refine_771453e5024aef25c5affda17b912259" ], 0, - "68e0f23ff9531c40336f07cf46445006" + "24e9d0aa3b83e0cf9106cef59272c4a5" ] ] ] \ No newline at end of file diff --git a/examples/lowparse/LowParse.SLow.Enum.fst.hints b/examples/lowparse/LowParse.SLow.Enum.fst.hints index 5c5fc2a1049..6e7af14e833 100644 --- a/examples/lowparse/LowParse.SLow.Enum.fst.hints +++ b/examples/lowparse/LowParse.SLow.Enum.fst.hints @@ -39,7 +39,7 @@ "typing_LowParse.Spec.Enum.list_map", "typing_Prims.uu___is_Cons" ], 0, - "733c2b1ff77ccd3890e3091ad76792fb" + "cc8788c99ef82747b4f6dbba6dbc2f8a" ], [ "LowParse.SLow.Enum.maybe_enum_key_of_repr'_t_cons_nil", @@ -105,7 +105,7 @@ "typing_LowParse.Spec.Enum.list_map" ], 0, - "b8728892218b002bcb7f016b0723932a" + "f06828dc5b3970cac81a7fe099fd4fa1" ], [ "LowParse.SLow.Enum.maybe_enum_key_of_repr'_t_cons", @@ -192,7 +192,7 @@ "typing_LowParse.Spec.Enum.list_mem" ], 0, - "4b237c40318b0548c72ba35e9e6466ff" + "52c768d63e649321eaf6b52ad0a0aa6a" ], [ "LowParse.SLow.Enum.parse32_maybe_enum_key_gen", @@ -267,7 +267,7 @@ "typing_LowParse.Spec.Enum.list_map", "unit_typing" ], 0, - "7ccdd55fadd9b9581d824de6579edd59" + "16432d941fe6747d35395123e661e48d" ], [ "LowParse.SLow.Enum.parse32_maybe_enum_key_gen", @@ -344,7 +344,7 @@ "typing_LowParse.Spec.Enum.list_map", "unit_typing" ], 0, - "856ea85a07f6cb9dd217c5179b2ed71f" + "128c143dcaa933662f13ec66d68e51c5" ], [ "LowParse.SLow.Enum.parse32_enum_key_gen", @@ -452,7 +452,7 @@ "unit_typing" ], 0, - "cfc80fa6a0a3f38796b097215f71ba9a" + "3b114d97fe78762969e3d5cbaa905e20" ], [ "LowParse.SLow.Enum.parse32_enum_key_gen", @@ -591,7 +591,7 @@ "unit_typing" ], 0, - "b461a76b46c74ea708caec974094abd8" + "5157afafcad95cec702d56ef003aab77" ], [ "LowParse.SLow.Enum.serialize32_enum_key_gen", @@ -623,7 +623,7 @@ "typing_LowParse.Spec.Enum.enum_repr_of_key" ], 0, - "43be3728f2796ad4cad9c6662f1ce94a" + "bee4f05958a53a58119fa4753f5ddb6b" ], [ "LowParse.SLow.Enum.serialize32_enum_key_gen", @@ -655,7 +655,7 @@ "typing_LowParse.Spec.Enum.enum_repr_of_key" ], 0, - "19d3642627c89d90e9818f88de40f513" + "8e6a0b8619565e077ff7500a5ad434b1" ], [ "LowParse.SLow.Enum.enum_repr_of_key_cons", @@ -727,7 +727,7 @@ "typing_LowParse.Spec.Enum.list_mem" ], 0, - "83a83832c61f9e5f79abd07e7de5a23b" + "60c2792e9697180f43d22ba6a1fa9be3" ], [ "LowParse.SLow.Enum.enum_repr_of_key_cons_nil", @@ -791,7 +791,7 @@ "typing_LowParse.Spec.Enum.list_map" ], 0, - "3660c0f4e512c3deb31b9befc6f68549" + "586f406ecd65436da75463888a3c0a92" ], [ "LowParse.SLow.Enum.serialize32_maybe_enum_key_gen'", @@ -839,7 +839,7 @@ "token_correspondence_LowParse.Spec.Enum.repr_of_maybe_enum_key" ], 0, - "adf4a09f7149ea994cfee7a7a691e9e7" + "c6ccc1cf50ec84f7ff6f9edfed7a26d7" ], [ "LowParse.SLow.Enum.serialize32_maybe_enum_key_gen", @@ -851,7 +851,7 @@ "refinement_interpretation_LowParse.SLow.Enum_Tm_refine_b0a424bed641ec3dd9c337eaf8186a6f" ], 0, - "cec14891b37f366c7548ee92a24f7ee0" + "90ad04ece044ef00766e4f75287b2c40" ], [ "LowParse.SLow.Enum.serialize32_maybe_enum_key_gen", @@ -863,7 +863,7 @@ "refinement_interpretation_LowParse.SLow.Enum_Tm_refine_b0a424bed641ec3dd9c337eaf8186a6f" ], 0, - "c7ebb7683cb19099970e8eeeac090bd4" + "23838da7dd8a8d95d2ef5012fbce87bd" ], [ "LowParse.SLow.Enum.enum_tail'", @@ -903,7 +903,7 @@ "typing_LowParse.Spec.Enum.list_map", "typing_Prims.uu___is_Cons" ], 0, - "f3830902533f73d4624820b3f969a10e" + "07ce9ef2fbce5b55ffa7032b49791a46" ], [ "LowParse.SLow.Enum.enum_tail'", @@ -915,7 +915,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "8114882f003ecc01cde377b1a0af2364" + "a22182ae9ecd1716a3219acc64c7f166" ], [ "LowParse.SLow.Enum.maybe_enum_key_of_repr'_t_cons_nil", @@ -999,7 +999,7 @@ "unit_typing" ], 0, - "6fa923d8ac66fb9d954444431634dec5" + "6cd533f73817c47789e9bc773511c1b3" ], [ "LowParse.SLow.Enum.maybe_enum_key_of_repr'_t_cons", @@ -1107,7 +1107,7 @@ "typing_LowParse.Spec.Enum.list_mem", "unit_typing" ], 0, - "431ca62585efe35668cf3a7e71102eab" + "876a71c1d7a66939b961f4355efbbfa4" ], [ "LowParse.SLow.Enum.parse32_maybe_enum_key_gen", @@ -1116,7 +1116,7 @@ 1, [ "@query" ], 0, - "a9693c6604bf063487f35f044a44129f" + "e524f6a1fa00fd0eaabe184f7cd7e69d" ], [ "LowParse.SLow.Enum.parse32_maybe_enum_key_gen", @@ -1189,7 +1189,7 @@ "typing_LowParse.Spec.Enum.enum_key_of_repr", "unit_typing" ], 0, - "eefe014c378c4c7d1efa6f4e7e798992" + "a3763183e6562704afe896f5b80b12f2" ], [ "LowParse.SLow.Enum.parse32_maybe_enum_key_gen", @@ -1198,7 +1198,7 @@ 1, [ "@query" ], 0, - "60baf089165fed57091dc2de86b31f7e" + "1de68b447e403e0d258c79c66525ca42" ], [ "LowParse.SLow.Enum.parse32_enum_key_gen", @@ -1207,7 +1207,7 @@ 1, [ "@query" ], 0, - "3c360d985386016518cc1a0d7385ec3d" + "910dbe6504a4b5d739620e1d3c2f0818" ], [ "LowParse.SLow.Enum.parse32_enum_key_gen", @@ -1349,7 +1349,7 @@ "unit_typing" ], 0, - "02d08ad428020bff4e144783a8f0f6fd" + "895e3154b6eec7f355d21afa45b47e82" ], [ "LowParse.SLow.Enum.parse32_enum_key_gen", @@ -1358,7 +1358,7 @@ 1, [ "@query" ], 0, - "bbe7bc2996c2065e23c00b92c8e5f3bb" + "d8c320cb347ab10672a7cd88ee1d71ed" ], [ "LowParse.SLow.Enum.serialize32_enum_key_gen", @@ -1367,7 +1367,7 @@ 1, [ "@query" ], 0, - "9293ed5adf8db38437660088a74b19ac" + "321c41bb44bcde4b4a601a49c3cfa772" ], [ "LowParse.SLow.Enum.serialize32_enum_key_gen", @@ -1393,7 +1393,7 @@ "refinement_interpretation_LowParse.Spec.Base_Tm_refine_9fc4b705eaf2fe68d9cc8785e7df72bf" ], 0, - "e998f6bdad015602bc85cd830c3132e3" + "a7260fcfadcb259f1addeb337f615eb7" ], [ "LowParse.SLow.Enum.serialize32_enum_key_gen", @@ -1402,7 +1402,7 @@ 1, [ "@query" ], 0, - "c7315ad364fe4312ba6ef425e97f6afc" + "250e3fd1d945904453f7c9bdb84a6f72" ], [ "LowParse.SLow.Enum.enum_repr_of_key_cons", @@ -1471,7 +1471,7 @@ "typing_LowParse.Spec.Enum.list_mem" ], 0, - "e7272ba4ecaa0e6f9ca797b9797436ef" + "9904bc98213b9635e33bdcad28423e5b" ], [ "LowParse.SLow.Enum.enum_repr_of_key_cons_nil", @@ -1530,7 +1530,7 @@ "typing_LowParse.Spec.Enum.list_map", "typing_Prims.uu___is_Cons" ], 0, - "3716e8f477d3aeed19a5acf62bd8319e" + "f09623a97bf89f7b807ce4e7238c10f3" ], [ "LowParse.SLow.Enum.serialize32_maybe_enum_key_gen'", @@ -1578,7 +1578,7 @@ "token_correspondence_LowParse.Spec.Enum.repr_of_maybe_enum_key" ], 0, - "293797a8c2df01b379c39763744b0a54" + "0193de3ee03e67d124ad3facbada0c81" ], [ "LowParse.SLow.Enum.serialize32_maybe_enum_key_gen", @@ -1587,7 +1587,7 @@ 1, [ "@query" ], 0, - "46accf9678593f56812e013103eb009c" + "663342f24d96e5403e879eb46eab8796" ], [ "LowParse.SLow.Enum.serialize32_maybe_enum_key_gen", @@ -1599,7 +1599,7 @@ "refinement_interpretation_LowParse.SLow.Enum_Tm_refine_b0a424bed641ec3dd9c337eaf8186a6f" ], 0, - "c3dc496d4eb900fd77f217f2105f4d6e" + "09dd310d67392e8884f02055276b211e" ], [ "LowParse.SLow.Enum.serialize32_maybe_enum_key_gen", @@ -1608,7 +1608,7 @@ 1, [ "@query" ], 0, - "839479fbb1e08ad08a053e90d9f3f06e" + "534b5d2c4cb3127fb0a168f424b642c0" ] ] ] \ No newline at end of file diff --git a/examples/lowparse/LowParse.Spec.Base.fst.hints b/examples/lowparse/LowParse.Spec.Base.fst.hints index 54e173fd2cc..77612d042a4 100644 --- a/examples/lowparse/LowParse.Spec.Base.fst.hints +++ b/examples/lowparse/LowParse.Spec.Base.fst.hints @@ -735,7 +735,7 @@ "typing_LowParse.Spec.Base.glb" ], 0, - "0ad274551a00346d11b9a01f738afb55" + "b010e933cabf8e9ba00de0a84e0b2da8" ], [ "LowParse.Spec.Base.glb_list", @@ -1500,7 +1500,7 @@ "typing_LowParse.Spec.Base.glb" ], 0, - "afb32af4113c48093cd393be770c58b9" + "216c65563e5ecd5627198b79a4d638f5" ], [ "LowParse.Spec.Base.glb_list", diff --git a/examples/lowparse/LowParse.Spec.Enum.fst.hints b/examples/lowparse/LowParse.Spec.Enum.fst.hints index 94aa24cec87..289de8479e2 100644 --- a/examples/lowparse/LowParse.Spec.Enum.fst.hints +++ b/examples/lowparse/LowParse.Spec.Enum.fst.hints @@ -22,7 +22,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "2d841af01e39390fa7a3fcf8e2a33a73" + "2cf314ab849dbde4b1e2d9773b68f119" ], [ "LowParse.Spec.Enum.list_mem", @@ -47,12 +47,12 @@ "projection_inverse_Prims.Cons_a", "projection_inverse_Prims.Cons_hd", "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a", - "refinement_interpretation_LowParse.Spec.Enum_Tm_refine_3468e2eb91350ed83d7b2136c59e3798", + "refinement_interpretation_LowParse.Spec.Enum_Tm_refine_839819343c242573542ee6508ebe807e", "refinement_interpretation_LowParse.Spec.Enum_Tm_refine_ff9441126166844650678431ddb446e5", "subterm_ordering_Prims.Cons", "typing_LowParse.Spec.Enum.list_mem" ], 0, - "1b6f712257312aa18d3cbfe645819f13" + "5d24597c0f8cc927f058055f48fcd423" ], [ "LowParse.Spec.Enum.enum_key", @@ -1172,7 +1172,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "cb9d9e9aa17588d633785d7e2c18166e" + "c4bbbe79223d420be486e7b236f1bc32" ], [ "LowParse.Spec.Enum.list_mem", @@ -1197,12 +1197,12 @@ "projection_inverse_Prims.Cons_a", "projection_inverse_Prims.Cons_hd", "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a", - "refinement_interpretation_LowParse.Spec.Enum_Tm_refine_3468e2eb91350ed83d7b2136c59e3798", + "refinement_interpretation_LowParse.Spec.Enum_Tm_refine_839819343c242573542ee6508ebe807e", "refinement_interpretation_LowParse.Spec.Enum_Tm_refine_ff9441126166844650678431ddb446e5", "subterm_ordering_Prims.Cons", "typing_LowParse.Spec.Enum.list_mem" ], 0, - "e5eb5a2b6ddd042c329445b5a7e932bd" + "6aee6d1369c1ed241ed0eab7251048fe" ], [ "LowParse.Spec.Enum.enum_key", diff --git a/examples/metatheory/LambdaOmega.fst.hints b/examples/metatheory/LambdaOmega.fst.hints index a235a8ab8b9..07dc072e84e 100644 --- a/examples/metatheory/LambdaOmega.fst.hints +++ b/examples/metatheory/LambdaOmega.fst.hints @@ -280,7 +280,7 @@ 1, [ "@MaxIFuel_assumption", "@query", - "LambdaOmega_interpretation_Tm_arrow_751fe869631add8f687bcf59f04fd515", + "LambdaOmega_interpretation_Tm_arrow_e71cdb4badd9fd89e491b78924d10edb", "LambdaOmega_pretyping_1c3eda042f75cb90bd281a839e46e47d", "binder_x_1c3eda042f75cb90bd281a839e46e47d_1", "binder_x_72be33445e3cf5d60d578600fdf4ad4e_0", "bool_inversion", @@ -295,7 +295,7 @@ "projection_inverse_BoxInt_proj_0", "projection_inverse_LambdaOmega.EVar__0", "refinement_interpretation_LambdaOmega_Tm_refine_16db7d9e55ec639a8c277fda1d255e67", - "refinement_interpretation_LambdaOmega_Tm_refine_20dc41ca5f7e04c7cae172a3c9663edd", + "refinement_interpretation_LambdaOmega_Tm_refine_56f87b10480d8b793782e851a52853df", "refinement_interpretation_LambdaOmega_Tm_refine_e966d49e99bb259fb40f929bd1862f96", "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", "subterm_ordering_LambdaOmega.EApp", @@ -305,7 +305,7 @@ "typing_LambdaOmega.uu___is_EVar", "well-founded-ordering-on-nat" ], 0, - "89fb77f5eb4d3061148a0705635209a3" + "13992364788b9156b6617755fc500f2d" ], [ "LambdaOmega.esubst", @@ -333,7 +333,7 @@ "well-founded-ordering-on-nat" ], 0, - "7586be620140a0aba51fe9bc45f3f702" + "9352c5a387c4c32dd08f3ba28c060aaf" ], [ "LambdaOmega.esub_lam_renaming", @@ -507,7 +507,7 @@ "typing_LambdaOmega.uu___is_TVar", "well-founded-ordering-on-nat" ], 0, - "11622edb0bab38f694415b9dcdd34539" + "ec88d96a989402b18b5ab47e4648524e" ], [ "LambdaOmega.tsub_lam", @@ -719,7 +719,7 @@ "well-founded-ordering-on-nat" ], 0, - "b5c3117081960dfbca1761500f4349e5" + "a071fd57af77729b62c0d0b2746e0d3f" ], [ "LambdaOmega.tsub_lam_comp", @@ -2217,7 +2217,7 @@ "typing_LambdaOmega.is_value", "typing_LambdaOmega.uu___is_ELam" ], 0, - "cb96085b98d5bc61c2c4b4765eb630b0" + "56c5a4bd6561ced13c1dfe252a414e93" ], [ "LambdaOmega.tappears_free_in", @@ -2243,7 +2243,7 @@ "subterm_ordering_LambdaOmega.TLam" ], 0, - "8efbe4f3fd81bef39f1178e3a1d5cbdd" + "978bf10d65a07df730d6d9305d32156c" ], [ "LambdaOmega.envEqualT", @@ -2321,7 +2321,7 @@ "typing_tok_LambdaOmega.KTyp@tok" ], 0, - "2dfbb96c22649d94b8392f67b4076434" + "a4419339f1606f5049df4e55050bbd3b" ], [ "LambdaOmega.kinding_extensional", @@ -2372,7 +2372,7 @@ "typing_tok_LambdaOmega.KTyp@tok" ], 0, - "f98088f48fe4afb686f4408ec26e9c8c" + "f565f276aaf860a120b1ec16915916a0" ], [ "LambdaOmega.kinding_weakening_ebnd", @@ -2512,7 +2512,7 @@ "typing_tok_LambdaOmega.KTyp@tok" ], 0, - "2d85528c69110dd4cdcdbb58157e4be3" + "72c2c165ffbf912c97522c76b7ec3755" ], [ "LambdaOmega.kinding_strengthening_ebnd", @@ -2555,7 +2555,7 @@ "projection_inverse_LambdaOmega.TArr__1" ], 0, - "e4c1e31bdb94074b707742b9c4aa727d" + "ff7d629a082ffba074bdb3e25cc611ef" ], [ "LambdaOmega.typing_to_kinding", @@ -2578,7 +2578,7 @@ "subterm_ordering_LambdaOmega.TyLam" ], 0, - "e31a414e4928fe5ae4bacd5cf9dfa7f7" + "76eec32326be8fe07a6cd5a3edeec522" ], [ "LambdaOmega.tshift_up_above_tsubst_beta_aux", @@ -2713,7 +2713,7 @@ "subterm_ordering_LambdaOmega.EqTran" ], 0, - "09f6578a8ead4e6c88da419ee7943e3d" + "08f4cfcb77cb8e182d22e4166c58d0d9" ], [ "LambdaOmega.is_renaming", @@ -2856,7 +2856,7 @@ "typing_tok_LambdaOmega.KTyp@tok", "well-founded-ordering-on-nat" ], 0, - "526f8e9f17496f0e2b1e011a9ddcfaf6" + "1666f6a48f30b7665faeb78e7dccd1a2" ], [ "LambdaOmega.typing_substitution", @@ -2898,7 +2898,7 @@ "token_correspondence_LambdaOmega.esub_beta" ], 0, - "f64be7c621934d5341f5dd45c3d5f437" + "e9921339d5132d609b3d95b4c0a63ab1" ], [ "LambdaOmega.tsubst_gen_tlam_aux", @@ -3378,7 +3378,7 @@ "subterm_ordering_LambdaOmega.TrLam" ], 0, - "5cd46c94cf2c37e8e6b9214c5f040b54" + "e6203739a1287b86b1da21305333d9cc" ], [ "LambdaOmega.subst_of_tred", @@ -3422,7 +3422,7 @@ "subterm_ordering_LambdaOmega.TLam" ], 0, - "9f2ed99558ff9a7c6d72af7c989af8e0" + "101ed39eea871c64c6cfc9c004207d2a" ], [ "LambdaOmega.shift_above_and_subst", @@ -3604,7 +3604,7 @@ "subterm_ordering_LambdaOmega.TrLam" ], 0, - "070434ee285075a5d3f24d29286ad745" + "c35d67201bba60635a50e17687074fb7" ], [ "LambdaOmega.ltup", @@ -3715,7 +3715,7 @@ "subterm_ordering_LambdaOmega.TrLam" ], 0, - "c2ad2bf2e4cf54e6bff52c982b740043" + "b5c9bfecea6fa40a900def6e83fdc532" ], [ "LambdaOmega.tred_star", @@ -3830,7 +3830,7 @@ "subterm_ordering_LambdaOmega.TsStep" ], 0, - "1dd2b5a112ca88a5c48a182527e0c81e" + "11a7e3624c59d0b7ae0f46b017fb6e43" ], [ "LambdaOmega.confluence", @@ -3847,7 +3847,7 @@ "subterm_ordering_LambdaOmega.TsStep" ], 0, - "e272e5194092d43b94eae9f885c44e4c" + "06596e854f3992d9a367ba12d3003439" ], [ "LambdaOmega.ts_tran", @@ -3864,7 +3864,7 @@ "subterm_ordering_LambdaOmega.TsStep" ], 0, - "166258a1323122a5b55dbe195da71e8a" + "7395f5c3d0864a3736f5af1a30e665af" ], [ "LambdaOmega.tred_star_sym", @@ -4062,7 +4062,7 @@ "subterm_ordering_LambdaOmega.TssTran" ], 0, - "7bc6cd23c27639144a1f13ff670b49ba" + "d834631f0a9b2ff5c35a1bbb5794f8a0" ], [ "LambdaOmega.trlam_tss", @@ -4081,7 +4081,7 @@ "subterm_ordering_LambdaOmega.TssTran" ], 0, - "5f533a03911369b8841ccb9a51306f0c" + "4e085d6ea84877ca1d4f61e90ef3b667" ], [ "LambdaOmega.trapp_tss_1", @@ -4100,7 +4100,7 @@ "subterm_ordering_LambdaOmega.TssTran" ], 0, - "552afce93938065230a0aef5fb21534f" + "08022c94d6900bd1184d2b9aa596be3e" ], [ "LambdaOmega.trapp_tss_2", @@ -4119,7 +4119,7 @@ "subterm_ordering_LambdaOmega.TssTran" ], 0, - "ba149aaafb7b703bf73310a7f41ca297" + "9319e638d67dac34e5c793c025cde91f" ], [ "LambdaOmega.trarr_tss_1", @@ -4138,7 +4138,7 @@ "subterm_ordering_LambdaOmega.TssTran" ], 0, - "6cb9bb24387364321c1ca966fd3164fa" + "f4d05bb58ce30ebee6e64f8fa7978946" ], [ "LambdaOmega.trarr_tss_2", @@ -4157,7 +4157,7 @@ "subterm_ordering_LambdaOmega.TssTran" ], 0, - "93e0362e4894801e5cd90f22dad4ee27" + "3e760123510484a778f10763732837ca" ], [ "LambdaOmega.tequiv_tss", @@ -4185,7 +4185,7 @@ "subterm_ordering_LambdaOmega.EqTran" ], 0, - "a0b023c6f97594b1990cef9853e666eb" + "30736c2b8e00a90830d1c591fd6da19b" ], [ "LambdaOmega.tred_tequiv", @@ -4209,7 +4209,7 @@ "subterm_ordering_LambdaOmega.TrLam" ], 0, - "fd230f07704234f8b2ab7aa7f954a62f" + "d0eadc84300b368a243c6f96e923d4f2" ], [ "LambdaOmega.tred_star_tequiv", @@ -4226,7 +4226,7 @@ "subterm_ordering_LambdaOmega.TsStep" ], 0, - "568b254ea54448d511de4c1841e886f4" + "7762ba3c195a41d7a219dba99678ad30" ], [ "LambdaOmega.tss_tequiv", @@ -4245,7 +4245,7 @@ "subterm_ordering_LambdaOmega.TssTran" ], 0, - "07d0da6f4e4ba3b1eff14ff3bdcd6229" + "4ae39e2c89e25ea9ac070b603c8b2f2e" ], [ "LambdaOmega.tred_tarr_preserved", @@ -4287,7 +4287,7 @@ "subterm_ordering_LambdaOmega.TsStep" ], 0, - "e13198d4761b145d7cf3af114d4b4c8e" + "6ed2e0d0c5967cf59d95bd87275ff1c2" ], [ "LambdaOmega.inversion_elam", @@ -4323,7 +4323,7 @@ "subterm_ordering_LambdaOmega.TyEqu" ], 0, - "d65869d55722f03ca380ea43ead68153" + "80d3c9c0bfe9b385de16dd00128711df" ], [ "LambdaOmega.preservation", @@ -4355,7 +4355,7 @@ "subterm_ordering_LambdaOmega.TyEqu" ], 0, - "7cb9993ec1d8497b100125499ff623e5" + "9fc9e6f5615fd027f8e6da2259dba584" ], [ "LambdaOmega.knd", @@ -4621,7 +4621,7 @@ 1, [ "@MaxIFuel_assumption", "@query", - "LambdaOmega_interpretation_Tm_arrow_751fe869631add8f687bcf59f04fd515", + "LambdaOmega_interpretation_Tm_arrow_e71cdb4badd9fd89e491b78924d10edb", "LambdaOmega_pretyping_1c3eda042f75cb90bd281a839e46e47d", "binder_x_1c3eda042f75cb90bd281a839e46e47d_1", "binder_x_72be33445e3cf5d60d578600fdf4ad4e_0", "bool_inversion", @@ -4636,7 +4636,7 @@ "projection_inverse_BoxInt_proj_0", "projection_inverse_LambdaOmega.EVar__0", "refinement_interpretation_LambdaOmega_Tm_refine_16db7d9e55ec639a8c277fda1d255e67", - "refinement_interpretation_LambdaOmega_Tm_refine_20dc41ca5f7e04c7cae172a3c9663edd", + "refinement_interpretation_LambdaOmega_Tm_refine_56f87b10480d8b793782e851a52853df", "refinement_interpretation_LambdaOmega_Tm_refine_e966d49e99bb259fb40f929bd1862f96", "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", "subterm_ordering_LambdaOmega.EApp", @@ -4646,7 +4646,7 @@ "typing_LambdaOmega.uu___is_EVar", "well-founded-ordering-on-nat" ], 0, - "8f18ae5b626411c1e3dbe3aede7c17d9" + "4f02b08453f0bd9a4acd66c96bb5a6ea" ], [ "LambdaOmega.esubst", @@ -4674,7 +4674,7 @@ "well-founded-ordering-on-nat" ], 0, - "bbbd844dba2a4ae023d09837fff64fb3" + "14f7fb39d43dd62a0663d4fddd5e3ad6" ], [ "LambdaOmega.esubst_extensional", @@ -4787,7 +4787,7 @@ "typing_LambdaOmega.uu___is_TVar", "well-founded-ordering-on-nat" ], 0, - "ace4fd6b8ff06a2ec5d627092caec501" + "8a8d044a50a9d7914230f29206e61da7" ], [ "LambdaOmega.tsub_lam", @@ -6251,7 +6251,7 @@ "subterm_ordering_LambdaOmega.TLam" ], 0, - "e367fb6f651256be2a12f28ccf115e5a" + "ad531f81398b152a421dbccd01504e9b" ], [ "LambdaOmega.envEqualT", diff --git a/examples/metatheory/ParSubst.fst.hints b/examples/metatheory/ParSubst.fst.hints index 9b375fc8e19..eca99d2f4f2 100644 --- a/examples/metatheory/ParSubst.fst.hints +++ b/examples/metatheory/ParSubst.fst.hints @@ -172,7 +172,7 @@ "typing_ParSubst.uu___is_EVar", "well-founded-ordering-on-nat" ], 0, - "de58751770e4a9b0c6a6a6afbcca5a62" + "bf7ab64efa3499069ca2d8417e33b152" ], [ "ParSubst.subst_eabs", @@ -395,7 +395,7 @@ "typing_ParSubst.uu___is_EVar", "well-founded-ordering-on-nat" ], 0, - "be305b80a4d0cf447744b52e8574e0d3" + "e378281d969268cc302a153e63c90ad6" ], [ "ParSubst.subst_eabs", diff --git a/examples/metatheory/StackMachine.fst.hints b/examples/metatheory/StackMachine.fst.hints index a9be8d6db72..2e577d11b04 100644 --- a/examples/metatheory/StackMachine.fst.hints +++ b/examples/metatheory/StackMachine.fst.hints @@ -140,7 +140,7 @@ "subterm_ordering_StackMachine.Binop" ], 0, - "ae15a24f2a2058d3d015789950927489" + "3a03e6b0308120804b9b809541c073f0" ], [ "StackMachine.instr", @@ -218,7 +218,7 @@ "typing_StackMachine.instrDenote" ], 0, - "fa86edb3baf11eb9140915a6d4cb30e6" + "4109f92eb6466fd80d788d315303760a" ], [ "StackMachine.compile", @@ -234,7 +234,7 @@ "subterm_ordering_StackMachine.Binop" ], 0, - "2995b9315bb77306b2b0054b9295158d" + "c461ec2231e0b1c4a848cbc23f863530" ], [ "StackMachine.app_assoc_reverse", @@ -336,7 +336,7 @@ "unit_typing" ], 0, - "1cefd73f380086940db46b97a40b012d" + "7ab899bc4a974367ccf3335057865115" ], [ "StackMachine.app_nil_end", @@ -607,7 +607,7 @@ "subterm_ordering_StackMachine.TBinop" ], 0, - "1fd002093608ee0869ca77f49b2163c7" + "c3691c74d08ccc7792302dbccfd690d4" ], [ "StackMachine.tinstr", @@ -877,7 +877,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "720c03fa06f8125e305fd1a5cad87ade" + "b26c6d5708264fbbce8c57e19b561922" ], [ "StackMachine.tinstrDenote", @@ -924,7 +924,7 @@ "typing_StackMachine.vstack", "typing_tok_StackMachine.Nat@tok" ], 0, - "2ab535ae202df98e08784f797526e7c0" + "e3ce94021eea835aa44895595d971024" ], [ "StackMachine.tprogDenote", @@ -941,7 +941,7 @@ "subterm_ordering_StackMachine.TCons" ], 0, - "4c9a2e515a8ae0ec05119898c0285093" + "348952e334c374292a9092abde90e9ad" ], [ "StackMachine.tconcat", @@ -958,7 +958,7 @@ "subterm_ordering_StackMachine.TCons" ], 0, - "32beed91c75f7607b2b7960344cca9f2" + "f7a974afd4b62f052efb0e7ddebbde96" ], [ "StackMachine.tcompile", @@ -979,7 +979,7 @@ "subterm_ordering_StackMachine.TBinop" ], 0, - "0e155f8d892a96d05202d517fff6e299" + "733861a5f055602d7ecd85ea8e27dbfb" ], [ "StackMachine.tconcat_correct", @@ -1011,7 +1011,7 @@ "subterm_ordering_StackMachine.TCons" ], 0, - "7a7f8dfde87b4e6bc4c619517c328466" + "4ed9858303a5f18d6c7af9928e0d0ae1" ], [ "StackMachine.tcompile_correct'", @@ -1101,7 +1101,7 @@ "typing_StackMachine.vstack" ], 0, - "5c3bc678ffaac1e8f1c053badf9b1bce" + "ab679e49bd241b9362c3b1513370ee20" ], [ "StackMachine.exp", @@ -1242,7 +1242,7 @@ "subterm_ordering_StackMachine.Binop" ], 0, - "90612d9f6a92bab685168a824be9ee90" + "1bc9bad9fb321872218ccee1406affac" ], [ "StackMachine.instr", @@ -1320,7 +1320,7 @@ "typing_StackMachine.instrDenote" ], 0, - "feb16312598799b6263bda447bff8be8" + "380c73bae1d897437184fbed661f4d31" ], [ "StackMachine.compile", @@ -1336,7 +1336,7 @@ "subterm_ordering_StackMachine.Binop" ], 0, - "f6edfdf853af30056e549e62b28e91f9" + "2879bb8ec8daa757be4619a3cd6e23f6" ], [ "StackMachine.compile_correct'", @@ -1600,7 +1600,7 @@ "subterm_ordering_StackMachine.TBinop" ], 0, - "5df8caab4d28a438e1fe9df7d96bae2f" + "800e2a27086dee743e5e15c066b7d7dc" ], [ "StackMachine.tinstr", @@ -1870,7 +1870,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "6075b3ec38da98e1648ae9767d80d86d" + "dc9737cab79945ea6371eff45e474776" ], [ "StackMachine.tinstrDenote", @@ -1917,7 +1917,7 @@ "typing_StackMachine.vstack", "typing_tok_StackMachine.Nat@tok" ], 0, - "b53c77b7642abbd66573d4e196b15ac6" + "5a41cedbef0ea7d0cc171bd0b395f857" ], [ "StackMachine.tprogDenote", @@ -1934,7 +1934,7 @@ "subterm_ordering_StackMachine.TCons" ], 0, - "e361518809155a81641dca1fa7eafb6c" + "38b4998b88564e45eada94ff773f5a8d" ], [ "StackMachine.tconcat", @@ -1951,7 +1951,7 @@ "subterm_ordering_StackMachine.TCons" ], 0, - "37b3af104a18a430af7bd1a745a1b14f" + "43eb07b3c9b419d6ea1f2c686315d7f3" ], [ "StackMachine.tcompile", @@ -1972,7 +1972,7 @@ "subterm_ordering_StackMachine.TBinop" ], 0, - "5fd8353e7f6fb0870447b6e831e02c01" + "8436911af49f93938a38db75138153ea" ] ] ] \ No newline at end of file diff --git a/examples/metatheory/StlcCbvDbParSubst.fst.hints b/examples/metatheory/StlcCbvDbParSubst.fst.hints index a821d036b59..f6bf84b6038 100644 --- a/examples/metatheory/StlcCbvDbParSubst.fst.hints +++ b/examples/metatheory/StlcCbvDbParSubst.fst.hints @@ -65,7 +65,7 @@ "typing_StlcCbvDbParSubst.sub_inc_above" ], 0, - "b4e23028b1dae9d7c981b5a47a06482e" + "b953547ae9210cfd412461597c89d626" ], [ "StlcCbvDbParSubst.step", @@ -86,7 +86,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "937c4c935f5ab964d0d81a2c0facdfb7" + "c4ef967d4289473c080b69dc08ed6a90" ], [ "StlcCbvDbParSubst.progress", @@ -206,7 +206,7 @@ "subterm_ordering_StlcStrongDbParSubst.ELam" ], 0, - "356b9419cb9f69a67bfe3a6bdcfdf416" + "e68e300a7d82d8fb6a163c8b7986540d" ], [ "StlcCbvDbParSubst.envEqualE", @@ -276,7 +276,7 @@ "typing_StlcCbvDbParSubst.appears_free_in" ], 0, - "0b7eebfdc9aeae5f6eae14cb96ce04e3" + "60ca6d76223dbaea15bec3381f99dd10" ], [ "StlcCbvDbParSubst.free_in_context", @@ -372,7 +372,7 @@ "subterm_ordering_StlcStrongDbParSubst.ELam" ], 0, - "25d7ba931ac4e38adabba72a15e2cfe1" + "c09f5bd1d5733c934e5cd075c70241d2" ], [ "StlcCbvDbParSubst.below_env", @@ -712,7 +712,7 @@ "typing_StlcStrongDbParSubst_Tm_abs_c636cdcc538f5ce27d02a83ecd813b7b" ], 0, - "957dfc34ca7945eb78cea18e658b7b21" + "46513957410afa27c7409b3f581aa7bc" ], [ "StlcCbvDbParSubst.subst_closed", @@ -933,7 +933,7 @@ "typing_StlcCbvDbParSubst.appears_free_in" ], 0, - "437b2f15cddb3458ff6b8e07b9c5177f" + "06a61fb25f955897e66dc6bec117883f" ], [ "StlcCbvDbParSubst.extend_gen_0_aux", @@ -1088,7 +1088,7 @@ "typing_StlcStrongDbParSubst.sub_beta" ], 0, - "794f32f0a7491a240685cf259df5cf5e" + "05d64243f07adb3fa01db74cf7a5d69c" ], [ "StlcCbvDbParSubst.sub_inc_above", @@ -1142,7 +1142,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "ee6375d20f9a5adcef2c1e5655cde4cb" + "b476052991028c845b0f28f5793d6cb8" ], [ "StlcCbvDbParSubst.appears_free_in", @@ -1170,7 +1170,7 @@ "subterm_ordering_StlcStrongDbParSubst.ELam" ], 0, - "9051d856225828db8dad44c77c9613a1" + "b7462c345835bcb613fe34f7af02eeb3" ], [ "StlcCbvDbParSubst.envEqualE", @@ -1240,7 +1240,7 @@ "typing_StlcCbvDbParSubst.appears_free_in" ], 0, - "f98f6036328d385bddbea8914ee90292" + "e75d53651fd5e271ca758610647bfea3" ], [ "StlcCbvDbParSubst.below", @@ -1264,7 +1264,7 @@ "subterm_ordering_StlcStrongDbParSubst.ELam" ], 0, - "2139f508d74caee16d02a65da0e0e83e" + "dcdbe18ebdd0bed338c12ca2a202817e" ], [ "StlcCbvDbParSubst.below_env", @@ -1550,7 +1550,7 @@ "typing_StlcCbvDbParSubst.appears_free_in" ], 0, - "c89e218436ecdd425233ccf90645efa1" + "3851c072514c5be8b6590bdeb6e3f3f5" ], [ "StlcCbvDbParSubst.extend_gen_0_aux", @@ -1651,7 +1651,7 @@ "typing_StlcStrongDbParSubst.sub_beta" ], 0, - "55e649dd5489053eeba3b078b555ecd9" + "681e13630f17f51ba8c751a4985d1736" ] ] ] \ No newline at end of file diff --git a/examples/metatheory/StlcCbvDbPntSubstNoLists.fst.hints b/examples/metatheory/StlcCbvDbPntSubstNoLists.fst.hints index fc9b216e86f..0dfd77528ad 100644 --- a/examples/metatheory/StlcCbvDbPntSubstNoLists.fst.hints +++ b/examples/metatheory/StlcCbvDbPntSubstNoLists.fst.hints @@ -122,7 +122,7 @@ "subterm_ordering_StlcCbvDbPntSubstNoLists.EApp" ], 0, - "e59c818c2c7071c26b59442ac2c3b711" + "15dc771b2099e61da8e92631dd564f63" ], [ "StlcCbvDbPntSubstNoLists.step", @@ -143,7 +143,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "f5dedac2f7be153e980f99d3df372766" + "6f6f1b28ddc6a3d6b27b93413a0d3651" ], [ "StlcCbvDbPntSubstNoLists.extend", @@ -480,7 +480,7 @@ "subterm_ordering_StlcCbvDbPntSubstNoLists.EApp" ], 0, - "b04bdeb90b38a665aba4b7378688a7ca" + "2fa473c1c8595df7ef85df2e523d7db5" ], [ "StlcCbvDbPntSubstNoLists.free_in_context", @@ -631,7 +631,7 @@ "typing_StlcCbvDbPntSubstNoLists.appears_free_in" ], 0, - "21b70448126e44b768697f3da5c4c704" + "18b37968c15ff04d3590a8746fe5a9d1" ], [ "StlcCbvDbPntSubstNoLists.typing_extensional", @@ -711,7 +711,7 @@ "typing_StlcCbvDbPntSubstNoLists.appears_free_in" ], 0, - "f626b36490f50bd9239ed4b078fe3f05" + "2a3569a041b8b4ba8dd4eb5c91023964" ], [ "StlcCbvDbPntSubstNoLists.preservation", @@ -772,7 +772,7 @@ "typing_StlcCbvDbPntSubstNoLists.step" ], 0, - "fff6b6d62d95bb7533a244f50d3d4065" + "e4355ab4c87d912293ff54c7931196b4" ], [ "StlcCbvDbPntSubstNoLists.ty", @@ -895,7 +895,7 @@ "subterm_ordering_StlcCbvDbPntSubstNoLists.EApp" ], 0, - "daba5b4852b1daab1fc7a8bb95c8db65" + "82c5621734ff7b8b09ecba9109e3acb9" ], [ "StlcCbvDbPntSubstNoLists.step", @@ -916,7 +916,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "212678ce622c910e5511f79465d1a81a" + "d6a4962b65935aa2e2adf78eb0003149" ], [ "StlcCbvDbPntSubstNoLists.extend", @@ -1202,7 +1202,7 @@ "subterm_ordering_StlcCbvDbPntSubstNoLists.EApp" ], 0, - "ccb9c8480f9bbce2b01136de7ee2d35f" + "9a11a36d402950b0783bdab5a93477a0" ], [ "StlcCbvDbPntSubstNoLists.equal", @@ -1284,7 +1284,7 @@ "typing_StlcCbvDbPntSubstNoLists.appears_free_in" ], 0, - "f3f7cc2cd1205c4e393b958fa9094216" + "3a84db6d3084c70360dcb54328bdcf0b" ], [ "StlcCbvDbPntSubstNoLists.typing_extensional", @@ -1364,7 +1364,7 @@ "typing_StlcCbvDbPntSubstNoLists.appears_free_in" ], 0, - "9f4103c81db29cb9619d80882a84c567" + "194fab99d840e9563786fc6f7865544e" ], [ "StlcCbvDbPntSubstNoLists.preservation", @@ -1413,7 +1413,7 @@ "typing_StlcCbvDbPntSubstNoLists.step" ], 0, - "14035b40aa28b436dae78b7ed957b71a" + "566b4a8a3d70f18b0905e0f161f5302c" ] ] ] \ No newline at end of file diff --git a/examples/metatheory/StlcStrongDbParSubst.fst.hints b/examples/metatheory/StlcStrongDbParSubst.fst.hints index 075e84e51ca..e0a7a92bf65 100644 --- a/examples/metatheory/StlcStrongDbParSubst.fst.hints +++ b/examples/metatheory/StlcStrongDbParSubst.fst.hints @@ -230,7 +230,7 @@ "well-founded-ordering-on-nat" ], 0, - "67aba933e7e6430c7b5b9797783fda9f" + "33e82e23b709dd97d6b3d0a705173417" ], [ "StlcStrongDbParSubst.sub_elam", @@ -757,7 +757,7 @@ "typing_StlcStrongDbParSubst.uu___is_EUnit" ], 0, - "8d0127e689803e938a1d628ed33d0d79" + "6ecc493a64d884687f9eeb49760f23fc" ], [ "StlcStrongDbParSubst.subst_extensional", @@ -912,7 +912,7 @@ "well-founded-ordering-on-nat" ], 0, - "0072edf4084a67cef4735884f4593794" + "8bbce28002d4fd41c384bf15f1ad9788" ], [ "StlcStrongDbParSubst.substitution_beta", @@ -940,7 +940,7 @@ "token_correspondence_StlcStrongDbParSubst.sub_beta" ], 0, - "78638c8e70475423b99aa3730eb69e21" + "2d7d57958a3f0996042d345de7fcf708" ], [ "StlcStrongDbParSubst.preservation", @@ -987,7 +987,7 @@ "subterm_ordering_StlcStrongDbParSubst.TyApp" ], 0, - "98e83c55812de94c8621a6e3032e15c3" + "34fc49251ac4791841e81929ba888e31" ], [ "StlcStrongDbParSubst.typ", @@ -1192,7 +1192,7 @@ "well-founded-ordering-on-nat" ], 0, - "e2c3ef3b5c33d56914ce7c2b1b6fd257" + "7099569b77574e33c15fc54b4f47362e" ], [ "StlcStrongDbParSubst.sub_elam", @@ -1711,7 +1711,7 @@ "typing_StlcStrongDbParSubst.uu___is_EUnit" ], 0, - "b67c2dcb4572d9b00124490a80df9e8b" + "b77dee1eaa5f938c851b9d5678210b0d" ], [ "StlcStrongDbParSubst.subst_extensional", @@ -1835,7 +1835,7 @@ "well-founded-ordering-on-nat" ], 0, - "710fc2ccc2f32e717891e846e2cf629e" + "a8e05e5ad6f30d581d63aba9420df752" ], [ "StlcStrongDbParSubst.substitution_beta", @@ -1863,7 +1863,7 @@ "token_correspondence_StlcStrongDbParSubst.sub_beta" ], 0, - "f9b480cb8e5b8bfed0d90192bf056a0a" + "5b342b3d4423139cd4c2c240d005fb6a" ], [ "StlcStrongDbParSubst.preservation", @@ -1910,7 +1910,7 @@ "subterm_ordering_StlcStrongDbParSubst.TyApp" ], 0, - "ed0d05f37fe847f29de25559b9e5ce2b" + "8cf8700f5e859d892b294df94708377b" ] ] ] \ No newline at end of file diff --git a/examples/metatheory/indind.fst.hints b/examples/metatheory/indind.fst.hints index 02ef6076eb0..e3cbd7c5674 100644 --- a/examples/metatheory/indind.fst.hints +++ b/examples/metatheory/indind.fst.hints @@ -79,7 +79,7 @@ "typing_tok_Indind.Nil@tok", "typing_tok_Indind.Z@tok" ], 0, - "9c4a9a4b1a082f58f1192f751e50bc02" + "57b80f1f4a17c8633b4cc4fd273bfda1" ], [ "Indind.vdl_valid", @@ -99,7 +99,7 @@ "typing_tok_Indind.Z@tok" ], 0, - "eeea67a383af77d94012c9b798edbe91" + "0345a2252bd45291a95af73d4f3687d1" ], [ "Indind.vdl_induction", @@ -159,7 +159,7 @@ "typing_tok_Indind.Nil@tok" ], 0, - "f53fbc9b927d9172204cdd08b37a2a45" + "f11889604f47d64c95a1b7682ed7c0a8" ], [ "Indind.vdl_induction", @@ -218,7 +218,7 @@ "subterm_ordering_Indind.Cons", "typing_tok_Indind.Nil@tok" ], 0, - "d828ca1e6e364351fdcbb53bfdc1a56b" + "3f7d15d98d18b38c3ad633279a3d5afa" ], [ "Indind.ctx0", @@ -427,7 +427,7 @@ "subterm_ordering_Indind.ConsCtx", "typing_tok_Indind.EmptyCtx@tok" ], 0, - "e557d6ff67456082e2451ce6fb6ea963" + "f8893a5f028be24a791b7461de5ada79" ], [ "Indind.ctx_valid", @@ -450,7 +450,7 @@ "subterm_ordering_Indind.Var", "typing_tok_Indind.EmptyCtx@tok" ], 0, - "18d0a3ab7978179703a7c240ed4bd091" + "4d364fbad5689da17554f11a8c140696" ], [ "Indind.ctx_valid", @@ -470,7 +470,7 @@ "typing_tok_Indind.EmptyCtx@tok" ], 0, - "db83d6c8972ae0fc2d6e132868ebbd75" + "6171af07d1cc5a8ed0350cae1de69feb" ], [ "Indind.empty_ctx", @@ -755,7 +755,7 @@ "typing_tok_Indind.Nil@tok", "typing_tok_Indind.Z@tok" ], 0, - "6a3fb0b39a14e8d710b45676a3355ab1" + "78c41aaf759cf3a13ceb6b8ad789122f" ], [ "Indind.vdl_valid", @@ -775,7 +775,7 @@ "typing_tok_Indind.Z@tok" ], 0, - "0efec60f7469ee5dcaccc33211a27bf3" + "c46824c84fd876c74d5bb5b7f1dd2706" ], [ "Indind.vdl_induction", @@ -835,7 +835,7 @@ "typing_tok_Indind.Nil@tok" ], 0, - "45ba9a0e5e12b005744ce346ecc3f163" + "6dcbdf84ff74e4c4666722f692e4cf2e" ], [ "Indind.vdl_induction", @@ -894,7 +894,7 @@ "subterm_ordering_Indind.Cons", "typing_tok_Indind.Nil@tok" ], 0, - "5851ba58f1cae27537bd3a4b8f0675e1" + "7b35803ca4fdbf9c8cfa5929841cf869" ], [ "Indind.ctx0", @@ -1103,7 +1103,7 @@ "subterm_ordering_Indind.ConsCtx", "typing_tok_Indind.EmptyCtx@tok" ], 0, - "8cec1182dd200bbe9de7d7c3ec5d9c30" + "8ba689dfc904c0639cac7833225a227c" ], [ "Indind.ctx_valid", @@ -1126,7 +1126,7 @@ "subterm_ordering_Indind.Var", "typing_tok_Indind.EmptyCtx@tok" ], 0, - "f41bd96b6ff2262b20be7e32b5ea5ef9" + "b96ce58685059f9b322d2def8c17d35f" ], [ "Indind.ctx_valid", @@ -1146,7 +1146,7 @@ "typing_tok_Indind.EmptyCtx@tok" ], 0, - "994f39d8ee5a5a0c4dc3c196cb67f3bc" + "b6ec610db361b865c844b7ca2bda44c1" ], [ "Indind.empty_ctx", diff --git a/examples/micro-benchmarks/DoNotation.fst.hints b/examples/micro-benchmarks/DoNotation.fst.hints index 2bfc2a04bfe..7bc367f453f 100644 --- a/examples/micro-benchmarks/DoNotation.fst.hints +++ b/examples/micro-benchmarks/DoNotation.fst.hints @@ -15,7 +15,7 @@ "well-founded-ordering-on-nat" ], 0, - "318764a7659b6aa44383cd7e3ef1ea65" + "7f8d9a593ac876f25002c9cbb7374edf" ], [ "DoNotation.uu___8", @@ -44,7 +44,7 @@ "well-founded-ordering-on-nat" ], 0, - "82907a5b5c5be16602618361d1ec8f1d" + "c29a8d04e9e49b54178fb22c5aec1cdb" ], [ "DoNotation.uu___8", diff --git a/examples/micro-benchmarks/FirstProofs.fst.hints b/examples/micro-benchmarks/FirstProofs.fst.hints index 362436e5c44..86a9adcf8df 100644 --- a/examples/micro-benchmarks/FirstProofs.fst.hints +++ b/examples/micro-benchmarks/FirstProofs.fst.hints @@ -16,7 +16,7 @@ "well-founded-ordering-on-nat" ], 0, - "cb9b128792cc9f6c934390eed0c21a80" + "2d6350896da35ef21a528e4477dbe246" ], [ "FirstProofs.factorial_is_positive", @@ -38,7 +38,7 @@ "well-founded-ordering-on-nat" ], 0, - "9aa5d19c943b0f8bb21982e0ecd85ac1" + "d68285c2bf1abd1363690ec4b260b71b" ], [ "FirstProofs.factorial_is_increasing", @@ -61,7 +61,7 @@ "well-founded-ordering-on-nat" ], 0, - "88a1ad580b29eb589d3afe4933046227" + "a9017bef815366a27de2a6484fb08963" ], [ "FirstProofs.factorial_is_doubling", @@ -85,7 +85,7 @@ "well-founded-ordering-on-nat" ], 0, - "e799a053cde4d29ffce7e3b65f5f42b0" + "bd1e9762506f54e342c46612750dba96" ], [ "FirstProofs.fibonacci", @@ -102,7 +102,7 @@ "well-founded-ordering-on-nat" ], 0, - "b950bf4178a9be4a6325e3a3d627be8b" + "59fd004edc0f6a1dcbcb5e1f27e7b76d" ], [ "FirstProofs.fibonacci_is_increasing", @@ -125,7 +125,7 @@ "typing_FirstProofs.fibonacci", "well-founded-ordering-on-nat" ], 0, - "a5fb510ad625fdec4601cdafc2cb0edb" + "41f3eda579adc32c941b3c3ae5587895" ], [ "FirstProofs.factorial", @@ -142,7 +142,7 @@ "well-founded-ordering-on-nat" ], 0, - "7dac2918fdedf448977e0703fc4dcd42" + "e63465965bbf9c5e2351a9dbb2a5e67f" ], [ "FirstProofs.fibonacci", @@ -159,7 +159,7 @@ "well-founded-ordering-on-nat" ], 0, - "a9dfeae9a77be49d36b0eb474e5d06ed" + "8d087376966ca83aa9a6bcc94338bc39" ] ] ] \ No newline at end of file diff --git a/examples/micro-benchmarks/IntNormalization.fst.hints b/examples/micro-benchmarks/IntNormalization.fst.hints index 5d6ab9ce263..3cfbe1b269d 100644 --- a/examples/micro-benchmarks/IntNormalization.fst.hints +++ b/examples/micro-benchmarks/IntNormalization.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq", "true_interp" ], 0, - "14e8e7c0500b5e8f202ee2760340c1f0" + "cf6587e6b57094a28363c376c32a1764" ], [ "IntNormalization.uu___66", @@ -17,7 +17,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq", "true_interp" ], 0, - "650630d24579b7c977f6b3d0d143a4a0" + "9d376c2bcb4765661e16cfa2e8f6b19e" ], [ "IntNormalization.uu___63", @@ -26,7 +26,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq", "true_interp" ], 0, - "d7f0f3bd2f2f2bc12baadd55479b3b48" + "174024ec80db6305f0e519dba38faaa3" ], [ "IntNormalization.uu___66", @@ -35,7 +35,7 @@ 1, [ "@query", "assumption_FStar.UInt32.t__uu___haseq", "true_interp" ], 0, - "5618d9305cb1fd934522444a210eb758" + "8f98c44987cb219a05123ad27abf1db1" ] ] ] \ No newline at end of file diff --git a/examples/micro-benchmarks/NegativeTests.Termination.fst.hints b/examples/micro-benchmarks/NegativeTests.Termination.fst.hints index 01cc1e764cf..3f32564dd8a 100644 --- a/examples/micro-benchmarks/NegativeTests.Termination.fst.hints +++ b/examples/micro-benchmarks/NegativeTests.Termination.fst.hints @@ -16,7 +16,7 @@ "well-founded-ordering-on-nat" ], 0, - "6380aacd586fe7083238eec168b02575" + "4bbb07639eb23f1c7c0fbd46bf1f9f85" ], [ "NegativeTests.Termination.snat", @@ -56,7 +56,7 @@ "well-founded-ordering-on-nat" ], 0, - "706c917638143d70efedd6959fd4cf0a" + "d5592c0b26124e694c38d9b4779c53cc" ], [ "NegativeTests.Termination.snat", diff --git a/examples/micro-benchmarks/Normalization.fst.hints b/examples/micro-benchmarks/Normalization.fst.hints index 10490380f3b..5d9b23c6def 100644 --- a/examples/micro-benchmarks/Normalization.fst.hints +++ b/examples/micro-benchmarks/Normalization.fst.hints @@ -25,7 +25,7 @@ "well-founded-ordering-on-nat" ], 0, - "57679fc7b06294d6b8447b2cc646cefb" + "011c63ea336c63c6b62581f64bfb90f9" ], [ "Normalization.test2", @@ -82,7 +82,7 @@ "well-founded-ordering-on-nat" ], 0, - "95759195b1557ced6b69638dd274f30c" + "f5eedf8f69d119f5f1ad4acc0ea08f62" ], [ "Normalization.pow2_values", diff --git a/examples/micro-benchmarks/Pruning.fst.hints b/examples/micro-benchmarks/Pruning.fst.hints index 8d4c9eba7da..109bbacea34 100644 --- a/examples/micro-benchmarks/Pruning.fst.hints +++ b/examples/micro-benchmarks/Pruning.fst.hints @@ -32,7 +32,7 @@ "typing_FStar.Seq.Base.slice" ], 0, - "f916600dbd64814cc254c31cfe01860b" + "a73eff44b7b1fb41786ca28939b1d6bc" ], [ "Pruning.lemma", @@ -48,7 +48,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "a9beb0e524e312040e129942352a7832" + "ce8acbcec7b124af0cca18fcf71e5f33" ] ] ] \ No newline at end of file diff --git a/examples/micro-benchmarks/TwoPhaseTC.fst.hints b/examples/micro-benchmarks/TwoPhaseTC.fst.hints index 55ab702fc68..def18d318a2 100644 --- a/examples/micro-benchmarks/TwoPhaseTC.fst.hints +++ b/examples/micro-benchmarks/TwoPhaseTC.fst.hints @@ -32,7 +32,7 @@ "refinement_interpretation_TwoPhaseTC_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "9d56c8a0ee105956b58fc4be54fbe486" + "0d8eb3c5fb9f499e849f69a78e746dbb" ], [ "TwoPhaseTC.f8", @@ -46,7 +46,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "2c616c72210cdd2763cb3b7655b06fe6" + "102ad5119a54276a663bc0615e0b78d6" ], [ "TwoPhaseTC.f12", @@ -55,7 +55,7 @@ 0, [ "@query" ], 0, - "83dc4f6799ceb5f8f2d83afacd338ae9" + "35542b2a90b6338abbc45513f1995861" ], [ "TwoPhaseTC.f13", @@ -72,7 +72,7 @@ "well-founded-ordering-on-nat" ], 0, - "4742dd474cd7e3d4e62d383525cebfda" + "f4528727fc4b0b65fe586d1e9b100c4a" ], [ "TwoPhaseTC.f14", @@ -81,7 +81,7 @@ 0, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "44129d02ff79ab6ebcdd6356ca27678f" + "3fffd59746f12fc2e233e3d615c3cbbc" ], [ "TwoPhaseTC.f18", @@ -90,7 +90,7 @@ 0, [ "@query" ], 0, - "d5362f72ec1e48b3c20b9ec347a21733" + "0486735a0864829f42aea5af855c93c2" ], [ "TwoPhaseTC.__proj__ExIntro__item___1", @@ -102,7 +102,7 @@ "projection_inverse_TwoPhaseTC.ExIntro_x" ], 0, - "e1c0ee94f5af4d9d5cf3b14739ab2612" + "88b0417bcb17aa56865a4eedd44116ae" ], [ "TwoPhaseTC.foo_1451", @@ -115,7 +115,7 @@ "projection_inverse_FStar.Pervasives.Native.Some_v" ], 0, - "700d5a4931204b2f1db85592d83779ca" + "9d8ae676e1a4bf15d75f5a2fc0a4ace2" ], [ "TwoPhaseTC.t2_1129", @@ -129,7 +129,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "8127539b14acdae1ef48894edaebe434" + "efcd2e24c5560b590f8a5e3355e6681e" ], [ "TwoPhaseTC.t3_1129", @@ -143,7 +143,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "46fc2524e993377a42041c03130bd4cb" + "464573b9883b1064cd5f9db23880f9aa" ], [ "TwoPhaseTC.solve_1124", @@ -155,7 +155,7 @@ "haseqTwoPhaseTC_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "b5247c32277cf200799126d29c26b9ac" + "3b5ee951d3cc2342d23e9609bbee7d8d" ], [ "TwoPhaseTC.nth_tot_1124", @@ -175,7 +175,7 @@ "typing_FStar.List.Tot.Base.nth" ], 0, - "902f568d7b926c00ce90b253847f2653" + "4b9de9d29cafa8a504ac1180152a41c1" ], [ "TwoPhaseTC.calc_1124", @@ -199,7 +199,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "ee25e4c80f9305f759f53fe0b3de8fa0" + "403214e008bf38d5fe1aaca3fc5e2489" ], [ "TwoPhaseTC.copy'_754", @@ -214,7 +214,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "b20e457b5a91d8156bc9bf722e9f80cc" + "12aa572e2847273d28bffcb144b245c5" ], [ "TwoPhaseTC.test2_754", @@ -229,7 +229,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "72c0bd57b963f966f9b8116e26658670" + "be440b189c810b5c6d1a858d49b2b7a6" ], [ "TwoPhaseTC.test2_754", @@ -238,7 +238,7 @@ 1, [ "@query" ], 0, - "43fa4cf5ac86e80796a58f9a9b19f376" + "bc5e2b1600b3de81ad17bdd3acd6a238" ], [ "TwoPhaseTC.conjunction_monoid", @@ -271,7 +271,7 @@ "refinement_interpretation_TwoPhaseTC_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "a15a0fc3c797d574057272ad15bf8a5d" + "fe87e2f691ecc182e91fec878ac20c45" ], [ "TwoPhaseTC.f8", @@ -283,7 +283,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "c80d64c483c7e2cf97452160bd97561c" + "0f5bea54ed09431bd4adefc187b7d68d" ], [ "TwoPhaseTC.f12", @@ -292,7 +292,7 @@ 0, [ "@query" ], 0, - "30458693fb36a0f2add48206742accb7" + "c3b401a963de83ad801b013693ae0a0a" ], [ "TwoPhaseTC.f13", @@ -309,7 +309,7 @@ "well-founded-ordering-on-nat" ], 0, - "991d2eee5dd4eda861e165143102bc54" + "7f4c04d2ce2857ae6b75613d1f8a723b" ], [ "TwoPhaseTC.f14", @@ -318,7 +318,7 @@ 0, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "75c378f85ffb0aa7884c28f07201b724" + "b1d55b575489696a340a9c73c672855f" ], [ "TwoPhaseTC.__proj__ExIntro__item___1", @@ -330,7 +330,7 @@ "projection_inverse_TwoPhaseTC.ExIntro_x" ], 0, - "394fc69ff5552e326af6ad2c1689f023" + "3f339a59a7ea7d2f91a4e10781cccad2" ], [ "TwoPhaseTC.foo_1451", @@ -343,7 +343,7 @@ "projection_inverse_FStar.Pervasives.Native.Some_v" ], 0, - "7d86e20448d2f5e8e8d4ea8841f606ad" + "246b3b59b4f8ec5a5810a27793eb02c8" ], [ "TwoPhaseTC.t2_1129", @@ -357,7 +357,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "e12743cee310d88f00e71bc48fc57ae1" + "28969e2dfeaf342fcc5b04c48ae2dd7d" ], [ "TwoPhaseTC.t3_1129", @@ -371,7 +371,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "dd1c5b6e5b1ea028694c0fa24a42fd4a" + "cd3636b41f9fac07b09769aa664566e6" ], [ "TwoPhaseTC.solve_1124", @@ -383,7 +383,7 @@ "haseqTwoPhaseTC_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "dd21559f78a02a312f22719872ac318c" + "dba6f954f1d131b4aaf933f6edc06196" ], [ "TwoPhaseTC.nth_tot_1124", @@ -403,7 +403,7 @@ "typing_FStar.List.Tot.Base.nth" ], 0, - "6ce25277d21725af60a91a5afef39554" + "f5a8fd0d52bdd156581fcc5273c1d36f" ], [ "TwoPhaseTC.calc_1124", @@ -427,7 +427,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "1a0d095afdb23deef1459817af18aa6c" + "bb0c8e3cf773a13af49b28a953a366ca" ], [ "TwoPhaseTC.copy'_754", @@ -442,7 +442,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "71a229189305081bf274ad794af3ee5f" + "d73cc6b8c9bdd00c6fc431db2bdc0228" ], [ "TwoPhaseTC.test2_754", @@ -457,7 +457,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "0ba326387595f0199dea820d75ba6dae" + "01a710aa2b40a406ac75576b5443ffdf" ] ] ] \ No newline at end of file diff --git a/examples/micro-benchmarks/UnifyMatch.fst.hints b/examples/micro-benchmarks/UnifyMatch.fst.hints index 76ffa8e2d42..3e39b4ff250 100644 --- a/examples/micro-benchmarks/UnifyMatch.fst.hints +++ b/examples/micro-benchmarks/UnifyMatch.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "7084641ebe97c879e02a761999be9416" + "aa1a1ada37ab88106cb7040e706d59cd" ], [ "UnifyMatch.__proj__S__item___0", @@ -21,7 +21,7 @@ "refinement_interpretation_UnifyMatch_Tm_refine_b909e5f5ff265386c08f5741455e23b9" ], 0, - "d2a387b38eb92f6da4f2c59a53e132ca" + "280cb89de0d0515d5af1ec9902907793" ], [ "UnifyMatch.nat2unary", @@ -37,7 +37,7 @@ "well-founded-ordering-on-nat" ], 0, - "1a6d06358f754860b56648578dd084f2" + "fc7dc2e9b68b9a4b12f9d6ac868d2765" ], [ "UnifyMatch.even", @@ -46,7 +46,7 @@ 1, [ "@query", "assumption_UnifyMatch.unat__uu___haseq" ], 0, - "6aa6b2006c2e6d86e065e6fbf3d0d49b" + "cba95c7c97ca0881047680d46013bf28" ], [ "UnifyMatch.__proj__Even_SS__item__n", @@ -59,7 +59,7 @@ "refinement_interpretation_UnifyMatch_Tm_refine_b82e9317628d0fc1fba9e36ac5ed44f2" ], 0, - "2926dd10d6a9dd6418292be9fde11f07" + "27b4cb14f241afcf7f35602edb282d17" ], [ "UnifyMatch.__proj__Even_SS__item___1", @@ -74,7 +74,7 @@ "refinement_interpretation_UnifyMatch_Tm_refine_b82e9317628d0fc1fba9e36ac5ed44f2" ], 0, - "fe2328a2c3ce439d4a51102bcddf929e" + "55f82d18cf8cc6d4e287dbf8df9e1d1c" ], [ "UnifyMatch.test1", @@ -89,14 +89,14 @@ "constructor_distinct_FStar.Tactics.Result.Success", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v", "unit_typing" ], 0, - "bfa35d2d120c1f61a7f53b2d9f969a49" + "d4a5059674a6c0fb267f20b7592655dc" ], [ "UnifyMatch.unat", @@ -105,7 +105,7 @@ 1, [ "@query" ], 0, - "fba9d1818bf091ecc56f898c7724f7b5" + "806015be5de3b7f086873c8609fa86bd" ], [ "UnifyMatch.__proj__S__item___0", @@ -118,7 +118,7 @@ "refinement_interpretation_UnifyMatch_Tm_refine_b909e5f5ff265386c08f5741455e23b9" ], 0, - "c831c78165aaf876d2f1663a2f98efc2" + "91550309f5a313d622ba60d4425bfeb7" ], [ "UnifyMatch.nat2unary", @@ -134,7 +134,7 @@ "well-founded-ordering-on-nat" ], 0, - "909feeb14135dc57589270fa585d77b0" + "329c3b59b3f1dd1f4b128bc3fda43409" ], [ "UnifyMatch.even", @@ -143,7 +143,7 @@ 1, [ "@query", "assumption_UnifyMatch.unat__uu___haseq" ], 0, - "8333fb911d3a955e28a028ca5f156662" + "206856f4c8acf86d34039fbced0bd81e" ], [ "UnifyMatch.__proj__Even_SS__item__n", @@ -156,7 +156,7 @@ "refinement_interpretation_UnifyMatch_Tm_refine_b82e9317628d0fc1fba9e36ac5ed44f2" ], 0, - "fe924894913af5a362aac8d8c2634b95" + "8cd434702248a74b9576eb1c92406ed8" ], [ "UnifyMatch.__proj__Even_SS__item___1", @@ -171,7 +171,7 @@ "refinement_interpretation_UnifyMatch_Tm_refine_b82e9317628d0fc1fba9e36ac5ed44f2" ], 0, - "941aa263dedb2cced0143b6bdf9212c2" + "4fb67e6d03d7670af5a001eb876c8699" ], [ "UnifyMatch.test1", @@ -186,14 +186,14 @@ "constructor_distinct_FStar.Tactics.Result.Success", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v", "unit_typing" ], 0, - "78c6d9a49ef45b5a7463820d6ae8391a" + "4dd1c43e2527ab3308e3e1119f67d806" ] ] ] \ No newline at end of file diff --git a/examples/micro-benchmarks/Unit1.Basic.fst.hints b/examples/micro-benchmarks/Unit1.Basic.fst.hints index cb4eb8285d5..66249e9ed9a 100644 --- a/examples/micro-benchmarks/Unit1.Basic.fst.hints +++ b/examples/micro-benchmarks/Unit1.Basic.fst.hints @@ -297,7 +297,7 @@ "well-founded-ordering-on-nat" ], 0, - "e089710fbb88541e5ad7f639f6e63573" + "05472a5f18733281b12a7fd09265143f" ], [ "Unit1.Basic.inat", @@ -339,7 +339,7 @@ "subterm_ordering_Unit1.Basic.S" ], 0, - "4448350682a22b5001e30e06b4c56e50" + "ef8d092ca021fae6d6aa8ce81aa9fa12" ], [ "Unit1.Basic.ackermann", @@ -359,7 +359,7 @@ "well-founded-ordering-on-nat" ], 0, - "c4fed77f2b4bf14e92e66c33adbcf09a" + "3683eb3596c776f537d7dd37cbf3d794" ], [ "Unit1.Basic.__proj__Seq__item__end_i", @@ -515,7 +515,7 @@ "subterm_ordering_Unit1.Basic.C", "typing_tok_Unit1.Basic.N@tok" ], 0, - "07a3ea9ef4cd61e19d98e9e607d75b35" + "b0bb59c23127d4af415c0b0630de9c6b" ], [ "Unit1.Basic.pre", @@ -654,7 +654,7 @@ "projection_inverse_BoxBool_proj_0", "subterm_ordering_Prims.Cons" ], 0, - "d06c7d7bb1b8321c0ad5b90b5e23abb7" + "3f9aff1c00161dc11b84fa32a7bb5c72" ], [ "Unit1.Basic.test_skolem_let", @@ -754,7 +754,7 @@ "token_correspondence_FStar.List.Tot.Base.op_At" ], 0, - "7b4b64de70bc0d60149e3064842a4cfb" + "031a221e9c661630190425c0b0a5f7b2" ], [ "Unit1.Basic.st_id_wrap", @@ -799,7 +799,7 @@ "well-founded-ordering-on-nat" ], 0, - "4904f29d0b747fc6e6df7ca778135e88" + "efbb50fe799a49f4d53d20bc73da7515" ], [ "Unit1.Basic.factorial_is_positive", @@ -825,7 +825,7 @@ "well-founded-ordering-on-nat" ], 0, - "a477a42a659bb44c51f6c787a9a18061" + "1d54802aa9fb55df4b9b4f97a93f1ae2" ], [ "Unit1.Basic.length", @@ -839,7 +839,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "d71727749a1153ffe6e5259029df8ad3" + "6e14e563773f0bbd33858eebafc383e0" ], [ "Unit1.Basic.map", @@ -853,7 +853,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "3f326560e115ad53db3bf4c768b45426" + "ee6232596ad3c0a87b4e6366d2ef34de" ], [ "Unit1.Basic.test_map1", @@ -931,7 +931,7 @@ "well-founded-ordering-on-nat" ], 0, - "94586c031089df1ebfb13b49116a1827" + "1da453bcdf01029d7fd4db774a0773c4" ], [ "Unit1.Basic.even", @@ -949,7 +949,7 @@ "well-founded-ordering-on-nat" ], 0, - "f4d320a1226d0d2af3cf473c536f9091" + "18d14896504ccdcfa6d47c6d6b258b44" ], [ "Unit1.Basic.test_even1", @@ -1373,7 +1373,7 @@ "well-founded-ordering-on-nat" ], 0, - "d0060dd317e221b99c0fdb50b2e9b17a" + "acdcff56b7500b0c9142a486256d6bbc" ], [ "Unit1.Basic.inat", @@ -1415,7 +1415,7 @@ "subterm_ordering_Unit1.Basic.S" ], 0, - "089b7b4f02762beff2d710edf08080a7" + "e051d28e83040b786b1930ac921ca272" ], [ "Unit1.Basic.ackermann", @@ -1435,7 +1435,7 @@ "well-founded-ordering-on-nat" ], 0, - "d57479feacb818ced1cc1428a60fd6f0" + "fe2a8896d89de5a3267614c372bebb02" ], [ "Unit1.Basic.__proj__Seq__item__end_i", @@ -1533,7 +1533,7 @@ "subterm_ordering_Unit1.Basic.C", "typing_tok_Unit1.Basic.N@tok" ], 0, - "d4fc106a7d51c0b836f84208f9c1fbaa" + "c5536402367f855572481ba438bde44f" ], [ "Unit1.Basic.pre", @@ -1669,7 +1669,7 @@ "projection_inverse_BoxBool_proj_0", "subterm_ordering_Prims.Cons" ], 0, - "e826494cf71cd22df78ab37f7bc2180f" + "b4229c1bd42a2bf82145b1a799d0e579" ], [ "Unit1.Basic.test_skolem_let", @@ -1756,7 +1756,7 @@ "token_correspondence_FStar.List.Tot.Base.op_At" ], 0, - "517afd481e5fd176c0260531dae073b8" + "8df8e90ae005cc3701ee78b0dd1ef656" ], [ "Unit1.Basic.st_id_wrap", @@ -1792,7 +1792,7 @@ "well-founded-ordering-on-nat" ], 0, - "2001d7d61615969da517d334dc6b74c2" + "fbbdeea1601f456e2d6438b332fa5390" ], [ "Unit1.Basic.length", @@ -1806,7 +1806,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "bc0f2dcc6001e9fbb89c03675ddb5309" + "49bc1a55ae0b067fdfaaca42e58517a2" ], [ "Unit1.Basic.map", @@ -1820,7 +1820,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "127cb96693b99a9e514659345e041321" + "ca83f4c28da4701d9fee3ed2b3057905" ], [ "Unit1.Basic.test_map1", @@ -1897,7 +1897,7 @@ "well-founded-ordering-on-nat" ], 0, - "8300b1e39d6511996f78f3f58b8994af" + "30a163e16b910f7a8156f504e3b509ec" ], [ "Unit1.Basic.even", @@ -1915,7 +1915,7 @@ "well-founded-ordering-on-nat" ], 0, - "310ac6e731f95edf2ac234090b1546ce" + "9edab948e8b41cdf27e78800104d45ba" ], [ "Unit1.Basic.test_even1", diff --git a/examples/micro-benchmarks/Unit1.RecursiveTypeFunctions.fst.hints b/examples/micro-benchmarks/Unit1.RecursiveTypeFunctions.fst.hints index 4e44eba8c47..e2f73fb3f08 100644 --- a/examples/micro-benchmarks/Unit1.RecursiveTypeFunctions.fst.hints +++ b/examples/micro-benchmarks/Unit1.RecursiveTypeFunctions.fst.hints @@ -83,7 +83,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.TofS" ], 0, - "0d63a39e3083cbb520df41fce3a009a7" + "7fe33f93edce70c823077144a4e648d3" ], [ "Unit1.RecursiveTypeFunctions.good_t", @@ -99,7 +99,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.SofT" ], 0, - "09d7a289a01ca3c09b2a25b5664782b6" + "cd2847a748cd138416843cbb0f8c4bec" ], [ "Unit1.RecursiveTypeFunctions.extract_nat_t", @@ -128,7 +128,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.TofS" ], 0, - "753c201b4a8d6218791b453fc41b90ac" + "8de81aba486f5e5d4285cec907e0cbe2" ], [ "Unit1.RecursiveTypeFunctions.extract_nat_t", @@ -158,7 +158,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.SofT" ], 0, - "a94dc6ec01da33fb147f0b1533215864" + "040c9a41c6ec5ec9093c125c2c57c7a6" ], [ "Unit1.RecursiveTypeFunctions.pointwise_eq", @@ -178,7 +178,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "726c72a3b77251028eae4b518ccf6519" + "bceae2b539397f578b8e88400cfd1a6d" ], [ "Unit1.RecursiveTypeFunctions.pointwise_eq_length", @@ -295,7 +295,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.TofS" ], 0, - "c66d76764bfe413ab2b7a0a4c8de0cf8" + "e40eecbc8b5256bc96d3035cd9c55f7c" ], [ "Unit1.RecursiveTypeFunctions.good_t", @@ -311,7 +311,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.SofT" ], 0, - "9c4f23f5ef9eb9ca753d93732a501016" + "000870d1173e500add46786afd18b188" ], [ "Unit1.RecursiveTypeFunctions.extract_nat_t", @@ -340,7 +340,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.TofS" ], 0, - "e7a83029e37f6e7aef2849a8238ce205" + "1c44d69b3d5d05f8ceb8123252de987c" ], [ "Unit1.RecursiveTypeFunctions.extract_nat_t", @@ -370,7 +370,7 @@ "subterm_ordering_Unit1.RecursiveTypeFunctions.SofT" ], 0, - "5deabfa7ebd0aef3a53480bbeb790190" + "9121ffcd207c29fe3cd3375caefa4338" ], [ "Unit1.RecursiveTypeFunctions.pointwise_eq", @@ -390,7 +390,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "a1323a0b96111c36b4e7a79be0bff86e" + "0e7706690fe43e0e75d9e09a422459eb" ], [ "Unit1.RecursiveTypeFunctions.pointwise_eq_length", diff --git a/examples/miniparse/MiniParse.Impl.Base.fst.hints b/examples/miniparse/MiniParse.Impl.Base.fst.hints index 8087f40ed5b..08b40092fda 100644 --- a/examples/miniparse/MiniParse.Impl.Base.fst.hints +++ b/examples/miniparse/MiniParse.Impl.Base.fst.hints @@ -16,7 +16,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "dd37246ef199339bb5ce4c72deac166a" + "8eb9382734b68b4b4eff7a1c669671f9" ], [ "MiniParse.Impl.Base.coerce_parser_impl", @@ -29,7 +29,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "d150b1cc6fba0d15f003c208e5d1d7c0" + "b09ba8f5db4157a8af2250d3bca0ae1e" ], [ "MiniParse.Impl.Base.serializer_impl", @@ -54,7 +54,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "b2948313409a957c4e8adc83e06842c2" + "598f633c6a604e9cf276fd09a7750c01" ], [ "MiniParse.Impl.Base.parser_impl", @@ -71,7 +71,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "4b4b79b564dd3637da9aac324785bf49" + "72a94b2f79ed612f67f063930e86719c" ], [ "MiniParse.Impl.Base.coerce_parser_impl", @@ -84,7 +84,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "1099c08d36554b10a53ee9c5516465ad" + "f08bce79777dcc2808669ab815a039af" ], [ "MiniParse.Impl.Base.coerce_parser_impl", @@ -97,7 +97,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "149aa5529c973a760a1c8c2ec67735a5" + "258a0a055887966d78bf945156941301" ], [ "MiniParse.Impl.Base.serializer_impl", @@ -122,7 +122,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "e4e377a7db00b4aaedf707926f260426" + "9c2f571efcd36b9bd4c8a40bc87008af" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Impl.Combinators.fst.hints b/examples/miniparse/MiniParse.Impl.Combinators.fst.hints index 61afd1822bd..59230e70475 100644 --- a/examples/miniparse/MiniParse.Impl.Combinators.fst.hints +++ b/examples/miniparse/MiniParse.Impl.Combinators.fst.hints @@ -60,7 +60,7 @@ "unit_typing" ], 0, - "59c384f5aea784d25a5300fe1a5b20f6" + "0106a5b1c8fd8a6f358c19887407bbb4" ], [ "MiniParse.Impl.Combinators.serialize_empty_impl", @@ -145,7 +145,7 @@ "typing_Prims.pow2", "unit_inversion", "unit_typing" ], 0, - "d41e9e7b3a21a0732ae121a6395a00ac" + "3c3210fbe3b1f16e1f6a4ec1e0efa6a6" ], [ "MiniParse.Impl.Combinators.parse_and_then_impl", @@ -240,7 +240,7 @@ "unit_typing" ], 0, - "f6160ec35bb2de1d25390c366b14c3c6" + "3b7f1f94b686c98e7bf775935d984a30" ], [ "MiniParse.Impl.Combinators.parse_nondep_then_impl", @@ -285,7 +285,7 @@ "unit_typing" ], 0, - "8b44fd0116a1176ba0384faae4e5956f" + "446509fcb2fe37ecf487a9fd8a7462cf" ], [ "MiniParse.Impl.Combinators.seq_append_slice", @@ -335,7 +335,7 @@ "unit_typing" ], 0, - "00fe890ab98a84a871f1c84aaf9a1cf0" + "d3aba607bfedbab5c0e9c8b811e028e0" ], [ "MiniParse.Impl.Combinators.serialize_nondep_then_impl", @@ -453,7 +453,7 @@ "unit_typing" ], 0, - "430e4e83b5b411db3aebdbb51702068a" + "3192f60446eb42f88ca449e72a319e3d" ], [ "MiniParse.Impl.Combinators.parse_synth_impl", @@ -519,7 +519,7 @@ "unit_typing" ], 0, - "2567827b40b4efa1221ae7179ae83f0c" + "03a15b672d1d24b7dfa66027fe4b16ca" ], [ "MiniParse.Impl.Combinators.serialize_synth_impl", @@ -545,7 +545,7 @@ "unit_inversion" ], 0, - "7132ecc5f3de407113f569920da79772" + "064810f795a8b4c4db97694b0d57320a" ], [ "MiniParse.Impl.Combinators.serialize_synth_impl'", @@ -556,12 +556,12 @@ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", "equation_Prims.l_and", "equation_Prims.squash", "fuel_guarded_inversion_MiniParse.Spec.Base.serializer_spec", - "l_and-interp", "l_quant_interp__4530", + "l_and-interp", "l_quant_interp__4532", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5", "unit_inversion" ], 0, - "e5e592693d7b48ff89f51a01b6f204c2" + "23cb7d5fb1b9d5a466f952ea7808d9b4" ], [ "MiniParse.Impl.Combinators.parse_filter_impl", @@ -638,7 +638,7 @@ "unit_typing" ], 0, - "1f7bb19b033f1f5c366f43691d6fecc2" + "3800e07b174709d5925fa458d3db870f" ], [ "MiniParse.Impl.Combinators.serialize_filter_impl", @@ -659,7 +659,7 @@ "token_correspondence_MiniParse.Spec.Base.__proj__Serializer__item__f" ], 0, - "c1526dd4d401de36ffc1a178e8ef5b75" + "4e06751c2d3cc768ee34b059b51e6e08" ], [ "MiniParse.Impl.Combinators.make_constant_size_parser_impl", @@ -677,7 +677,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "ed20d8113ae2ca462aebebf60261193d" + "205540f94e6c8b22970d18b89fecf0b6" ], [ "MiniParse.Impl.Combinators.make_constant_size_parser_impl", @@ -776,7 +776,7 @@ "unit_typing" ], 0, - "4a7c2f5e2647da0e8d97693e1ea784c6" + "f232137497ebd0ac15478a7c980cc1d0" ], [ "MiniParse.Impl.Combinators.make_total_constant_size_parser_impl", @@ -794,7 +794,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "53019a9ccc8bf947d8d374e205e4ed7c" + "53b23de0672de3e898dce56740f3eef4" ], [ "MiniParse.Impl.Combinators.make_total_constant_size_parser_impl", @@ -887,7 +887,7 @@ "unit_typing" ], 0, - "d6c8d266e4586934aaa1adc8ffbada72" + "f576c811eb95a6aaf315e6c9dd9b6ed1" ], [ "MiniParse.Impl.Combinators.parse_ret_impl", @@ -948,7 +948,7 @@ "unit_typing" ], 0, - "7a2f9ce9e3b251ff0103b15eab525455" + "ca113167d1b2728949302f859423742d" ], [ "MiniParse.Impl.Combinators.serialize_empty_impl", @@ -1034,7 +1034,7 @@ "typing_Prims.pow2", "unit_inversion", "unit_typing" ], 0, - "9115d5e69fe233ca3f82861cc30e2e54" + "3068d4920001dc3aa0450177e920e5a3" ], [ "MiniParse.Impl.Combinators.parse_and_then_impl", @@ -1139,7 +1139,7 @@ "unit_typing" ], 0, - "6d7751a304930e544780ab955115e881" + "07722a8b49feddef617df06ced5f39f3" ], [ "MiniParse.Impl.Combinators.parse_and_then_impl", @@ -1153,7 +1153,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "f4871adb78fae8b45d4fbc9291b3a0ce" + "df3736ef9393032145f5b827d1bb4672" ], [ "MiniParse.Impl.Combinators.parse_nondep_then_impl", @@ -1198,7 +1198,7 @@ "unit_typing" ], 0, - "40e21dbcb8be9568e1bc88f518793dfb" + "2b7fbb539a3169caf09010adc520d86e" ], [ "MiniParse.Impl.Combinators.seq_append_slice", @@ -1224,7 +1224,7 @@ "unit_typing" ], 0, - "b25b2aff9f3c088763ac8e3ad0512d8b" + "02510e2ef5f8aec2f69276cbaf7dad31" ], [ "MiniParse.Impl.Combinators.serialize_nondep_then_impl", @@ -1342,7 +1342,7 @@ "unit_typing" ], 0, - "f3f0238cf9f5aa3c652a782c29aa32a8" + "1646ce8a5092896070e30212311eef72" ], [ "MiniParse.Impl.Combinators.parse_synth_impl", @@ -1408,7 +1408,7 @@ "unit_typing" ], 0, - "f832bd3fce1b3967df972a5a9da4701a" + "03082cefe51b11164a7ad594b6dbbcdf" ], [ "MiniParse.Impl.Combinators.parse_synth_impl", @@ -1420,7 +1420,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "e1f1b2978334ae87c1791bf3d8142fd0" + "0819b1b618129663a760ff72f430101e" ], [ "MiniParse.Impl.Combinators.serialize_synth_impl", @@ -1446,7 +1446,7 @@ "unit_inversion" ], 0, - "8ebc7ead0fd898fd0d7cdf0342384413" + "0d214d6f25f5c739a8d250c7a31ccbe0" ], [ "MiniParse.Impl.Combinators.serialize_synth_impl", @@ -1459,7 +1459,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "68611b8a7b3757be041f736331fbd1de" + "9fc67485044f2c2e8125e273adf45915" ], [ "MiniParse.Impl.Combinators.serialize_synth_impl'", @@ -1470,12 +1470,12 @@ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", "equation_Prims.l_and", "equation_Prims.squash", "fuel_guarded_inversion_MiniParse.Spec.Base.serializer_spec", - "l_and-interp", "l_quant_interp__4953", + "l_and-interp", "l_quant_interp__4955", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5", "unit_inversion" ], 0, - "31ce8882daf991a36aaa0c77b8d5b832" + "e1a599b7c8665b31659807902a931fa4" ], [ "MiniParse.Impl.Combinators.serialize_synth_impl'", @@ -1488,7 +1488,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "93138fafc43dbbbe4916bb716e87983b" + "6499f1ab61c90be2ba70d81cf90100e7" ], [ "MiniParse.Impl.Combinators.parse_filter_impl", @@ -1565,7 +1565,7 @@ "unit_typing" ], 0, - "6c67decebba4243b14e411a488ff75f4" + "058dd6ffdf14090b5aec563fdb312f90" ], [ "MiniParse.Impl.Combinators.serialize_filter_impl", @@ -1586,7 +1586,7 @@ "token_correspondence_MiniParse.Spec.Base.__proj__Serializer__item__f" ], 0, - "30e58552497ffda633d1cc9891ce7aa4" + "4d7d5361ac6693bfb479c1b103959cf2" ], [ "MiniParse.Impl.Combinators.make_constant_size_parser_impl", @@ -1604,7 +1604,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "1cbc44270c92a4a5e9daa2bc7f4cadd6" + "2e65ca6745f646da1916114dba457f95" ], [ "MiniParse.Impl.Combinators.make_constant_size_parser_impl", @@ -1703,7 +1703,7 @@ "unit_typing" ], 0, - "09b76c8738dea6a5678eab41894b3245" + "f5cbff89c713608dad0209bb95e4ffa9" ], [ "MiniParse.Impl.Combinators.make_constant_size_parser_impl", @@ -1723,7 +1723,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "8bffad598af8fde377b6e59afaab04cc" + "7f5ee88e1ab10e86129fdf0b1bbb8eb6" ], [ "MiniParse.Impl.Combinators.make_total_constant_size_parser_impl", @@ -1741,7 +1741,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "2faa6ef9dda23ebaa6dfcfa90783b7f8" + "75d1b27816802d542ccbf34dbdcdaa69" ], [ "MiniParse.Impl.Combinators.make_total_constant_size_parser_impl", @@ -1834,7 +1834,7 @@ "unit_typing" ], 0, - "4ce44c13af0c9bb11b094ffd7fec3c3e" + "3f4861d3e62e84edab60a8ddd4ee088a" ], [ "MiniParse.Impl.Combinators.make_total_constant_size_parser_impl", @@ -1854,7 +1854,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "ffcac91162eea2001a89ae021dbec75d" + "1aa9fdb9c619c791119ecdcd618294d5" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Impl.Int.fst.hints b/examples/miniparse/MiniParse.Impl.Int.fst.hints index 12e4a16a82b..fb086ae8157 100644 --- a/examples/miniparse/MiniParse.Impl.Int.fst.hints +++ b/examples/miniparse/MiniParse.Impl.Int.fst.hints @@ -32,7 +32,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "e165e0c4d852991b831d49a9a97bc8f9" + "54b271bebeb6c144f77be8c87f3d840f" ], [ "MiniParse.Impl.Int.serialize_u8_impl", @@ -150,7 +150,7 @@ "unit_typing" ], 0, - "0cbf2c58c47b7fb2b2f17e69a2c44951" + "cc1375bdcca407e638d9d8ab0da357cf" ], [ "MiniParse.Impl.Int.parse_u16_impl", @@ -173,7 +173,7 @@ "refinement_interpretation_MiniParse.Spec.Int_Tm_refine_ac00760bd8a5172a9a770c310fccc248" ], 0, - "4d95c19bcd90de976cb0ed008b144766" + "92c8a99aeb0c46d02aabce17802afef8" ], [ "MiniParse.Impl.Int.serialize_u16_impl", @@ -317,7 +317,7 @@ "unit_typing" ], 0, - "1d07d45436bb8690de1bbf8414f82e9c" + "bffb3972a7a6ce09e13de0dfcc970aa7" ], [ "MiniParse.Impl.Int.parse_bounded_u16_impl", @@ -448,7 +448,7 @@ "typing_MiniParse.Spec.Int.parse_bounded_u16", "unit_typing" ], 0, - "796ef0ef6a707d8accf4671299428901" + "59db24905eb8d75871ea5f2dc91e9ff9" ], [ "MiniParse.Impl.Int.serialize_bounded_u16_impl", @@ -479,7 +479,7 @@ "token_correspondence_MiniParse.Spec.Base.__proj__Serializer__item__f" ], 0, - "a23a6f43191fc99a5e7e46f74ff13bf5" + "2d4468613436a565689f9d47e61959e4" ], [ "MiniParse.Impl.Int.parse_u8_impl", @@ -512,7 +512,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "9e4057fddcb51c7c5e6c3863f7aa3012" + "50c47c1637b2b6f34ec98852e2108895" ], [ "MiniParse.Impl.Int.serialize_u8_impl", @@ -631,7 +631,7 @@ "unit_typing" ], 0, - "ffe36449c6b911033516a0307201d6a6" + "1d6af7a47c1175677520c9d3c979106a" ], [ "MiniParse.Impl.Int.parse_u16_impl", @@ -654,7 +654,7 @@ "refinement_interpretation_MiniParse.Spec.Int_Tm_refine_ac00760bd8a5172a9a770c310fccc248" ], 0, - "a22cd4d005ad19988c4d3dd17adf6832" + "8cdf3a5e84d0e8c7a366f68c2c7da564" ], [ "MiniParse.Impl.Int.serialize_u16_impl", @@ -800,7 +800,7 @@ "unit_typing" ], 0, - "7bcb1387287bb393a4d46d1fdd0076b4" + "241fb9b7f570dbd89e3b8bb431ab3c70" ], [ "MiniParse.Impl.Int.parse_bounded_u16_impl", @@ -932,7 +932,7 @@ "typing_MiniParse.Spec.Int.parse_bounded_u16", "unit_typing" ], 0, - "2d39e49c9e892a47ad681d4542f8cec5" + "2395db3f64252301acec6aec27a2ee35" ], [ "MiniParse.Impl.Int.serialize_bounded_u16_impl", @@ -963,7 +963,7 @@ "token_correspondence_MiniParse.Spec.Base.__proj__Serializer__item__f" ], 0, - "c180175ebe4909a710cb8f221568c084" + "3bb36f6ed4e2077bb881e0312e66b822" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Impl.List.fst.hints b/examples/miniparse/MiniParse.Impl.List.fst.hints index 6432dadb7bd..1958824fdca 100644 --- a/examples/miniparse/MiniParse.Impl.List.fst.hints +++ b/examples/miniparse/MiniParse.Impl.List.fst.hints @@ -36,7 +36,7 @@ "unit_typing" ], 0, - "6752ccf1016785f74f465c14612d5d5d" + "32ba5ada9020bb2fdfb884b1c07fede9" ], [ "MiniParse.Impl.List.list_assoc_append", @@ -60,7 +60,7 @@ "token_correspondence_FStar.List.Tot.Base.op_At" ], 0, - "3a386fb201e20d7c479d650c44fbded5" + "0c633cdc540f2f716c3342d060329ee3" ], [ "MiniParse.Impl.List.parse_nlist_impl_inv_false_intro", @@ -78,7 +78,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "41a17d294d156e4aee533116eca087bc" + "4e169ecf7c0be9690d825072978be5eb" ], [ "MiniParse.Impl.List.parse_nlist_impl_inv_false_intro", @@ -183,7 +183,7 @@ "unit_typing" ], 0, - "09a8efa272c3d7b01727c4f6f1ccc3c8" + "a032462a5156d955016621784b0f2f86" ], [ "MiniParse.Impl.List.parse_nlist_impl_body", @@ -196,7 +196,7 @@ "refinement_interpretation_MiniParse.Impl.List_Tm_refine_8d69b5d507ff95b91fc5e7b55106875a" ], 0, - "6b49bb5a5b969477e3a5a59b69dd19b6" + "c0f0c7ef1c5a77f53913f1b1d1c47abf" ], [ "MiniParse.Impl.List.parse_nlist_impl_body", @@ -358,7 +358,7 @@ "typing_MiniParse.Spec.List.parse_nlist", "unit_typing" ], 0, - "8a495cd87da856863462ebc80da6a64a" + "5e275d30363ff3ccb1d4cf0982d59782" ], [ "MiniParse.Impl.List.list_rev", @@ -389,7 +389,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "8d08e07331960ff7ff7a15e1908ca5f0" + "86629904e1ee656f98313d2b911598c0" ], [ "MiniParse.Impl.List.parse_nlist_impl", @@ -398,7 +398,7 @@ 1, [ "@query" ], 0, - "04d0de914ad7929aa2bc833f84f7ebd0" + "fc56a7abd31aa1699095b29bb567b858" ], [ "MiniParse.Impl.List.parse_nlist_impl", @@ -416,6 +416,7 @@ "@fuel_irrelevance_FStar.List.Tot.Base.length.fuel_instrumented", "@fuel_irrelevance_Prims.pow2.fuel_instrumented", "@query", "FStar.Monotonic.HyperStack_pretyping_cd115f719b336f9a8366e4b68a41d001", + "FStar.Pervasives.Native_pretyping_b53dbd183c526bc5d0f20d7b966ae125", "FStar.UInt32_pretyping_041e3a67a2d2b51fd702f1f88cfc3b44", "MiniParse.Spec.Combinators_interpretation_Tm_arrow_2d0cb30a46b94c9495a3fd95ee1abbd6", "Prims_interpretation_Tm_arrow_9cb3c953faf527c316d427b2ce8bd81b", @@ -425,12 +426,14 @@ "assumption_Prims.HasEq_int", "b2t_def", "bool_inversion", "bool_typing", "constructor_distinct_FStar.Pervasives.Native.None", "constructor_distinct_FStar.Pervasives.Native.Some", - "constructor_distinct_Prims.Nil", "constructor_distinct_Tm_unit", + "constructor_distinct_Prims.Cons", "constructor_distinct_Prims.Nil", + "constructor_distinct_Tm_unit", "data_elim_FStar.Pervasives.Native.Mktuple2", "data_elim_FStar.Pervasives.Native.Some", - "data_elim_MiniParse.Spec.Base.Serializer", + "data_elim_MiniParse.Spec.Base.Serializer", "data_elim_Prims.Cons", "data_typing_intro_Prims.Nil@tok", "disc_equation_FStar.Pervasives.Native.None", + "disc_equation_FStar.Pervasives.Native.Some", "equation_FStar.HyperStack.ST.equal_domains", "equation_FStar.HyperStack.ST.inline_stack_inv", "equation_FStar.List.Tot.Base.op_At", @@ -475,6 +478,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option", "fuel_guarded_inversion_FStar.Pervasives.Native.tuple2", "fuel_guarded_inversion_MiniParse.Spec.Base.parser_spec", + "fuel_guarded_inversion_Prims.list", "function_token_typing_FStar.Monotonic.Heap.emp", "function_token_typing_FStar.Monotonic.Heap.heap", "function_token_typing_FStar.Monotonic.HyperHeap.rid", @@ -491,6 +495,7 @@ "int_inversion", "int_typing", "interpretation_LowStar.Buffer_Tm_abs_d359dc64ac5a79b32b9828a25bf0bd72", "interpretation_MiniParse.Spec.Combinators_Tm_abs_c5c8acf53d4399faf3399288d7fe5742", + "kinding_FStar.Pervasives.Native.tuple2@tok", "kinding_Prims.list@tok", "lemma_FStar.HyperStack.ST.lemma_same_refs_in_all_regions_elim", "lemma_FStar.HyperStack.ST.lemma_same_refs_in_all_regions_intro", @@ -502,15 +507,14 @@ "lemma_FStar.Map.lemma_UpdDomain", "lemma_FStar.Monotonic.HyperStack.lemma_mk_mem__projectors", "lemma_FStar.Monotonic.HyperStack.lemma_tip_top_smt", + "lemma_FStar.Pervasives.invertOption", "lemma_FStar.Seq.Base.lemma_index_create", - "lemma_FStar.Seq.Base.lemma_len_slice", "lemma_FStar.Seq.Properties.slice_length", "lemma_FStar.Set.lemma_equal_elim", "lemma_FStar.Set.lemma_equal_intro", "lemma_FStar.Set.mem_complement", "lemma_FStar.Set.mem_intersect", "lemma_FStar.Set.mem_singleton", "lemma_FStar.Set.mem_union", - "lemma_FStar.UInt.pow2_values", "lemma_FStar.UInt32.uv_inv", - "lemma_FStar.UInt32.vu_inv", + "lemma_FStar.UInt.pow2_values", "lemma_FStar.UInt32.vu_inv", "lemma_LowStar.Monotonic.Buffer.as_seq_gsub", "lemma_LowStar.Monotonic.Buffer.fresh_frame_modifies_inert", "lemma_LowStar.Monotonic.Buffer.len_gsub", @@ -560,7 +564,9 @@ "projection_inverse_FStar.Pervasives.Native.Some_a", "projection_inverse_FStar.Pervasives.Native.Some_v", "projection_inverse_MiniParse.Spec.Base.Parser_f", - "projection_inverse_Prims.Nil_a", + "projection_inverse_Prims.Cons_a", + "projection_inverse_Prims.Cons_hd", + "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a", "refinement_interpretation_FStar.List.Tot.Properties_Tm_refine_fbb3412f12fd58a91571022d7c9fa36d", "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", "refinement_interpretation_FStar.Seq.Base_Tm_refine_5514fbe9e08dfda40f950a7b9f1b2b98", @@ -570,7 +576,6 @@ "refinement_interpretation_FStar.UInt32_Tm_refine_6c25b42778726de94cd4dac42edb4860", "refinement_interpretation_FStar.UInt32_Tm_refine_6c5b5bfca8736b34d6f700f752d1df10", "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", - "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_4fa8e2dd96f8bb1e23e6574326e9e019", "refinement_interpretation_MiniParse.Impl.Combinators_Tm_refine_15d901d34c4a684eec9e5c2f749ce352", "refinement_interpretation_MiniParse.Impl.List_Tm_refine_01e2193142610fbe981196d2824242ac", "refinement_interpretation_MiniParse.Impl.List_Tm_refine_51063a777a1e9a0f9bc59c6793064953", @@ -584,6 +589,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", "refinement_interpretation_Prims_Tm_refine_c16bc1b61f58b349bf6fc1c94dcaf83b", "refinement_kinding_FStar.List.Tot.Properties_Tm_refine_fbb3412f12fd58a91571022d7c9fa36d", + "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b", "refinement_kinding_MiniParse.Impl.List_Tm_refine_6c04604a6818a270d2fa48a388019163", "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented", "true_interp", "typing_FStar.List.Tot.Base.rev", @@ -595,11 +601,11 @@ "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.Monotonic.HyperStack.live_region", "typing_FStar.Monotonic.HyperStack.remove_elt", - "typing_FStar.Seq.Base.length", "typing_FStar.Set.complement", - "typing_FStar.Set.mem", "typing_FStar.Set.singleton", - "typing_FStar.Set.union", "typing_FStar.UInt.fits", - "typing_FStar.UInt32.sub", "typing_FStar.UInt32.v", - "typing_LowStar.Buffer.trivial_preorder", + "typing_FStar.Seq.Base.length", "typing_FStar.Seq.Base.slice", + "typing_FStar.Set.complement", "typing_FStar.Set.mem", + "typing_FStar.Set.singleton", "typing_FStar.Set.union", + "typing_FStar.UInt.fits", "typing_FStar.UInt32.sub", + "typing_FStar.UInt32.v", "typing_LowStar.Buffer.trivial_preorder", "typing_LowStar.Monotonic.Buffer.as_addr", "typing_LowStar.Monotonic.Buffer.as_seq", "typing_LowStar.Monotonic.Buffer.frameOf", @@ -610,7 +616,6 @@ "typing_LowStar.Monotonic.Buffer.loc_buffer", "typing_LowStar.Monotonic.Buffer.loc_regions", "typing_LowStar.Monotonic.Buffer.loc_union", - "typing_LowStar.Monotonic.Buffer.mgsub", "typing_MiniParse.Spec.Base.parse", "typing_MiniParse.Spec.Combinators_Tm_abs_5d6f2d5bebd6034a03a4471fa6682fb3", "typing_MiniParse.Spec.List.nlist", @@ -618,7 +623,7 @@ "typing_MiniParse.Spec.List.parse_nlist", "unit_typing" ], 0, - "5d67af7ca5ffcaf29e0fcb0119e17513" + "b16eff850d830c7f11d990feb4ec778b" ], [ "MiniParse.Impl.List.serialize_nlist_impl_inv", @@ -646,7 +651,7 @@ "unit_typing" ], 0, - "355bc4cb447e908b400b4abd2e2beed5" + "a926826b9303b9eaa457f57d23091350" ], [ "MiniParse.Impl.List.serialize_nlist_impl_body", @@ -791,7 +796,7 @@ "typing_MiniParse.Spec.List.serialize_nlist", "unit_typing" ], 0, - "f2cc1c5c970abdef2fe4553f43559412" + "1a794967c69f509ae202228ac91891c0" ], [ "MiniParse.Impl.List.serialize_nlist_impl", @@ -800,7 +805,7 @@ 1, [ "@query" ], 0, - "1a11fdff126d963e2d19f25fb863522c" + "d65cc64552695999cc73f192dc08d303" ], [ "MiniParse.Impl.List.serialize_nlist_impl", @@ -996,7 +1001,7 @@ "typing_MiniParse.Spec.List.serialize_nlist", "unit_typing" ], 0, - "12f2f90bbdc343824893cfa402b780ff" + "c3482b9873d0d4f39c0fa4002786a0a1" ], [ "MiniParse.Impl.List.parse_nlist_impl_inv", @@ -1033,7 +1038,7 @@ "unit_typing" ], 0, - "a51b3ed96cff3f03729655d708f3cb5b" + "4b139945f4608c1c259716a6dd33c068" ], [ "MiniParse.Impl.List.parse_nlist_impl_inv_false_intro", @@ -1094,7 +1099,7 @@ "unit_typing" ], 0, - "75b20ea088ba7444a56747b8067456c5" + "f280f2eddeb0ccc94144ac12f4c31a84" ], [ "MiniParse.Impl.List.parse_nlist_impl_body", @@ -1107,7 +1112,7 @@ "refinement_interpretation_MiniParse.Impl.List_Tm_refine_8d69b5d507ff95b91fc5e7b55106875a" ], 0, - "70b2602dfe7a11bcc2733a2812bcac5f" + "91b85bd974c87a290bc5ed4c97a75927" ], [ "MiniParse.Impl.List.list_rev", @@ -1138,7 +1143,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "d288dd1a9b944f20bc426816ae453798" + "8623ccf8395140bb8d8d847c83de7e2f" ], [ "MiniParse.Impl.List.parse_nlist_impl", @@ -1147,7 +1152,7 @@ 1, [ "@query" ], 0, - "eb76427c0bc2f20710b922508a10bf9f" + "87e8fb4a051eb03deacccb1bbe1b4836" ], [ "MiniParse.Impl.List.parse_nlist_impl", @@ -1165,6 +1170,7 @@ "@fuel_irrelevance_FStar.List.Tot.Base.length.fuel_instrumented", "@fuel_irrelevance_Prims.pow2.fuel_instrumented", "@query", "FStar.Monotonic.HyperStack_pretyping_cd115f719b336f9a8366e4b68a41d001", + "FStar.Pervasives.Native_pretyping_b53dbd183c526bc5d0f20d7b966ae125", "FStar.UInt32_pretyping_041e3a67a2d2b51fd702f1f88cfc3b44", "MiniParse.Spec.Combinators_interpretation_Tm_arrow_2d0cb30a46b94c9495a3fd95ee1abbd6", "Prims_interpretation_Tm_arrow_9cb3c953faf527c316d427b2ce8bd81b", @@ -1174,12 +1180,14 @@ "assumption_Prims.HasEq_int", "b2t_def", "bool_inversion", "bool_typing", "constructor_distinct_FStar.Pervasives.Native.None", "constructor_distinct_FStar.Pervasives.Native.Some", - "constructor_distinct_Prims.Nil", "constructor_distinct_Tm_unit", + "constructor_distinct_Prims.Cons", "constructor_distinct_Prims.Nil", + "constructor_distinct_Tm_unit", "data_elim_FStar.Pervasives.Native.Mktuple2", "data_elim_FStar.Pervasives.Native.Some", - "data_elim_MiniParse.Spec.Base.Serializer", + "data_elim_MiniParse.Spec.Base.Serializer", "data_elim_Prims.Cons", "data_typing_intro_Prims.Nil@tok", "disc_equation_FStar.Pervasives.Native.None", + "disc_equation_FStar.Pervasives.Native.Some", "equation_FStar.HyperStack.ST.equal_domains", "equation_FStar.HyperStack.ST.inline_stack_inv", "equation_FStar.List.Tot.Base.op_At", @@ -1224,6 +1232,7 @@ "fuel_guarded_inversion_FStar.Pervasives.Native.option", "fuel_guarded_inversion_FStar.Pervasives.Native.tuple2", "fuel_guarded_inversion_MiniParse.Spec.Base.parser_spec", + "fuel_guarded_inversion_Prims.list", "function_token_typing_FStar.Monotonic.Heap.emp", "function_token_typing_FStar.Monotonic.Heap.heap", "function_token_typing_FStar.Monotonic.HyperHeap.rid", @@ -1240,6 +1249,7 @@ "int_inversion", "int_typing", "interpretation_LowStar.Buffer_Tm_abs_d359dc64ac5a79b32b9828a25bf0bd72", "interpretation_MiniParse.Spec.Combinators_Tm_abs_c5c8acf53d4399faf3399288d7fe5742", + "kinding_FStar.Pervasives.Native.tuple2@tok", "kinding_Prims.list@tok", "lemma_FStar.HyperStack.ST.lemma_same_refs_in_all_regions_elim", "lemma_FStar.HyperStack.ST.lemma_same_refs_in_all_regions_intro", @@ -1251,15 +1261,14 @@ "lemma_FStar.Map.lemma_UpdDomain", "lemma_FStar.Monotonic.HyperStack.lemma_mk_mem__projectors", "lemma_FStar.Monotonic.HyperStack.lemma_tip_top_smt", + "lemma_FStar.Pervasives.invertOption", "lemma_FStar.Seq.Base.lemma_index_create", - "lemma_FStar.Seq.Base.lemma_len_slice", "lemma_FStar.Seq.Properties.slice_length", "lemma_FStar.Set.lemma_equal_elim", "lemma_FStar.Set.lemma_equal_intro", "lemma_FStar.Set.mem_complement", "lemma_FStar.Set.mem_intersect", "lemma_FStar.Set.mem_singleton", "lemma_FStar.Set.mem_union", - "lemma_FStar.UInt.pow2_values", "lemma_FStar.UInt32.uv_inv", - "lemma_FStar.UInt32.vu_inv", + "lemma_FStar.UInt.pow2_values", "lemma_FStar.UInt32.vu_inv", "lemma_LowStar.Monotonic.Buffer.as_seq_gsub", "lemma_LowStar.Monotonic.Buffer.fresh_frame_modifies_inert", "lemma_LowStar.Monotonic.Buffer.len_gsub", @@ -1309,7 +1318,9 @@ "projection_inverse_FStar.Pervasives.Native.Some_a", "projection_inverse_FStar.Pervasives.Native.Some_v", "projection_inverse_MiniParse.Spec.Base.Parser_f", - "projection_inverse_Prims.Nil_a", + "projection_inverse_Prims.Cons_a", + "projection_inverse_Prims.Cons_hd", + "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a", "refinement_interpretation_FStar.List.Tot.Properties_Tm_refine_fbb3412f12fd58a91571022d7c9fa36d", "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", "refinement_interpretation_FStar.Seq.Base_Tm_refine_5514fbe9e08dfda40f950a7b9f1b2b98", @@ -1319,7 +1330,6 @@ "refinement_interpretation_FStar.UInt32_Tm_refine_6c25b42778726de94cd4dac42edb4860", "refinement_interpretation_FStar.UInt32_Tm_refine_6c5b5bfca8736b34d6f700f752d1df10", "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", - "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_4fa8e2dd96f8bb1e23e6574326e9e019", "refinement_interpretation_MiniParse.Impl.Combinators_Tm_refine_15d901d34c4a684eec9e5c2f749ce352", "refinement_interpretation_MiniParse.Impl.List_Tm_refine_01e2193142610fbe981196d2824242ac", "refinement_interpretation_MiniParse.Impl.List_Tm_refine_51063a777a1e9a0f9bc59c6793064953", @@ -1333,6 +1343,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", "refinement_interpretation_Prims_Tm_refine_c16bc1b61f58b349bf6fc1c94dcaf83b", "refinement_kinding_FStar.List.Tot.Properties_Tm_refine_fbb3412f12fd58a91571022d7c9fa36d", + "refinement_kinding_FStar.Seq.Base_Tm_refine_cd046bc4a887ee7e1b05946e0bf5772b", "refinement_kinding_MiniParse.Impl.List_Tm_refine_6c04604a6818a270d2fa48a388019163", "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented", "true_interp", "typing_FStar.List.Tot.Base.rev", @@ -1344,11 +1355,11 @@ "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.Monotonic.HyperStack.live_region", "typing_FStar.Monotonic.HyperStack.remove_elt", - "typing_FStar.Seq.Base.length", "typing_FStar.Set.complement", - "typing_FStar.Set.mem", "typing_FStar.Set.singleton", - "typing_FStar.Set.union", "typing_FStar.UInt.fits", - "typing_FStar.UInt32.sub", "typing_FStar.UInt32.v", - "typing_LowStar.Buffer.trivial_preorder", + "typing_FStar.Seq.Base.length", "typing_FStar.Seq.Base.slice", + "typing_FStar.Set.complement", "typing_FStar.Set.mem", + "typing_FStar.Set.singleton", "typing_FStar.Set.union", + "typing_FStar.UInt.fits", "typing_FStar.UInt32.sub", + "typing_FStar.UInt32.v", "typing_LowStar.Buffer.trivial_preorder", "typing_LowStar.Monotonic.Buffer.as_addr", "typing_LowStar.Monotonic.Buffer.as_seq", "typing_LowStar.Monotonic.Buffer.frameOf", @@ -1359,7 +1370,6 @@ "typing_LowStar.Monotonic.Buffer.loc_buffer", "typing_LowStar.Monotonic.Buffer.loc_regions", "typing_LowStar.Monotonic.Buffer.loc_union", - "typing_LowStar.Monotonic.Buffer.mgsub", "typing_MiniParse.Spec.Base.parse", "typing_MiniParse.Spec.Combinators_Tm_abs_5d6f2d5bebd6034a03a4471fa6682fb3", "typing_MiniParse.Spec.List.nlist", @@ -1367,7 +1377,7 @@ "typing_MiniParse.Spec.List.parse_nlist", "unit_typing" ], 0, - "21d73612ee0857c4cc82ad0b6e0a4fcf" + "c518397f2cbec40470518c8c726eddca" ], [ "MiniParse.Impl.List.parse_nlist_impl", @@ -1376,7 +1386,7 @@ 1, [ "@query" ], 0, - "9df19eccdf6420bf3fa9e68967141e5f" + "f92bc4fbab444b555b4edd48f46a3b93" ], [ "MiniParse.Impl.List.serialize_nlist_impl_inv", @@ -1404,7 +1414,7 @@ "unit_typing" ], 0, - "236c6df5e89fbaa77c2838c227ad3fcd" + "0b0f086eb98b7896855112fd566ef99b" ], [ "MiniParse.Impl.List.serialize_nlist_impl_body", @@ -1417,7 +1427,7 @@ "refinement_interpretation_MiniParse.Impl.List_Tm_refine_8d69b5d507ff95b91fc5e7b55106875a" ], 0, - "92fdb65afa919f75840c79123892793a" + "3173cd080915ebb1fde490a8b96caa3a" ], [ "MiniParse.Impl.List.serialize_nlist_impl", @@ -1426,7 +1436,7 @@ 1, [ "@query" ], 0, - "4f26cb40d91721c8cb890fee1053cd2b" + "2ce4b5af52cee145c3e3e39d5cb6e455" ], [ "MiniParse.Impl.List.serialize_nlist_impl", @@ -1435,9 +1445,7 @@ 1, [ "@MaxFuel_assumption", "@MaxIFuel_assumption", - "@fuel_correspondence_FStar.List.Tot.Base.length.fuel_instrumented", "@fuel_correspondence_MiniParse.Spec.List.serialize_nlist_.fuel_instrumented", - "@fuel_irrelevance_FStar.List.Tot.Base.length.fuel_instrumented", "@query", "FStar.Monotonic.HyperStack_pretyping_cd115f719b336f9a8366e4b68a41d001", "FStar.UInt32_pretyping_041e3a67a2d2b51fd702f1f88cfc3b44", @@ -1449,8 +1457,7 @@ "assumption_Prims.HasEq_int", "b2t_def", "bool_inversion", "bool_typing", "constructor_distinct_FStar.Pervasives.Native.None", "constructor_distinct_FStar.Pervasives.Native.Some", - "constructor_distinct_Tm_unit", - "data_elim_MiniParse.Spec.Base.Serializer", "data_elim_Prims.Cons", + "data_elim_MiniParse.Spec.Base.Serializer", "disc_equation_FStar.Pervasives.Native.None", "disc_equation_FStar.Pervasives.Native.Some", "equation_FStar.HyperStack.ST.equal_domains", @@ -1484,10 +1491,8 @@ "equation_MiniParse.Spec.List.nlist", "equation_Prims.eqtype", "equation_Prims.l_True", "equation_Prims.logical", "equation_Prims.nat", - "equation_with_fuel_FStar.List.Tot.Base.length.fuel_instrumented", "equation_with_fuel_MiniParse.Spec.List.serialize_nlist_.fuel_instrumented", "fuel_guarded_inversion_MiniParse.Spec.Base.serializer_spec", - "fuel_guarded_inversion_Prims.list", "function_token_typing_FStar.Monotonic.Heap.emp", "function_token_typing_FStar.Monotonic.Heap.heap", "function_token_typing_FStar.Monotonic.HyperHeap.rid", @@ -1525,7 +1530,6 @@ "lemma_FStar.Set.mem_complement", "lemma_FStar.Set.mem_intersect", "lemma_FStar.Set.mem_singleton", "lemma_FStar.Set.mem_union", "lemma_FStar.UInt32.vu_inv", - "lemma_LowStar.Monotonic.Buffer.as_seq_gsub", "lemma_LowStar.Monotonic.Buffer.fresh_frame_loc_not_unused_in_disjoint", "lemma_LowStar.Monotonic.Buffer.fresh_frame_modifies_inert", "lemma_LowStar.Monotonic.Buffer.len_gsub", @@ -1598,7 +1602,6 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", "refinement_interpretation_Prims_Tm_refine_c16bc1b61f58b349bf6fc1c94dcaf83b", "refinement_kinding_MiniParse.Impl.List_Tm_refine_6c04604a6818a270d2fa48a388019163", - "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented", "token_correspondence_MiniParse.Spec.Base.__proj__Serializer__item__f", "true_interp", "typing_FStar.Map.contains", "typing_FStar.Map.domain", "typing_FStar.Map.restrict", @@ -1629,7 +1632,7 @@ "typing_MiniParse.Spec.List.serialize_nlist", "unit_typing" ], 0, - "4ed81bd61766e128a1ad9e1af2388b74" + "adabe1d95202fd5495a6722e64a884fe" ], [ "MiniParse.Impl.List.serialize_nlist_impl", @@ -1638,7 +1641,7 @@ 1, [ "@query" ], 0, - "d0717f9f4879b1d8f0c2333c34b2fff3" + "c096304829e09e90da6a2c03a9a19f44" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Impl.TSum.fst.hints b/examples/miniparse/MiniParse.Impl.TSum.fst.hints index 738f10a72ed..905bca7fcb4 100644 --- a/examples/miniparse/MiniParse.Impl.TSum.fst.hints +++ b/examples/miniparse/MiniParse.Impl.TSum.fst.hints @@ -116,7 +116,7 @@ "unit_typing" ], 0, - "5e14df75ad5b5b8808679e52279ac9c2" + "9e859350753219f068e7857cfa3988e2" ], [ "MiniParse.Impl.TSum.serialize_tagged_union_impl", @@ -222,7 +222,7 @@ "unit_typing" ], 0, - "903035b9a0b21c9a94a9b9d4afb0d6a8" + "79d3c4da6140b15c33f69a65d320af08" ], [ "MiniParse.Impl.TSum.parse_tagged_union_impl", @@ -339,7 +339,7 @@ "unit_typing" ], 0, - "e0aa60fb234209d5c1593f67978b519f" + "257eeb05b8b2f4623f9f2eb06d9e3879" ], [ "MiniParse.Impl.TSum.serialize_tagged_union_impl", @@ -445,7 +445,7 @@ "unit_typing" ], 0, - "f55a09b8ba79f85a3c3acb0b4a2c9016" + "e89608eeb2960bc125d2a54e04f593a2" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Spec.Int.fst.hints b/examples/miniparse/MiniParse.Spec.Int.fst.hints index 20b9ef441f1..9f6ea1fee43 100644 --- a/examples/miniparse/MiniParse.Spec.Int.fst.hints +++ b/examples/miniparse/MiniParse.Spec.Int.fst.hints @@ -445,7 +445,7 @@ "well-founded-ordering-on-nat" ], 0, - "aac9cd416bf34f594798f137df680c98" + "5538bd4bac96590649faefb13a3c002e" ], [ "MiniParse.Spec.Int.forall_bounded_u16_elim", @@ -504,7 +504,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "5c46c05d9943d39433960eaf33fabf56" + "3017e48cf4135bcc6c047fb0cc51808b" ], [ "MiniParse.Spec.Int.parse_bounded_u16", @@ -1016,7 +1016,7 @@ "well-founded-ordering-on-nat" ], 0, - "18d9098255338fc7823cf74e188b2820" + "521233ee266e636c8ea64090cefeaab5" ], [ "MiniParse.Spec.Int.parse_bounded_u16", diff --git a/examples/miniparse/MiniParse.Spec.List.fst.hints b/examples/miniparse/MiniParse.Spec.List.fst.hints index ae1ba57b9e0..f9d529d2fcc 100644 --- a/examples/miniparse/MiniParse.Spec.List.fst.hints +++ b/examples/miniparse/MiniParse.Spec.List.fst.hints @@ -273,7 +273,7 @@ "well-founded-ordering-on-nat" ], 0, - "941b10e8f8cc4cf9f830f187f9e42637" + "a7fb1e5ef1c03b21700e4cf129c2612e" ], [ "MiniParse.Spec.List.parse_nlist_eq", @@ -389,7 +389,7 @@ "unit_typing", "well-founded-ordering-on-nat" ], 0, - "1b123ea93338a807130ac5bdca34126a" + "d57ed364c24216626301bcc0e1745f51" ], [ "MiniParse.Spec.List.serialize_nlist_nil", @@ -821,7 +821,7 @@ "well-founded-ordering-on-nat" ], 0, - "0625393f1183230b151505b72fc39119" + "edec3f4749f34df4d6b22dac080d60be" ], [ "MiniParse.Spec.List.parse_nlist_eq", @@ -980,7 +980,7 @@ "well-founded-ordering-on-nat" ], 0, - "6c8f5d1d1a40a74b1812045b5d498c3c" + "ae1cb72a396a9635ec875f469755aef6" ], [ "MiniParse.Spec.List.serialize_nlist_nil", diff --git a/examples/miniparse/MiniParse.Spec.TEnum.fst.hints b/examples/miniparse/MiniParse.Spec.TEnum.fst.hints index 27ef90899f0..1cc8b6e0fb4 100644 --- a/examples/miniparse/MiniParse.Spec.TEnum.fst.hints +++ b/examples/miniparse/MiniParse.Spec.TEnum.fst.hints @@ -20,7 +20,7 @@ "function_token_typing_FStar.UInt32.n", "int_inversion", "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -28,7 +28,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "16a3adc99599e07aee16959242a329fe" + "5e729fb3d8aa3b21a35ee5a91a7d435a" ], [ "MiniParse.Spec.TEnum.get_inductive_constructors", @@ -46,7 +46,7 @@ "typing_FStar.Reflection.Basic.lookup_typ" ], 0, - "ce6364db527b583dcf627c99967377d7" + "a1c0bc2342631322555a1a4cfcdd060d" ], [ "MiniParse.Spec.TEnum.invert_branches_with_cascade", @@ -67,7 +67,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "2552ea19c004f399ee1ae2a4b4ab4c00" + "0b667d64554fe57e55e26da89b35703d" ], [ "MiniParse.Spec.TEnum.synth_inverse_forall_bounded_u16_intro", @@ -85,7 +85,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "84c896b6d0dcb4098f2bc0a4252dfb1d" + "8827bcc9abc0087fb5ef2eceb2c382b3" ], [ "MiniParse.Spec.TEnum.mk_tenum_branches", @@ -106,7 +106,7 @@ "function_token_typing_FStar.UInt32.n", "int_inversion", "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -114,7 +114,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "9aea1191fb3d75c5848c5b9b1e6f61f8" + "cc893b7475149e2bce0fdfb2b1acd4a3" ], [ "MiniParse.Spec.TEnum.get_inductive_constructors", @@ -132,7 +132,7 @@ "typing_FStar.Reflection.Basic.lookup_typ" ], 0, - "8ba231557f02592841a9e42176706261" + "13d2e286a435b05e003c23cc11484ad4" ], [ "MiniParse.Spec.TEnum.invert_branches_with_cascade", @@ -153,7 +153,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "af4da55b03dbbf9b72472fe4fc65b27d" + "70d381e9949059aa630213f1d24a3bd3" ], [ "MiniParse.Spec.TEnum.synth_inverse_forall_bounded_u16_intro", @@ -171,7 +171,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "4c2e2b57aa8615fc8c6ca1e511c561b5" + "855b4ac629071bfb41e6bb92ee7ee864" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Tac.Base.fst.hints b/examples/miniparse/MiniParse.Tac.Base.fst.hints index ee7a1b7846d..88182d83fcb 100644 --- a/examples/miniparse/MiniParse.Tac.Base.fst.hints +++ b/examples/miniparse/MiniParse.Tac.Base.fst.hints @@ -11,7 +11,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "de5da045d176193ccec7e9d00c466cd3" + "b210172a7dce4bfb2a689a516a7ee86f" ], [ "MiniParse.Tac.Base.mk_if_t", @@ -20,7 +20,7 @@ 1, [ "@MaxIFuel_assumption", "@query", "bool_inversion" ], 0, - "769567dc39989e0398bd52530c0db13b" + "b1b9d4556b5ba684715ba2090bc1acd1" ], [ "MiniParse.Tac.Base.string_of_name", @@ -35,7 +35,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "400de6d9521a3f1ecfa1c54774957096" + "2c339a522731e67cd9cde3c6a7958fbf" ], [ "MiniParse.Tac.Base.to_all_goals", @@ -47,7 +47,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "ed7405da78add9cca167428cce0ed278" + "dba85472b5bab5b5de7efbea1e0f5a3c" ], [ "MiniParse.Tac.Base.solve_goal", @@ -59,7 +59,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "fff866b04ed75f2c0c8c6bcb362ffe23" + "57f439e23924038937ded820f7a13943" ], [ "MiniParse.Tac.Base.app_head_rev_tail", @@ -71,7 +71,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "1cdaf2daa6dec6a974ad8e38302fcc8d" + "d1b08b11c01bdd6a46527ae456a02b11" ], [ "MiniParse.Tac.Base.mk_if_t", @@ -80,7 +80,7 @@ 1, [ "@MaxIFuel_assumption", "@query", "bool_inversion" ], 0, - "d077e9f4bd9fa2a97d296770d635d0fe" + "6a8b4b7d9fb3deb08d7f3b31acab1854" ], [ "MiniParse.Tac.Base.string_of_name", @@ -95,7 +95,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "84fcb859c640914e96d6f7c66e720f5a" + "6d7da122f72d5c8554b68f921b323e15" ], [ "MiniParse.Tac.Base.to_all_goals", @@ -107,7 +107,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "84edaf96a7ed45d9b13b625cba0e1819" + "b6f089a978f962eae7b4bf0b87bb0742" ], [ "MiniParse.Tac.Base.solve_goal", @@ -119,7 +119,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "4ab0e1cf61974feb2874869e6a0583a0" + "e0ffde767fe3318c3ead49e50aebaabc" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Tac.Impl.fst.hints b/examples/miniparse/MiniParse.Tac.Impl.fst.hints index 7252eb51f2b..86bb9b1b7d1 100644 --- a/examples/miniparse/MiniParse.Tac.Impl.fst.hints +++ b/examples/miniparse/MiniParse.Tac.Impl.fst.hints @@ -23,7 +23,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "3958eef624ec45dc91f77284cd669fa3" + "b6f2998b6f7887c7933419d0cb9b65d3" ], [ "MiniParse.Tac.Impl.r", @@ -39,7 +39,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "38ed885d1b800e1e33c7e089c2863f24" + "c7102c89a3b9f77d5c931a01c14c8bbe" ], [ "MiniParse.Tac.Impl.r'", @@ -55,7 +55,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "a35af1d16594be407e5008b28b927e11" + "ba17870c9fd4a7d8a689a71d369b7137" ], [ "MiniParse.Tac.Impl.mk_u32", @@ -79,7 +79,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "a54971752d88dddee6d8732f0e854973" + "d265dd07eb2cf1e2c70e0f48abbc29e1" ], [ "MiniParse.Tac.Impl.r", @@ -95,7 +95,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "9fbe53ecf906b5c10eb6bca7667b283d" + "be629e8ee8ee2938da52a261138d5cb0" ], [ "MiniParse.Tac.Impl.r'", @@ -111,7 +111,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "7d722470bf3f8988d8763b980b01fc5b" + "305b84c3950a6dd5ae70c6e6883c4fd7" ], [ "MiniParse.Tac.Impl.j32", @@ -151,7 +151,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "7d0f7d8d4d3b2845751166a6acc2527e" + "4e4ccb9fb55396e4679d118cb451a62b" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParse.Tac.Spec.fst.hints b/examples/miniparse/MiniParse.Tac.Spec.fst.hints index 98d8000e089..fa6fe86870a 100644 --- a/examples/miniparse/MiniParse.Tac.Spec.fst.hints +++ b/examples/miniparse/MiniParse.Tac.Spec.fst.hints @@ -11,7 +11,7 @@ "projection_inverse_MiniParse.Tac.Spec.Package_p" ], 0, - "50d847d886e5e4ca3551e2ad8e858968" + "1e808f83954def8e217775b6e9de21a6" ], [ "MiniParse.Tac.Spec.gen_package'", @@ -23,7 +23,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "a81b269d0f8541ac9d31bf5a833ea00a" + "6f74553c85f1c70931bd9fe53ec33234" ], [ "MiniParse.Tac.Spec.__proj__Package__item__s", @@ -35,7 +35,7 @@ "projection_inverse_MiniParse.Tac.Spec.Package_p" ], 0, - "2080f191aff710b48c4cd25456a37810" + "59f84ff3feb5da1c4f14839b3e740ed1" ], [ "MiniParse.Tac.Spec.gen_package'", @@ -47,7 +47,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "fb841810b1efc49040002922f99e64aa" + "8740e87341f16606454f478e6b6a4d24" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParseExample.fst.hints b/examples/miniparse/MiniParseExample.fst.hints index eb5179634a5..9ae86eb7861 100644 --- a/examples/miniparse/MiniParseExample.fst.hints +++ b/examples/miniparse/MiniParseExample.fst.hints @@ -107,7 +107,7 @@ "unit_typing" ], 0, - "ab8a96fa16f586233e3ca8b1eea4ae1f" + "d44e7fac308a00ee52be9c7260563c65" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParseExample2.fst.hints b/examples/miniparse/MiniParseExample2.fst.hints index ef4d30c7024..42a0b3b8103 100644 --- a/examples/miniparse/MiniParseExample2.fst.hints +++ b/examples/miniparse/MiniParseExample2.fst.hints @@ -13,7 +13,7 @@ "refinement_interpretation_MiniParseExample2_Tm_refine_fb807a479aa69c50ca430264cffc40b0" ], 0, - "1bf978e493ac0c001515132ebe7c8068" + "793984feac9c33a0ccef3f7afc347352" ], [ "MiniParseExample2.c3", @@ -88,7 +88,7 @@ "unit_inversion", "unit_typing" ], 0, - "8bd533793132072e2853c63e2bee596e" + "9628f83b6ee5655d30bcb59cbc356b84" ], [ "MiniParseExample2.c2", @@ -172,7 +172,7 @@ "typing_tok_MiniParseExample2.X@tok", "unit_inversion", "unit_typing" ], 0, - "7687ed2dc3df2686c1b6ca72aa470f64" + "709e03e083c1666e7624f7493c2a1488" ], [ "MiniParseExample2.c1", @@ -265,7 +265,7 @@ "typing_tok_MiniParseExample2.X@tok", "unit_inversion", "unit_typing" ], 0, - "a9aacf380e96cfcd13d23b03b342dc0b" + "61f8130c26dd093630455c2e47a39936" ], [ "MiniParseExample2.c0", @@ -340,7 +340,7 @@ "typing_tok_MiniParseExample2.V@tok", "unit_typing" ], 0, - "cb00994043545fc3d5c693857b2fd8db" + "58a69ea6cba3be887e001760de86c3ae" ], [ "MiniParseExample2.__proj__U__item___0", @@ -354,7 +354,7 @@ "refinement_interpretation_MiniParseExample2_Tm_refine_fb807a479aa69c50ca430264cffc40b0" ], 0, - "10096d729653cbdcc1f9b4c181707089" + "8e212eba61d837e1982322dbe86a65be" ], [ "MiniParseExample2.c3", @@ -429,7 +429,7 @@ "unit_inversion", "unit_typing" ], 0, - "d56548f9017a0c71e34ea92a8535e6ec" + "467a3487b8da11f00d23ad00118f8731" ], [ "MiniParseExample2.c2", @@ -529,7 +529,7 @@ "typing_tok_MiniParseExample2.X@tok", "unit_inversion", "unit_typing" ], 0, - "b4694fda8eec96e02ddddf6187057e51" + "8f253ed9875fe89e39f1b479a2d14afb" ], [ "MiniParseExample2.c1", @@ -622,7 +622,7 @@ "typing_tok_MiniParseExample2.X@tok", "unit_inversion", "unit_typing" ], 0, - "2debe1e5a3cc8a3ebe52f5086825bdf0" + "fa15da6f0f587017134f7334d3aaa804" ], [ "MiniParseExample2.c0", @@ -697,7 +697,7 @@ "typing_tok_MiniParseExample2.V@tok", "unit_typing" ], 0, - "f0c67ef83ba8b77199e78355a36a72c2" + "7fc6f13d655048a10f253e9516e939f8" ] ] ] \ No newline at end of file diff --git a/examples/miniparse/MiniParseExample3.fst.hints b/examples/miniparse/MiniParseExample3.fst.hints index d9f7fad8fc2..39996061997 100644 --- a/examples/miniparse/MiniParseExample3.fst.hints +++ b/examples/miniparse/MiniParseExample3.fst.hints @@ -12,7 +12,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "23af1dae70626bc721260f526d6ac9c8" + "f3c1cf301e1ae9a37aa55198c1d652f7" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Arith.fst.hints b/examples/native_tactics/Arith.fst.hints index 7f0e683813a..269c2704486 100644 --- a/examples/native_tactics/Arith.fst.hints +++ b/examples/native_tactics/Arith.fst.hints @@ -12,7 +12,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "c9a243aaa0477eaaf724f2b99b337063" + "4a587082319856920c9ea8a92042466a" ], [ "Arith.lem1", @@ -30,7 +30,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "a9824022279b433c79145598aa90b0db" + "cfa3304ef2a27496b8b8ef1a2fe5611b" ], [ "Arith.lem1", @@ -43,7 +43,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "405f50cd5513ca4df837213b31aa49e4" + "abc9048bf90ff6a07c7ec1943d10630c" ], [ "Arith.lem2", @@ -56,7 +56,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "f927192dba46f9387d983152c115e6a0" + "8de7aefba7926d8303c59022bc6e4cce" ], [ "Arith.lem2", @@ -74,7 +74,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "6cae369dcdebdf9f50690d9d85ae5736" + "71fb3a4c27e8e88b4f8d202650f1a484" ], [ "Arith.lem3", @@ -89,7 +89,7 @@ "projection_inverse_Prims.Cons_tl", "true_interp" ], 0, - "4c24a1898e92fc860917d9bf34bb18f7" + "d7fc8f881659cdd8232a34a111625721" ], [ "Arith.lem3", @@ -114,7 +114,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "a66d2a6c4359ec540b079b368002798e" + "f253a8c09d7a4a53d07974e2e82c5c11" ], [ "Arith.lem3", @@ -129,7 +129,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "89fb1ce957f1ea4af72a427dc462eb61" + "ee631c727d4bff1efd270de98720e6d8" ], [ "Arith.lem4", @@ -144,7 +144,7 @@ "projection_inverse_Prims.Cons_tl", "true_interp" ], 0, - "c3794b51f1390bf2c38b63aec7f2ee34" + "4b36b58088c006227ba47d32f496f2a7" ], [ "Arith.lem4", @@ -162,7 +162,7 @@ "unit_inversion", "unit_typing" ], 0, - "6a52b6a034408f4c1487871629b08a9e" + "a91e45a5a31322cb201e8441107243c8" ], [ "Arith.lem4", @@ -173,11 +173,11 @@ "@MaxIFuel_assumption", "@query", "Prims_interpretation_Tm_arrow_f82c3fb9ac6610efb97620a59b378092", "equation_Prims.l_Forall", "equation_Prims.squash", "int_inversion", - "l_quant_interp__7992", + "l_quant_interp__8018", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "61fa0fb6d0131ca67d8ac3317c12b565" + "54f9ac1369fbc49ad355154388cec21e" ], [ "Arith.lem4", @@ -202,7 +202,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "c9d16200b6ddf0a5c5ae13970b96f97b" + "f434abb3c7886be65ca4341c5b9c96cf" ], [ "Arith.lem4", @@ -211,12 +211,12 @@ 1, [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", - "equation_Prims.squash", "int_typing", "l_quant_interp__8008", + "equation_Prims.squash", "int_typing", "l_quant_interp__8034", "projection_inverse_BoxInt_proj_0", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "7f1579ce2edcb86ed78a1ecb738d2518" + "4290515daa3295495e1b981968bb3656" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/BV.Test.fst.hints b/examples/native_tactics/BV.Test.fst.hints index a2bb011370b..3b31b6b150b 100644 --- a/examples/native_tactics/BV.Test.fst.hints +++ b/examples/native_tactics/BV.Test.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "27f8f7cebf08c2c9a703001f046abc78" + "9482e9fbd8d21174bd757093b254fd5a" ], [ "BV.Test.test2", @@ -17,7 +17,7 @@ 1, [ "@query" ], 0, - "8bc6524227f8c6984de04091264657fb" + "6efb093b796d5494d5b374eec9d4b495" ], [ "BV.Test.test3", @@ -26,7 +26,7 @@ 1, [ "@query" ], 0, - "ef36a3c2ca09f75b2962a45ac5bc4e3b" + "20e311b31fbb16c15ec7829f6922f6a6" ], [ "BV.Test.test4", @@ -35,7 +35,7 @@ 1, [ "@query" ], 0, - "e71f0a39eda6bc1b7590193429a5f873" + "20770a7621314491937036f4247c2079" ], [ "BV.Test.test5", @@ -44,7 +44,7 @@ 1, [ "@query" ], 0, - "69ae7fb6b434fbe6c18aa5834aad2672" + "03d30a3400e0a9d1a78b64287d5b5dc9" ], [ "BV.Test.test6", @@ -53,7 +53,7 @@ 1, [ "@query" ], 0, - "20ec477e457ad59285456bcede039743" + "35aa69b9160d2d4800219df0e52beb0c" ], [ "BV.Test.test7", @@ -62,7 +62,7 @@ 1, [ "@query" ], 0, - "0ce0dab5c7c719301aea0603b24a3143" + "f7fc9b72f22fc3c7cc6a2f98d4bd7326" ], [ "BV.Test.test8", @@ -71,7 +71,7 @@ 1, [ "@query" ], 0, - "a89abd9709bf265e2fb6ec02680177b2" + "39937b80dabce324258c8b0ed2a81c8a" ], [ "BV.Test.test9", @@ -80,7 +80,7 @@ 1, [ "@query" ], 0, - "014f438543a8a3568bcd6f73a41f0185" + "8ee0bf20e181c5640d1fae87efc1e6c5" ], [ "BV.Test.test10", @@ -89,7 +89,7 @@ 1, [ "@query" ], 0, - "b9df9aa95bb84b3d718027e66bef1c77" + "c511cd6696d87887b9d46bd3ae86250c" ], [ "BV.Test.test11", @@ -98,7 +98,7 @@ 1, [ "@query", "true_interp" ], 0, - "ff16d7271d0f2b98bf3bd052cc8b45a3" + "e768d5bf83650cd8fddb13960fd4ac31" ], [ "BV.Test.test11", @@ -107,7 +107,7 @@ 1, [ "@query" ], 0, - "2a4c06ae75d83a8940f1494088c77f51" + "cdc8e6b0a9ade1d1e1fe0480e7153a3b" ], [ "BV.Test.test12", @@ -116,7 +116,7 @@ 1, [ "@query", "true_interp" ], 0, - "3c0dc2de691dbd0354e8014ad324b604" + "7360cd1ffdb551985d1d8692deb8d3c0" ], [ "BV.Test.test12", @@ -125,7 +125,7 @@ 1, [ "@query" ], 0, - "e44ff9210095d3f0602a3564dfe6772c" + "191b843ec5565899ef4af5fb90fdcdb4" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/BV.fst.hints b/examples/native_tactics/BV.fst.hints index 1e60180c3f6..9dc35d56e4a 100644 --- a/examples/native_tactics/BV.fst.hints +++ b/examples/native_tactics/BV.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "1233b29a07b276ef3db729e75c3ce2c2" + "28f7119ee7b255d5c8c91203f1e1f1fb" ], [ "BV.cong_bvand", @@ -20,7 +20,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "b6b06c8686f5157da21e08110b6cfd80" + "8a037ad7a9e3dc84b78e1cc74f327e62" ], [ "BV.cong_bvand", @@ -33,7 +33,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "5a489fbc986996a34ba89763f5a9f1ed" + "83cd30330080e689496cef4057ab9767" ], [ "BV.cong_bvxor", @@ -45,7 +45,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "3b99c3a7679d18dba25671e258fb7b92" + "b50d92bb96d631c8a7fef37ed81c6d99" ], [ "BV.cong_bvxor", @@ -57,7 +57,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "2d8c278777bd7ffdb27751b7a2a00c2d" + "bb68dac3280349c6e0e92a8376fbd8b2" ], [ "BV.cong_bvxor", @@ -69,7 +69,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "030f512cb80dc68ce1a156234679c993" + "9d70b9186e1dadc7be3b9b5b75e6e915" ], [ "BV.cong_bvxor", @@ -82,7 +82,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "6a8647e8fc272dc2fe21306b27b6fa0a" + "ff25365d7f666e447516021b50160348" ], [ "BV.cong_bvor", @@ -94,7 +94,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "b4501e8eea1e1aafd9f26099b77cc180" + "99bbbddaf9763e2f24e96a5b3bba682b" ], [ "BV.cong_bvor", @@ -106,7 +106,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "53542fee96a81d729420fd5e7668cc27" + "5a4934cc112cc8cf94fb12d860b0f7f7" ], [ "BV.cong_bvor", @@ -118,7 +118,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "dd39ac9be73e101adc3371734c1c8b0d" + "ad04e852a673e73fdb398777da4a6703" ], [ "BV.cong_bvor", @@ -131,7 +131,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "3e84d3726555b0fcf18f49d993511f9c" + "b6c4ee01699acc6d39afdd9e704398e1" ], [ "BV.cong_bvshl", @@ -143,7 +143,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "69fec1c2414fe90991935a2c165b6ee7" + "f1cd89f1207e71f8e777dced623d110f" ], [ "BV.cong_bvshl", @@ -155,7 +155,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "ad5543e345a083313a8d614f8895339f" + "3e2bd9703b90c09b83d62e46e4b1ff6a" ], [ "BV.cong_bvshl", @@ -175,7 +175,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "561c879e9df6540a72d70d66bd5353e8" + "47de7c6f3f9ad22a473ad35daff839e3" ], [ "BV.cong_bvshl", @@ -188,7 +188,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "0f6f6912cb2bf70eabe3c6f8de8213a9" + "faeab2b94c799ced90e8ee0f90c625f8" ], [ "BV.cong_bvshr", @@ -197,7 +197,7 @@ 1, [ "@query" ], 0, - "ca07cddb55109131dc284ef3a334c701" + "c3eb380fbcf40a415b8427e4a6b9b7e8" ], [ "BV.cong_bvshr", @@ -217,7 +217,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "f38e39563b1ea0fbc8967574aa9aa383" + "2befa365cb74e55aa7a35509fab04ef5" ], [ "BV.cong_bvshr", @@ -230,7 +230,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "16c476b31f8422fd4a01011f48a44fad" + "7da5eb5cbfbc4801d8bb8c46bf638eb3" ], [ "BV.cong_bvdiv", @@ -239,7 +239,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "04b004a39455986be4442c900758af78" + "2cbd19d9959e758f3b0f95292545a34d" ], [ "BV.cong_bvdiv", @@ -248,7 +248,7 @@ 1, [ "@query" ], 0, - "6b2e0c6c1d40718b69a23c0d6b4b31d1" + "dd5e37ef9497b02227282fae4e7dd5ba" ], [ "BV.cong_bvdiv", @@ -260,7 +260,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "d47da19125bc22c5099aaf74c8438b86" + "563a4218f9a589753371ed0d433a4ad2" ], [ "BV.cong_bvdiv", @@ -273,7 +273,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "da1165d830fc24fb37e25d06cb013560" + "82d75b601635cdcb91fd73bf6afb9b28" ], [ "BV.cong_bvmod", @@ -282,7 +282,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "e17c37ce64abea47ed83f51c08794d51" + "0719e52392450a3ec9ba25f98545f7e0" ], [ "BV.cong_bvmod", @@ -291,7 +291,7 @@ 1, [ "@query" ], 0, - "86138bb093d059fe5226b7a8787cb241" + "c04d030726f8d57ba98bd53a4019c7e6" ], [ "BV.cong_bvmod", @@ -303,7 +303,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "c9d476b495a063c8e53c8b62b4936a3c" + "5bcb6411b713d4ff3ea0184ad36a6ebe" ], [ "BV.cong_bvmod", @@ -316,7 +316,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "e97cf82356d6f7ac4003685baeefdd65" + "991e33d7914a6cbd8d041990aa156df4" ], [ "BV.cong_bvmul", @@ -325,7 +325,7 @@ 1, [ "@query" ], 0, - "1ad5b3bdded7f8a6165fb468dda11068" + "acc882c0c6406d515d04ae94f494f032" ], [ "BV.cong_bvmul", @@ -337,7 +337,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "0d1ee5f78216fc6473032d09752e3417" + "8910fdfd4a88e67d423bdfeca2cfe9e9" ], [ "BV.cong_bvmul", @@ -350,7 +350,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "89560745c57df4cb275b1728c13f8dda" + "2bae654f2f2c9dbe5ba12a8b5e55461e" ], [ "BV.cong_bvadd", @@ -362,7 +362,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "aabc42a84fd9a8ba8960a2bb22a3a6ad" + "c6f1a2596d15344cabfe1c0a372ce739" ], [ "BV.cong_bvadd", @@ -374,7 +374,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "9031c048d3b60feb562068b08db2f1cb" + "8a8a84a66b6cff2439fa5a24bb77e419" ], [ "BV.cong_bvadd", @@ -386,7 +386,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "a97300b16df741271c7f46bbde7c23bf" + "52e855aef99d6f837917ae4ceaccfc35" ], [ "BV.cong_bvadd", @@ -399,7 +399,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "c30a075aacfb2727a045695666559a11" + "5e2bf7d5f3f08b69f3f192e6230e3f85" ], [ "BV.cong_bvsub", @@ -411,7 +411,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "0789ed6c84ab3e8d098aa309566f5d4b" + "f0ac4f4099e0dff5535f3445b3c4719f" ], [ "BV.cong_bvsub", @@ -423,7 +423,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "ce746f9f2708313d79ebd4eb0806d873" + "7379b5b63282ef6298002dcec4f7838f" ], [ "BV.cong_bvsub", @@ -435,7 +435,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "7a403cda57dd8c8f950fcf9945bbdd48" + "98dc2b185bcb0628d9dfc3e498136366" ], [ "BV.cong_bvsub", @@ -448,7 +448,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "dce0243a70bab13be150efb195b0dee5" + "cdf69bb8306585cc4f045236237bcfcc" ], [ "BV.eq_to_bv", @@ -457,7 +457,7 @@ 1, [ "@query" ], 0, - "92f29643e4d7f626c1ba6cd5a5bfa4d3" + "221f4a4a5b3ec0a8e965eebec725f5be" ], [ "BV.eq_to_bv", @@ -469,7 +469,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "a1eac9a8c582834eb9bc9f6d97da7fd7" + "dbc011e18db87e6245285b0cc6b92ab7" ], [ "BV.eq_to_bv", @@ -482,7 +482,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "098bef4ab78a7a842ef7e72370fa6592" + "df15080244072c6653999f68df078511" ], [ "BV.lt_to_bv", @@ -494,7 +494,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "ada6b883e7e7165680c5ffc45e39babd" + "0b2096a446743699151e9bf5b8da2131" ], [ "BV.lt_to_bv", @@ -503,7 +503,7 @@ 1, [ "@query", "b2t_def" ], 0, - "c5e593c0ec8e26e56f2cb6b1b893b9a0" + "11cee5cda84de10aab94e0aa1142fc1d" ], [ "BV.trans", @@ -515,7 +515,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "d1c950f8acd567689672e22af8af2e6f" + "67a4a8e5a1f722912b383196b7807ca8" ], [ "BV.trans", @@ -528,7 +528,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "88de68f752d245997280ccf98d200008" + "1bff1a92c5f7c0f966f5db19661277b3" ], [ "BV.trans_lt", @@ -540,7 +540,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "82189fb71df182f5cb448200dad10aa3" + "81aece286186601b12a76e5818495eab" ], [ "BV.trans_lt", @@ -553,7 +553,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "6616fd355ceeff716620aaf3190873da" + "31315ba4c9b1717929f59438b1e7573c" ], [ "BV.trans_lt2", @@ -562,7 +562,7 @@ 1, [ "@query" ], 0, - "47dad0b2455d60066c3ecae4150df95d" + "3f6698d5ce195bfce3937f6442ef7d87" ], [ "BV.trans_lt2", @@ -571,7 +571,7 @@ 1, [ "@query" ], 0, - "a806260cf73d2c7d2891fea9c49dac60" + "9079f916697a99338f61e537afe1b7cd" ], [ "BV.trans_lt2", @@ -583,7 +583,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "8f1d6514fdfcd37fa4b9e83aad53541d" + "b0e38c30356c08f25e327576d0b58d26" ], [ "BV.trans_lt2", @@ -596,7 +596,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "263cc0acb780b3816dc15ce25308247d" + "3e0148be3f9bfac2292291f4cd00f743" ], [ "BV.v64_eq", @@ -605,7 +605,7 @@ 1, [ "@query", "lemma_FStar.UInt64.uv_inv" ], 0, - "a4277f63ec6acf6f83439c0d1207fcd8" + "a7d1f1c0226aa5e28e5d9d1e49e2a56d" ], [ "BV.unfold_logand64", @@ -619,7 +619,7 @@ "typing_FStar.UInt64.logand" ], 0, - "de25793d1ab57026decef71d3ed65bc4" + "af822af32035f2ca3b20b81f5106af4f" ], [ "BV.unfold_logor64", @@ -633,7 +633,7 @@ "typing_FStar.UInt64.logor" ], 0, - "4485e119c6b95e2e09c1e74c8283718e" + "e5b5a0a1645cad40915167439bca2fad" ], [ "BV.unfold_logxor64", @@ -647,7 +647,7 @@ "typing_FStar.UInt64.logxor" ], 0, - "8568fac7820c8d29f8fe1de34b415dde" + "36051ce0a553daae0e4376597ee40de3" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Bane.fst.hints b/examples/native_tactics/Bane.fst.hints index 92aadb6a7a4..5df424c9de5 100644 --- a/examples/native_tactics/Bane.fst.hints +++ b/examples/native_tactics/Bane.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "28ddcbd4be3e26574c9828be52e5b9e7" + "19cbc51fb2a5b27c3cd70fe0857d10e8" ], [ "Bane.repeat_or_fail", @@ -26,7 +26,7 @@ "lemma_FStar.Pervasives.invertOption", "unit_typing" ], 0, - "fe454a7d36b3ff440a0bb63fee60294d" + "747335fec36304062b4a638b7b572211" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Canon.Test.fst.hints b/examples/native_tactics/Canon.Test.fst.hints index 3d8bb91be36..cd888a267e1 100644 --- a/examples/native_tactics/Canon.Test.fst.hints +++ b/examples/native_tactics/Canon.Test.fst.hints @@ -12,7 +12,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "f41bbdcdaf0fc5ed1f9ec49cac535af6" + "903d6a5ba31ea6e19e4ffb60b9492788" ], [ "Canon.Test.lem8", @@ -21,7 +21,7 @@ 1, [ "@query", "true_interp" ], 0, - "af7c122b50f4efce6731b28e8113d398" + "50105dbb3825ff3a07433333764948a3" ], [ "Canon.Test.lem9", @@ -30,7 +30,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "5d03082cd2ec3f7a4166c1b493fdae51" + "b7e987e0502c9e660bd86980ecc41907" ], [ "Canon.Test.lem10", @@ -39,7 +39,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "e1214b1c0bac8e31167b12f289bf3f69" + "d10987de15dee8d1147a70ab112c8516" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/CanonDeep.fst.hints b/examples/native_tactics/CanonDeep.fst.hints index 03c7c2eb4a5..da82b7e98de 100644 --- a/examples/native_tactics/CanonDeep.fst.hints +++ b/examples/native_tactics/CanonDeep.fst.hints @@ -28,7 +28,7 @@ "fuel_guarded_inversion_FStar.Reflection.Arith.expr" ], 0, - "4d1a39a57e9723bbff8b7841895befac" + "07b8abe219a1641c2ca206031d981e2e" ], [ "CanonDeep.expr_to_term", @@ -74,7 +74,7 @@ "subterm_ordering_FStar.Reflection.Arith.Umod" ], 0, - "74cda0cea00640ea3bc7368bf5200925" + "f156e7ed57dd968d218a0300e89e72fe" ], [ "CanonDeep.canon_correct", @@ -83,7 +83,7 @@ 1, [ "@query", "equation_CanonDeep.canon_expr_" ], 0, - "a5241d7513d52d9e9ec45d87bed6bf8b" + "5c7d97691017f0732269391df1cbb851" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Clear.fst.hints b/examples/native_tactics/Clear.fst.hints index 8e0d0254b0c..a45487a30db 100644 --- a/examples/native_tactics/Clear.fst.hints +++ b/examples/native_tactics/Clear.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "cb2985d9c1ab8dacc6927ed5ef72bb99" + "3c176c2a002d4b8c8efd5f78eb4999eb" ], [ "Clear.l2", @@ -21,7 +21,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "828d6daaf9f6390fd6335b7f145f1cf4" + "b9dc11bd6839a8979f1bfacd9bcf4470" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/DependentSynth.fst.hints b/examples/native_tactics/DependentSynth.fst.hints index 18b035a8db5..62e3b605a93 100644 --- a/examples/native_tactics/DependentSynth.fst.hints +++ b/examples/native_tactics/DependentSynth.fst.hints @@ -11,7 +11,7 @@ "equation_DependentSynth.myty", "int_typing", "unit_typing" ], 0, - "04db54c4ce16221b5482cbecb391fdd1" + "e0485ae0b91a2911bc978071789e9db8" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Evens.fst.hints b/examples/native_tactics/Evens.fst.hints index fc4829ee374..b51a59740f3 100644 --- a/examples/native_tactics/Evens.fst.hints +++ b/examples/native_tactics/Evens.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "22227100a94b11d32d48d93044267402" + "160332317f3047786205a623e1e29032" ], [ "Evens.__proj__US__item___0", @@ -21,7 +21,7 @@ "refinement_interpretation_Evens_Tm_refine_7094be438dbc16658c0caec70fa7452e" ], 0, - "5c8183dcaaaf61d097de0541d198312a" + "7841eef0b2fb7d754a388baac5ef621e" ], [ "Evens.even", @@ -30,7 +30,7 @@ 1, [ "@query", "assumption_Evens.unary_nat__uu___haseq" ], 0, - "552df410a05ef5d66d17b0a421765015" + "5ec8136b738c78655d0132031ce981c4" ], [ "Evens.__proj__Even_SSn__item__n", @@ -43,7 +43,7 @@ "refinement_interpretation_Evens_Tm_refine_6b35b246e3f3e217f09d76d285c6fcd3" ], 0, - "6ebb09334421d2d2cb1672559d1ddacc" + "92527027cbe7850ee010d85f4d4da385" ], [ "Evens.__proj__Even_SSn__item___1", @@ -58,7 +58,7 @@ "refinement_interpretation_Evens_Tm_refine_6b35b246e3f3e217f09d76d285c6fcd3" ], 0, - "48f54e1c6de18954e698fa276dd85fd9" + "f97c6d1024ae885c67a223a3e92a5191" ], [ "Evens.nat2unary", @@ -73,7 +73,7 @@ "well-founded-ordering-on-nat" ], 0, - "07481ed11533e83eb4ef3cab1660ef35" + "52f1daaef8d54cb11006a1353ca26222" ], [ "Evens.nat2unary", @@ -82,7 +82,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "424476f16f107cd5a949d00ef4583303" + "24fc97cef086659299988016a85b789a" ], [ "Evens.even0", @@ -94,7 +94,7 @@ "equality_tok_Evens.U0@tok", "typing_tok_Evens.Even0@tok" ], 0, - "88fd69e943995e20cd04d369f474fc11" + "70d23dccfabf5f31e083b9e06bef649c" ], [ "Evens.evenSSn", @@ -103,7 +103,7 @@ 1, [ "@query", "true_interp" ], 0, - "64001597806345604f63317dae434d09" + "14e46f680284ad64f335db61e5378618" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Imp.fst.hints b/examples/native_tactics/Imp.fst.hints index b41dc24c908..ddf7f8f6136 100644 --- a/examples/native_tactics/Imp.fst.hints +++ b/examples/native_tactics/Imp.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "equation_Imp.f" ], 0, - "2756520922dea54c6d802c55b67a4446" + "ad3e2914e126b8047b74272c869fbc87" ], [ "Imp.uu___64", @@ -17,7 +17,7 @@ 1, [ "@query", "equation_Imp.g" ], 0, - "6ba933e3ce54565811164b2d5003e4ad" + "957d7b3ca4f790379f4df613d5b5fdec" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Plugins.Test.fst.hints b/examples/native_tactics/Plugins.Test.fst.hints index e9bc0186391..0482752987a 100644 --- a/examples/native_tactics/Plugins.Test.fst.hints +++ b/examples/native_tactics/Plugins.Test.fst.hints @@ -12,7 +12,7 @@ "function_token_typing_Prims.bool", "function_token_typing_Prims.int" ], 0, - "e41d8a8e4fd66d73b793d87063802088" + "c3bdfbef396ac59bf1a48eb48c31b344" ], [ "Plugins.Test.uu___63", @@ -21,7 +21,7 @@ 1, [ "@query" ], 0, - "357b697b34979b895d76dc385b8c421f" + "b3c3a4e2cbcce671e9cf05ef20a4cdb0" ], [ "Plugins.Test.uu___64", @@ -34,7 +34,7 @@ "function_token_typing_Prims.bool", "function_token_typing_Prims.int" ], 0, - "aca95e6c21e122cee1d430425827ffc5" + "936d4348161ef6b434b8383b67a18c5c" ], [ "Plugins.Test.uu___64", @@ -43,7 +43,7 @@ 1, [ "@query" ], 0, - "e4ec3a904bf0e5453d5cac395b98a7b2" + "3923a8818523abb74022cfa17f8defd8" ], [ "Plugins.Test.uu___65", @@ -56,7 +56,7 @@ "function_token_typing_Prims.int" ], 0, - "81076f76f82278470b4cde2a40e77989" + "a585db42284d58751c02fd52ff8859c6" ], [ "Plugins.Test.uu___65", @@ -65,7 +65,7 @@ 1, [ "@query" ], 0, - "efa87f4e0c27734ba8182d759c2d4f3e" + "69842c725fcae84e0a4c4acbd243cd22" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Print.Test.fst.hints b/examples/native_tactics/Print.Test.fst.hints index e907efc6590..834beb8cbed 100644 --- a/examples/native_tactics/Print.Test.fst.hints +++ b/examples/native_tactics/Print.Test.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "0ca9665661ace618a765208432c4449b" + "b9c9e83fbe842814b959cb20d63e4418" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Pruning.fst.hints b/examples/native_tactics/Pruning.fst.hints index 0d015a3f0ba..50c3a470684 100644 --- a/examples/native_tactics/Pruning.fst.hints +++ b/examples/native_tactics/Pruning.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "6e4ebd2cc252c6576e51e1ba51f65693" + "636c37e466de8b94b10a4b1c219bc52b" ], [ "Pruning.uu___70", @@ -26,7 +26,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "cd6e5d177f30374c73d350c11a5464be" + "575522a782c47bd48b43c88fbbf0dae2" ], [ "Pruning.uu___71", @@ -44,7 +44,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "0cfd4441464457da073391a2cc39cc65" + "7a341bd5c5e7167e6639112098943b37" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Registers.List.fst.hints b/examples/native_tactics/Registers.List.fst.hints index e3a5d353da2..8eeb43192e5 100644 --- a/examples/native_tactics/Registers.List.fst.hints +++ b/examples/native_tactics/Registers.List.fst.hints @@ -25,7 +25,7 @@ "typing_FStar.Pervasives.Native.__proj__Mktuple2__item___1" ], 0, - "4479708071b04e22ae5fa3f0e5d126c5" + "a13ee33f4b13320ef3ccba85511fde14" ], [ "Registers.List.sel", @@ -34,7 +34,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "6c45a24f056b9ebd981d3411c5d84b2c" + "f46b438545cf3f3ecd692946f11e7664" ], [ "Registers.List.const_map_n", @@ -49,7 +49,7 @@ "well-founded-ordering-on-nat" ], 0, - "a26ce35ba17d7e1c20ca2719a76662c7" + "d461ade1b3163e2d0640570bd38cfeae" ], [ "Registers.List.const_map_n", @@ -58,7 +58,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "113b096c12d9867fcf0affc55418fd3b" + "7d4351a2c47a836397a71c6c7b95768a" ], [ "Registers.List.identity_map", @@ -73,7 +73,7 @@ "well-founded-ordering-on-nat" ], 0, - "ff608b0cb04de480dd5bbfd9017d32c9" + "6d600d7e44731cc161843ec3ced3aca8" ], [ "Registers.List.identity_map", @@ -82,7 +82,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "5a39218c5d3126060c131cc9744b4652" + "7da0d25952e68bb7208c158671595985" ], [ "Registers.List.eta_map", @@ -97,7 +97,7 @@ "well-founded-ordering-on-nat" ], 0, - "31d5a58ba9ebb7e76fede362c616f6b8" + "ba94d0248ffbfb0d195077ccf431f2db" ], [ "Registers.List.eta_map", @@ -106,7 +106,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "14be80ad09367c200a54268903d6778d" + "6bb955fc7f77d544961e82202346f34a" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Sequences.fst.hints b/examples/native_tactics/Sequences.fst.hints index 42b70acf147..9d7f0e28087 100644 --- a/examples/native_tactics/Sequences.fst.hints +++ b/examples/native_tactics/Sequences.fst.hints @@ -12,7 +12,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "d417e368bdf5e0077809f9feb812c76b" + "9d42b81d81c3a1f43c0882c70f03b97c" ], [ "Sequences.test", @@ -35,7 +35,7 @@ "typing_FStar.Seq.Base.length" ], 0, - "384c51b0d47034f48d2f928fd8ef95b0" + "6cb008ee39cc178339e14d256aff5a38" ], [ "Sequences.test", @@ -67,7 +67,7 @@ "typing_FStar.Seq.Properties.snoc" ], 0, - "dcc7155a6afdd875bb76325e24159811" + "7d7597db8ba6ee22848f0bad03c1fa2e" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Simple.fst.hints b/examples/native_tactics/Simple.fst.hints index fca8b257a59..0c71cf36d37 100644 --- a/examples/native_tactics/Simple.fst.hints +++ b/examples/native_tactics/Simple.fst.hints @@ -16,7 +16,7 @@ "well-founded-ordering-on-nat" ], 0, - "60347bdfc38a84b972047b9f8a55aa5b" + "b3f077eaa3f5269736508956ba134e29" ], [ "Simple.id", @@ -25,7 +25,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "fde5b554225c8190b7e61b8323e33f77" + "a2bffa832faff947178901e29ef73ac8" ], [ "Simple.poly_id", @@ -42,7 +42,7 @@ "well-founded-ordering-on-nat" ], 0, - "90edcccf3ddaa48bdc625bb864b6032e" + "23f8e733b80c0278a5346660b030e09f" ], [ "Simple.poly_id", @@ -51,7 +51,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "2555b2e9ef76b6c68e7e9e6dd6f96715" + "81bbe3c8e5999803952e65868f6f0ac3" ], [ "Simple.mk_n_list", @@ -67,7 +67,7 @@ "well-founded-ordering-on-nat" ], 0, - "df9e72d50f6f372d2755f152a8dd27b0" + "03f956f0d0d972208fc8df020e520855" ], [ "Simple.mk_n_list", @@ -76,7 +76,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "21d9737681eb4b4ad115ba7a42d1b94c" + "65636f57b24c4c466dcf64e06928a408" ], [ "Simple.poly_list_id", @@ -89,7 +89,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "60ed7611a275fbc8820e3e7f16d41b2c" + "1b55a974eaecdc94187d0cbeae3f4cfd" ], [ "Simple.eq_int_list", @@ -104,7 +104,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "2584f5fdab98374bd4e086cec1676fab" + "6245c8e54d2087e1b8d54cacc4ae892a" ], [ "Simple.eq_int_list", @@ -113,7 +113,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "47abd974be712a76505a88cf0d894ce9" + "133eca315e063aacd9907ed71e9d9b23" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/SimpleTactic.Test.fst.hints b/examples/native_tactics/SimpleTactic.Test.fst.hints index f00311099dd..b0bf2b76b64 100644 --- a/examples/native_tactics/SimpleTactic.Test.fst.hints +++ b/examples/native_tactics/SimpleTactic.Test.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "34191bdaf024f706fe4683872a218cc5" + "7311cc30a2bc767d6de2a3c3f68a0a9c" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Split.fst.hints b/examples/native_tactics/Split.fst.hints index 846b2afa325..1e3bd440a83 100644 --- a/examples/native_tactics/Split.fst.hints +++ b/examples/native_tactics/Split.fst.hints @@ -11,7 +11,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "31fccc326e566cfee811cb0481124504" + "d87b49407da36444023cd4d210d2acd5" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Tutorial.fst.hints b/examples/native_tactics/Tutorial.fst.hints index 390f7f50feb..a44fca9f534 100644 --- a/examples/native_tactics/Tutorial.fst.hints +++ b/examples/native_tactics/Tutorial.fst.hints @@ -12,7 +12,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "34a9870556e3499d8238d238b2d664f9" + "ca09d0fbf61596bfdc7ca8a8f412bfe3" ], [ "Tutorial.ex3'", @@ -25,7 +25,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "522fa31056d048232061ea0dd2c25ceb" + "3c3beb6971090e2ce79dcb69df905db5" ], [ "Tutorial.ex4", @@ -38,7 +38,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "4c5db8c54ae3a00733a64fd2f99964c6" + "b7746d87de104efb90ad0670c3beb8ed" ], [ "Tutorial.ex4", @@ -51,7 +51,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "8c7e11ca4a8f30d51f296e110b89c615" + "0920ff959f1540b3a708c2609bbf9359" ] ] ] \ No newline at end of file diff --git a/examples/native_tactics/Unify.fst.hints b/examples/native_tactics/Unify.fst.hints index e7ad6aa9442..1e1fc63e3e7 100644 --- a/examples/native_tactics/Unify.fst.hints +++ b/examples/native_tactics/Unify.fst.hints @@ -12,7 +12,7 @@ "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0" ], 0, - "b56b125ebe18ec3e872ee663e98e0960" + "982cc8fca7a20f13e103ce41a8682ec4" ] ] ] \ No newline at end of file diff --git a/examples/printf/SimplePrintf.fst.hints b/examples/printf/SimplePrintf.fst.hints index 141152a3ceb..0124d55e5cd 100644 --- a/examples/printf/SimplePrintf.fst.hints +++ b/examples/printf/SimplePrintf.fst.hints @@ -74,7 +74,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__hd" ], 0, - "d7227cc3532c4105074bf80134a89425" + "dae3cc54943b0ebc9a36f7d648fbc32e" ], [ "SimplePrintf.string_of_dirs", @@ -124,7 +124,7 @@ "typing_SimplePrintf_Tm_abs_f9392fb11968dc07bfc5643a7c50c36d" ], 0, - "d237f011dbaa28dfe1795bb03000ef52" + "7a42a15b107c6f205c4004d8d82e638a" ], [ "SimplePrintf.add_dir", @@ -162,7 +162,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "7e83d989dedc9131ade991de99c6f9e0" + "42190258f1064a9f97788096d9a5737c" ], [ "SimplePrintf.sprintf", @@ -287,7 +287,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__hd" ], 0, - "984901ea88ed9ceeeba2535dc5221345" + "54a8de8a8b8a9edd913a806e4b0cde19" ], [ "SimplePrintf.string_of_dirs", @@ -328,7 +328,7 @@ "typing_SimplePrintf_Tm_abs_f9392fb11968dc07bfc5643a7c50c36d" ], 0, - "fede352b20bfb8b6504e0fb7840e82a2" + "9ed7fc7e1c6c72412df08b13bbb483f1" ], [ "SimplePrintf.add_dir", @@ -366,7 +366,7 @@ "subterm_ordering_Prims.Cons", "typing_Prims.__proj__Cons__item__tl" ], 0, - "538f27e00848f62d6d63df86e2c6c8e8" + "fe1d6e540eb724be7b512f30974f5321" ], [ "SimplePrintf.sprintf", diff --git a/examples/rel/Benton2004.DDCC.fst.hints b/examples/rel/Benton2004.DDCC.fst.hints index 59e108fa67c..4d251a40a61 100644 --- a/examples/rel/Benton2004.DDCC.fst.hints +++ b/examples/rel/Benton2004.DDCC.fst.hints @@ -971,7 +971,7 @@ "typing_Benton2004.while", "well-founded-ordering-on-nat" ], 0, - "c04570f916d3e17da3092eae5968258a" + "ac10169e93bd84a3095e7670a07fe6b4" ], [ "Benton2004.DDCC.d_whl", @@ -1030,7 +1030,7 @@ "well-founded-ordering-on-nat" ], 0, - "86930311d29ba2edf66eabe0cf7dd025" + "3ff0945d8b451f682d74a5b5d162ac7f" ], [ "Benton2004.DDCC.d_su1", @@ -1530,7 +1530,7 @@ "unit_typing", "well-founded-ordering-on-nat" ], 0, - "7e047551b605946922b4528d62975a9e" + "5673ad1a93c55b66cfae96c4259b74f1" ], [ "Benton2004.DDCC.ns_f", diff --git a/examples/rel/Benton2004.RHL.fst.hints b/examples/rel/Benton2004.RHL.fst.hints index c3a326fdf60..f3ab3e9e5f5 100644 --- a/examples/rel/Benton2004.RHL.fst.hints +++ b/examples/rel/Benton2004.RHL.fst.hints @@ -792,7 +792,7 @@ "typing_tok_Benton2004.RHL.Right@tok", "well-founded-ordering-on-nat" ], 0, - "295eb296e9a0d3d1a86ed82f272f9e98" + "484407a43b422f749efa49a1a198b62c" ], [ "Benton2004.RHL.holds_interp_flip", @@ -958,7 +958,7 @@ "typing_tok_Benton2004.RHL.Right@tok", "well-founded-ordering-on-nat" ], 0, - "c3ff97c74ef0590d0a2949f9d3d6096e" + "6bfb50886ddc011066e22adb2d02b7eb" ], [ "Benton2004.RHL.r_while", diff --git a/examples/rel/Benton2004.SmithVolpano.fst.hints b/examples/rel/Benton2004.SmithVolpano.fst.hints index eb0eb6b7a85..cc6ca118003 100644 --- a/examples/rel/Benton2004.SmithVolpano.fst.hints +++ b/examples/rel/Benton2004.SmithVolpano.fst.hints @@ -84,7 +84,7 @@ "typing_FStar.List.Tot.Base.mem" ], 0, - "6cd8c2d2ece32288f89a9ff0240c54ab" + "f1504bffebfd4d656841107a09f396fb" ], [ "Benton2004.SmithVolpano.eval_equiv_def", @@ -579,7 +579,7 @@ "typing_FStar.List.Tot.Base.mem" ], 0, - "d937cd6e60f1cadcd400522591a5dd87" + "d3f72b5266b55da1846ad0a119b31e5f" ], [ "Benton2004.SmithVolpano.exec_equiv_def", diff --git a/examples/rel/Benton2004.fst.hints b/examples/rel/Benton2004.fst.hints index f6e3e1fcfa2..c661020c6b9 100644 --- a/examples/rel/Benton2004.fst.hints +++ b/examples/rel/Benton2004.fst.hints @@ -205,7 +205,7 @@ "well-founded-ordering-on-nat" ], 0, - "e8f637e9644ce289eb622e34f2ea0f38" + "b5183470040865dc0f98ba51a51d01e4" ], [ "Benton2004.fuel_monotonic_while", @@ -246,7 +246,7 @@ "well-founded-ordering-on-nat" ], 0, - "b342b6681cf580e360e35947b53d8f64" + "378b15db96b2e620ee05dc88681f630a" ], [ "Benton2004.while", @@ -1015,7 +1015,7 @@ "unit_typing", "well-founded-ordering-on-nat" ], 0, - "d8e9c5db15524bfacb7f3c0bf702be6d" + "1a31447fb415b173125d351ae4373159" ], [ "Benton2004.d_bre", @@ -1255,7 +1255,7 @@ "well-founded-ordering-on-nat" ], 0, - "925d3c1d5da4447d8e05c12137fcfcdc" + "bbcef345d137d92557b92f0bfd23798c" ], [ "Benton2004.while", diff --git a/examples/rel/IfcDelimitedRelease.fst.hints b/examples/rel/IfcDelimitedRelease.fst.hints index ee11c2cd06d..aa645807aea 100644 --- a/examples/rel/IfcDelimitedRelease.fst.hints +++ b/examples/rel/IfcDelimitedRelease.fst.hints @@ -17,7 +17,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "8cacd503fa47987952d3742611a909d6" + "1243964780d98f5fc67806a6dfdb615f" ], [ "IfcDelimitedRelease.prog", @@ -70,7 +70,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "8ec1b6f96f07b57375e1058cddf061e4" + "8b2713e24d9aebc46585e1dac6a2a27f" ], [ "IfcDelimitedRelease.del_rel", @@ -940,7 +940,7 @@ "well-founded-ordering-on-nat" ], 0, - "65bb4f7bd801d92827d84a4c9c8bd8cd" + "4e5b55a96f3e5ebda7ff983df2c49d20" ], [ "IfcDelimitedRelease.wallet_attack", @@ -1038,7 +1038,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "7b7dac8c27c700287994e1eff192619a" + "883c3886760f28336dd9991cf9f254eb" ], [ "IfcDelimitedRelease.prog", @@ -1091,7 +1091,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "4d825cf4fb9c6d05d8d9049e4eae7d37" + "9b3195b3823be4a5f31cb4227c67ab0b" ], [ "IfcDelimitedRelease.del_rel", @@ -1583,7 +1583,7 @@ "well-founded-ordering-on-nat" ], 0, - "7350d5d84703dced12df04aa92fa27d5" + "3c464f84d0d9d662a5048344290defc5" ], [ "IfcDelimitedRelease.wallet_attack", diff --git a/examples/rel/IfcDelimitedReleaseReify.fst.hints b/examples/rel/IfcDelimitedReleaseReify.fst.hints index b75a7f0d126..d10561f9803 100644 --- a/examples/rel/IfcDelimitedReleaseReify.fst.hints +++ b/examples/rel/IfcDelimitedReleaseReify.fst.hints @@ -1287,7 +1287,7 @@ "well-founded-ordering-on-nat" ], 0, - "0faa5594fafcd60ac2fa2a0d7ac1f859" + "b1ccb0c19b612cfae3f32a5ecd0e5966" ], [ "IfcDelimitedReleaseReify.wallet_attack", @@ -1963,7 +1963,7 @@ "well-founded-ordering-on-nat" ], 0, - "2ab91172b9e91fe2cfe47879897c8ff4" + "36788415a990ed63147445b0e0e185bf" ], [ "IfcDelimitedReleaseReify.wallet_attack", diff --git a/examples/rel/IfcRecursiveReify.fst.hints b/examples/rel/IfcRecursiveReify.fst.hints index c300dd2d24d..f1346618632 100644 --- a/examples/rel/IfcRecursiveReify.fst.hints +++ b/examples/rel/IfcRecursiveReify.fst.hints @@ -34,7 +34,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "49e5b254506e9628fba6f6739976eceb" + "6d1771c0b82cc3c9af87fd8d3ac904b3" ], [ "IfcRecursiveReify.ni_p1", @@ -91,7 +91,7 @@ "unit_typing", "well-founded-ordering-on-nat" ], 0, - "0ce3e356aa24c62a2dd2768af2dfe678" + "9df39862514d990e8c8e88b1e126fa61" ], [ "IfcRecursiveReify.p2", @@ -117,7 +117,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "6d43eae8f09f3b5e14c925c390b68cf2" + "1d019f951a3c26777f65c5e343996c95" ], [ "IfcRecursiveReify.ni_p2", @@ -175,7 +175,7 @@ "unit_typing", "well-founded-ordering-on-nat" ], 0, - "5bd371f46fbf6d060c0780d1d8e806b0" + "c5b45235275a8fee2fc3a6be49eac24f" ], [ "IfcRecursiveReify.ni_p3", @@ -232,7 +232,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "fd6a4b38d2ea1b70634fd42dd98a1c5a" + "922052f6a6239c513c450ec283dd12cc" ], [ "IfcRecursiveReify.p2", @@ -258,7 +258,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "5857970a27d350d6db0e05211d42a438" + "e1a57d83446c35daa175bade4adfa12c" ] ] ] \ No newline at end of file diff --git a/examples/rel/IfcRules.fst.hints b/examples/rel/IfcRules.fst.hints index d14ea55bf26..3507ed7fcd7 100644 --- a/examples/rel/IfcRules.fst.hints +++ b/examples/rel/IfcRules.fst.hints @@ -419,7 +419,7 @@ "unit_inversion", "unit_typing", "well-founded-ordering-on-nat" ], 0, - "54b81f51f557f313de2a4fc17abe634e" + "e76dc0d8d63478af42ce9a1e105da533" ], [ "IfcRules.while_com", diff --git a/examples/rel/IfcRulesReify.fst.hints b/examples/rel/IfcRulesReify.fst.hints index 8bb496088d3..efa31cebaeb 100644 --- a/examples/rel/IfcRulesReify.fst.hints +++ b/examples/rel/IfcRulesReify.fst.hints @@ -1043,7 +1043,7 @@ "well-founded-ordering-on-nat" ], 0, - "c5cf28c13adf5cb929f79eaff0a64c3d" + "6b8b5c8d711915d966b91e32208de835" ], [ "IfcRulesReify.while_ni_com'", diff --git a/examples/rel/IfcTypechecker.fst.hints b/examples/rel/IfcTypechecker.fst.hints index 2fe6e1c83fc..5c0a75c6725 100644 --- a/examples/rel/IfcTypechecker.fst.hints +++ b/examples/rel/IfcTypechecker.fst.hints @@ -38,7 +38,7 @@ "typing_IfcRulesReify.uu___is_Low" ], 0, - "ba5319244ee6a267f26b4e280228d004" + "e3e26631ac3b5044f87d6533605ab3ab" ], [ "IfcTypechecker.tc_com", @@ -197,7 +197,7 @@ "typing_IfcRulesReify.uu___is_Low" ], 0, - "b43a5c7322f99dd86eebd676b36f99b3" + "0bd1e5ca04605e7f96268ed25b5edfe7" ], [ "IfcTypechecker.tc_com", diff --git a/examples/rel/Loops.fst.hints b/examples/rel/Loops.fst.hints index 92a53ccbea5..dab5da1ed16 100644 --- a/examples/rel/Loops.fst.hints +++ b/examples/rel/Loops.fst.hints @@ -19,7 +19,7 @@ "well-founded-ordering-on-nat" ], 0, - "cddef63511e29eec0dfb33db0a597268" + "9625a81c2266e6b8bf7f5ab441dea7bc" ], [ "Loops.sum_up_eq", @@ -73,7 +73,7 @@ "unit_typing", "well-founded-ordering-on-nat" ], 0, - "13f5d68bfdce0717339a2680557a8592" + "93a76c08de296bed6a0127d5c931a050" ], [ "Loops.sum_up_commute", @@ -147,7 +147,7 @@ "well-founded-ordering-on-nat" ], 0, - "cc04db40193b7dc863edf9ef053ca1e2" + "517010122293181805a72914f9ed4035" ], [ "Loops.sum_dn_eq", @@ -201,7 +201,7 @@ "unit_typing", "well-founded-ordering-on-nat" ], 0, - "d945f8d62a6eb85c73bfe41463f62767" + "faaa260a8dfc0ac26edba943f9a104d3" ], [ "Loops.sum_dn_commute", @@ -392,7 +392,7 @@ "well-founded-ordering-on-nat" ], 0, - "f83bbe54847dc8b97513001d31eb85dc" + "7860374234de351b2733284a6c4d40e1" ], [ "Loops.sum_up_eq", @@ -438,7 +438,7 @@ "well-founded-ordering-on-nat" ], 0, - "f3b65d1d2a60d36b7c03cfaad9b60feb" + "2ab07afa2768a3407c3783b82b150690" ], [ "Loops.sum_dn_eq", diff --git a/examples/rel/Memo.fst.hints b/examples/rel/Memo.fst.hints index f21f54bbcff..60a58c04330 100644 --- a/examples/rel/Memo.fst.hints +++ b/examples/rel/Memo.fst.hints @@ -113,7 +113,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "b001be708b0cabd5bcbe2b56c198e5fa" + "0b1147bac9410863bd2f5dc84afecc89" ], [ "Memo.for_all_prop_assoc_lemma", @@ -215,7 +215,7 @@ "subterm_ordering_Prims.Cons", "true_interp" ], 0, - "b5a9a0bb31bed603d37cd680c552b681" + "9c48779d59bb5e73e63e2b6125504597" ], [ "Memo.valid_memo_to_memo_heap", @@ -240,7 +240,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "0c88e9620313f02963b2239e488f7835" + "e9d03aa7423831e30d51d2af43797d6d" ], [ "Memo.valid_memo_id_lemma", @@ -635,7 +635,7 @@ "subterm_ordering_Memo.Need" ], 0, - "bb6cecd7470e2c82b3cd3071d30ff515" + "e214972117302a5a4d362f7183f6e32a" ], [ "Memo.complete_fixp", @@ -647,7 +647,7 @@ "projection_inverse_BoxInt_proj_0", "well-founded-ordering-on-nat" ], 0, - "76370caa2e83984fd23aaf498cc49389" + "6083abe074ab4b1192bf7e419634a092" ], [ "Memo.__proj__Later__item__x", @@ -739,7 +739,7 @@ "projection_inverse_Memo.Need_cont", "subterm_ordering_Memo.Need" ], 0, - "d598c5fe031ebac30fff1abf7cd1f8af" + "aa6ec7e6c5ce0c9be659557260cabe84" ], [ "Memo.fpartial_result_lemma", @@ -767,7 +767,7 @@ "subterm_ordering_Memo.Need" ], 0, - "34d7e7680d2191f46b603174884edeb9" + "0f7bd92aa642c4f87766e9eb9f1d9ff6" ], [ "Memo.valid_memo_rec_lemma", @@ -850,7 +850,7 @@ "typing_Memo_Tm_abs_646741795853dc34eae6a4013bf77e10", "unit_typing" ], 0, - "da53a5edec482fef4778c7f0696f1a51" + "20e26a52fcf507d7d2c660d7931183ff" ], [ "Memo.memo_rec", @@ -922,7 +922,7 @@ "well-founded-ordering-on-nat" ], 0, - "034cb0f76653ee8620abb5d2150facee" + "a8bc26de411c8b72df722eab0fdc482a" ], [ "Memo.complete_memo_rec_extr", @@ -935,7 +935,7 @@ "projection_inverse_LexCons_1", "projection_inverse_LexCons_2" ], 0, - "b66a5971addda6afce36bf838e208224" + "bc33bae1435b2eb0ac7565f50a9920e1" ], [ "Memo.complete_memo_rec_extr", @@ -947,7 +947,7 @@ "projection_inverse_BoxInt_proj_0", "well-founded-ordering-on-nat" ], 0, - "959f39035852971807226a9cb7b93c54" + "3acbd2c87477471fa65ae2dfce2ae5f0" ], [ "Memo.complete_memo_rec_extr_computes", @@ -1096,7 +1096,7 @@ "projection_inverse_Memo.Need_cont", "subterm_ordering_Memo.Need" ], 0, - "ad4001504b8ebedfe6eaf1af41b89f20" + "bb7031614a36d13dd8992779a81d2785" ], [ "Memo.complete_fixp_eq", @@ -1126,7 +1126,7 @@ "subterm_ordering_Memo.Need" ], 0, - "0673a17c3dd650e14dfd1b7d02604c3e" + "ed60efe38444fbebd4c633543a507a0c" ], [ "Memo.complete_fixp_eq", @@ -1144,7 +1144,7 @@ "projection_inverse_BoxInt_proj_0", "well-founded-ordering-on-nat" ], 0, - "94481ba00b686bce608f131eb12d37c1" + "25e6381c58241fa5eaa83125821a339c" ], [ "Memo.fixp_eq", @@ -1182,7 +1182,7 @@ "well-founded-ordering-on-nat" ], 0, - "2a76a31c3f02b9fdbc9595e6f63ec488" + "a46459f81c90aaa7fc831dffc262cfa0" ], [ "Memo.fibo_complete_fixp_eq_proof", @@ -1416,7 +1416,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "f128fdab8c3b7eeb22feb0a83e1a44fc" + "65578902d113da65d6d69ed0d34c0904" ], [ "Memo.memo_heap_to_valid_memo", @@ -1450,7 +1450,7 @@ "subterm_ordering_Prims.Cons", "true_interp" ], 0, - "16037215b5588fba398ae826e4f8cb8d" + "21ff8f6a331ec3eb8c25aa4f2b12948b" ], [ "Memo.valid_memo_to_memo_heap", @@ -1475,7 +1475,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "86e87e147d348bd36d2b24cbed5a1909" + "c753c941bbd7a2c6d22747c3e2869ee2" ], [ "Memo.memo_heap_id", @@ -1681,7 +1681,7 @@ "subterm_ordering_Memo.Need" ], 0, - "8ab1ec8f9672eea8399d0d42feac1072" + "12168f8d9c15bce073e276b1e9bc7771" ], [ "Memo.complete_fixp", @@ -1693,7 +1693,7 @@ "projection_inverse_BoxInt_proj_0", "well-founded-ordering-on-nat" ], 0, - "74bd947ffbd91d15868a4fdfe2fd2316" + "5c5b2760e01aea79bad656794314b7a9" ], [ "Memo.__proj__Later__item__x", @@ -1753,7 +1753,7 @@ "projection_inverse_Memo.Need_cont", "subterm_ordering_Memo.Need" ], 0, - "b73e3aeaf078d3d67f22c224a2c9095a" + "4d84ea5e64e36a7877cd2483920417b4" ], [ "Memo.complete_memo_rec", @@ -1822,7 +1822,7 @@ "typing_Memo_Tm_abs_646741795853dc34eae6a4013bf77e10", "unit_typing" ], 0, - "53e1bc6f8ab9b28d2b3a1c92fa450591" + "4641df2e1dadb52b16277f55caff696b" ], [ "Memo.memo_rec", @@ -1894,7 +1894,7 @@ "well-founded-ordering-on-nat" ], 0, - "a5e8555e8495992b69b32350ce48f796" + "374f53aea361eaf3f21e0dbb8ebe711b" ], [ "Memo.complete_memo_rec_extr", @@ -1907,7 +1907,7 @@ "projection_inverse_LexCons_1", "projection_inverse_LexCons_2" ], 0, - "248cd7ae6ace16f0d9fe38594fcde5ea" + "8e6966a82df7efd01108be2becc40146" ], [ "Memo.complete_memo_rec_extr", @@ -1919,7 +1919,7 @@ "projection_inverse_BoxInt_proj_0", "well-founded-ordering-on-nat" ], 0, - "cf8e3c78b4e970c25d6caea4ce0b631c" + "e81982f463bae8b49392a9a6a2c7ba6e" ], [ "Memo.to_memo_pack_rec", @@ -1952,7 +1952,7 @@ "projection_inverse_Memo.Need_cont", "subterm_ordering_Memo.Need" ], 0, - "2838abb466b45de16087fb18d64ad996" + "fc2b44a77cef80b03876c4c5a6297941" ], [ "Memo.fibonnacci_partial", @@ -1981,7 +1981,7 @@ "well-founded-ordering-on-nat" ], 0, - "b417ad4f2b8a7afad8988f3ef5853554" + "1a5c026005dfde544c0df37cdb69be69" ], [ "Memo.fibo", diff --git a/examples/rel/ProgramEquivalence.fst.hints b/examples/rel/ProgramEquivalence.fst.hints index 6b38fab556a..900c8fef38e 100644 --- a/examples/rel/ProgramEquivalence.fst.hints +++ b/examples/rel/ProgramEquivalence.fst.hints @@ -311,7 +311,7 @@ "well-founded-ordering-on-nat" ], 0, - "09e52394a5db4803bcf4dfb1dacaae42" + "d9311f3f88bd5cde04dffe75b1ac28d2" ], [ "ProgramEquivalence.ref_not_in_fp", @@ -436,7 +436,7 @@ "well-founded-ordering-on-nat" ], 0, - "40e1c35b8e6689d2768c29d53dde2310" + "d00927b527c7c5d9208875dc95d27082" ], [ "ProgramEquivalence.counts_even_numbers", @@ -521,7 +521,7 @@ "well-founded-ordering-on-nat" ], 0, - "0146a17fb1dd6d2ca133d18695bf7d40" + "3ca497ec36306dfbe578f8cc0281b9f5" ], [ "ProgramEquivalence.__proj__C__item__c", @@ -833,7 +833,7 @@ "well-founded-ordering-on-nat" ], 0, - "5ab50ecd9970398f7fe1bd111ad926be" + "d28bad0debaac7958ea672c8096cb283" ], [ "ProgramEquivalence.ref_not_in_fp", diff --git a/examples/rel/ProgramOptimizations.fst.hints b/examples/rel/ProgramOptimizations.fst.hints index 2687ea01785..a569a707d7a 100644 --- a/examples/rel/ProgramOptimizations.fst.hints +++ b/examples/rel/ProgramOptimizations.fst.hints @@ -356,7 +356,7 @@ "typing_FStar.DM4F.Heap.IntStoreFixed.index" ], 0, - "5c89601aaceb3bcd616bced518493adb" + "144795c02240ad381c6e95d7ac699d19" ], [ "ProgramOptimizations.b_exp_denotation", @@ -395,7 +395,7 @@ "subterm_ordering_ProgramOptimizations.Not" ], 0, - "444f2f633f81962b05acd11ca05e3749" + "3ae8347041b793a9ff050bb9ae476841" ], [ "ProgramOptimizations.com_denotation", @@ -427,7 +427,7 @@ "unit_typing" ], 0, - "b05332d73ef1cd84f892b96d09b2f926" + "0bcc99fac6c59a659216124e6ac2d278" ], [ "ProgramOptimizations.g_exp", @@ -658,7 +658,7 @@ "subterm_ordering_ProgramOptimizations.GIOp" ], 0, - "d491ceaec7fea2c78252521fd07a0ba4" + "9597dec75d2941598bfadd837acb37bc" ], [ "ProgramOptimizations.rel_exp_denotation", @@ -685,7 +685,7 @@ "subterm_ordering_ProgramOptimizations.RNot" ], 0, - "d8451f589512fc1ef7ba0d0d80a9d5a9" + "93e46847252dcd420b75c44f2c8968e6" ], [ "ProgramOptimizations.lemma_sound_optimization1", @@ -1515,7 +1515,7 @@ "typing_FStar.DM4F.Heap.IntStoreFixed.index" ], 0, - "ad1e972e31b194b5d78f6e71ebaf8430" + "a24bcea582a09ba119698b3ca8a62afd" ], [ "ProgramOptimizations.b_exp_denotation", @@ -1554,7 +1554,7 @@ "subterm_ordering_ProgramOptimizations.Not" ], 0, - "78e151262534dae61508330552634c99" + "3eabe0ad8e6fe21a1accfae58b23565b" ], [ "ProgramOptimizations.com_denotation", @@ -1586,7 +1586,7 @@ "unit_typing" ], 0, - "60c519b00e6599eb51fc7259f02150ef" + "a72b5cade2b05589a03e41651faeeaa2" ], [ "ProgramOptimizations.g_exp", @@ -1817,7 +1817,7 @@ "subterm_ordering_ProgramOptimizations.GIOp" ], 0, - "113375e1fd9ec7907616a13e4a82ef7d" + "e7ac53210f03e4887f44ce48225efe80" ], [ "ProgramOptimizations.rel_exp_denotation", @@ -1844,7 +1844,7 @@ "subterm_ordering_ProgramOptimizations.RNot" ], 0, - "bce78646d5bf54d0dab8e17991f6153c" + "ffc5fc3a46dc4120554ccc98380c52bf" ] ] ] \ No newline at end of file diff --git a/examples/rel/Recursive.fst.hints b/examples/rel/Recursive.fst.hints index 4fa30488146..9de668787c2 100644 --- a/examples/rel/Recursive.fst.hints +++ b/examples/rel/Recursive.fst.hints @@ -16,7 +16,7 @@ "well-founded-ordering-on-nat" ], 0, - "11d1cf851c0768f03bffeb71e6bc81ec" + "e96ca123b14c5733ab36ca2a12750d8c" ], [ "Recursive.fac_mon", @@ -43,7 +43,7 @@ "typing_Recursive.fac", "well-founded-ordering-on-nat" ], 0, - "7d199eca058b28616170367adcf508b6" + "284ebc7807b2aab9de973adbff1f6519" ], [ "Recursive.fac_sum", @@ -89,7 +89,7 @@ "well-founded-ordering-on-nat" ], 0, - "ddfb331c31ec1fe410fe1341b0f553a0" + "8b45fc9f6821fc08cc41b5a447206ddb" ], [ "Recursive.fac_sum", diff --git a/examples/rel/UnionFind.Forest.fst.hints b/examples/rel/UnionFind.Forest.fst.hints index d966fa97350..0e21880d1a8 100644 --- a/examples/rel/UnionFind.Forest.fst.hints +++ b/examples/rel/UnionFind.Forest.fst.hints @@ -40,7 +40,7 @@ "well-founded-ordering-on-nat" ], 0, - "32263e03d873bb69c5de856301aeea6e" + "afec08c144cd802cb2499375687d90e7" ], [ "UnionFind.Forest.uf_forest", @@ -156,7 +156,7 @@ "well-founded-ordering-on-nat" ], 0, - "3a7765837176f263d6321fe0077fc0cc" + "935373f2907045492a8f09d6f86c99d5" ], [ "UnionFind.Forest.uf_forest", diff --git a/examples/rel/UnionFind.Functions.fst.hints b/examples/rel/UnionFind.Functions.fst.hints index dd9170362f5..a7f27e0b109 100644 --- a/examples/rel/UnionFind.Functions.fst.hints +++ b/examples/rel/UnionFind.Functions.fst.hints @@ -145,7 +145,7 @@ "well-founded-ordering-on-nat" ], 0, - "5d83101126c2049d5422f6ff0da9e311" + "d189ddbe01aedae7f97fc11e5dc0b85e" ], [ "UnionFind.Functions.find_opt", @@ -214,7 +214,7 @@ "well-founded-ordering-on-nat" ], 0, - "af3163b8bea695330c02f4048cd0d791" + "300186daa6dcf01806f3368146a74379" ], [ "UnionFind.Functions.well_formed_decreases_lemma", @@ -530,7 +530,7 @@ "well-founded-ordering-on-nat" ], 0, - "16c6a28bd7aa6807402b760640a8a95b" + "00ef829dd8d4f2f2ee6f33bc1279529f" ], [ "UnionFind.Functions.find_opt", @@ -599,7 +599,7 @@ "well-founded-ordering-on-nat" ], 0, - "d0a8956582f49e06ab2a67be73471d62" + "0e325597b340ea0b57fcf9c4969acea5" ], [ "UnionFind.Functions.well_formed_decreases_lemma", diff --git a/examples/rel/While.fst.hints b/examples/rel/While.fst.hints index d15d72541af..ab8bcdaa764 100644 --- a/examples/rel/While.fst.hints +++ b/examples/rel/While.fst.hints @@ -92,7 +92,7 @@ "fuel_guarded_inversion_While.exp", "subterm_ordering_While.AOp" ], 0, - "f34d0d601f416c89dc82e0808fdc6e04" + "35dcff1394269819508ff6aa623929b9" ], [ "While.__proj__Assign__item__var", @@ -253,7 +253,7 @@ "typing_While.interpret_exp", "well-founded-ordering-on-nat" ], 0, - "af4be0f5bc5e9615b9d05ff49a5d978c" + "57c0f3fc0ddc7cb5ee1867ca75ff2833" ], [ "While.interpret_while", @@ -277,7 +277,7 @@ "well-founded-ordering-on-nat" ], 0, - "eab1e390742b99fa1afe260c9d2ca9a3" + "11d021e9dd5de54a1d720ce77e1b173a" ], [ "While.interpret_exp_st", @@ -426,7 +426,7 @@ "fuel_guarded_inversion_While.exp", "subterm_ordering_While.AOp" ], 0, - "a6701cf36287cb39c4d648e83cf96ca1" + "df3084bf53d897d51fa9b834f6cb2b3d" ], [ "While.__proj__Assign__item__var", @@ -587,7 +587,7 @@ "typing_While.interpret_exp", "well-founded-ordering-on-nat" ], 0, - "ef83c80f8bfd381c23a36f7c74edd706" + "862e69f2ec9d1e71e4b707942ad3e0a3" ], [ "While.interpret_while", @@ -611,7 +611,7 @@ "well-founded-ordering-on-nat" ], 0, - "2afa4f67517e6e8d4d83a8681db07c3d" + "77e5e1d73e12f59f415302644cc29966" ], [ "While.interpret_exp_st", diff --git a/examples/rel/WhileReify.fst.hints b/examples/rel/WhileReify.fst.hints index 0e13af0fe68..e0df76d5fd4 100644 --- a/examples/rel/WhileReify.fst.hints +++ b/examples/rel/WhileReify.fst.hints @@ -255,7 +255,7 @@ "typing_FStar.DM4F.Heap.IntStoreFixed.index" ], 0, - "bfd6a626b0efab2f82dcb8166e0fcfdf" + "952f25d453d0453c5f1a636c3372a8e1" ], [ "WhileReify.interpret_exp'", @@ -303,7 +303,7 @@ "well-founded-ordering-on-nat" ], 0, - "6b9b7825ab31f9bdac29caee6f7fcfc8" + "1a6430ab3706d66dd6fb3a9cfb4b7dde" ], [ "WhileReify.interpret_com", @@ -653,7 +653,7 @@ "typing_FStar.DM4F.Heap.IntStoreFixed.index" ], 0, - "510983485a10a9f85cac2a6e44f2b811" + "b11bb5409b9330477a6f53f2b3599c51" ], [ "WhileReify.interpret_exp'", @@ -701,7 +701,7 @@ "well-founded-ordering-on-nat" ], 0, - "8c7c00f58745529535a10b7f981ba1f5" + "9cbd0e321efad42277d47b536c7615e4" ], [ "WhileReify.interpret_com", diff --git a/examples/seplogic/Examples.fst.hints b/examples/seplogic/Examples.fst.hints index 853076fd700..4c52803944c 100644 --- a/examples/seplogic/Examples.fst.hints +++ b/examples/seplogic/Examples.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "b97bf5c8bf44f95495e6e56ce5694f0d" + "bec1b5695b0a3301e2f18f363b9230fd" ], [ "Examples.increment_ok", @@ -25,7 +25,7 @@ "unit_inversion", "unit_typing" ], 0, - "866de3e12e02f29e842d48e46caf9148" + "52ce4d6e4a7133b41e970dde5f8099bb" ], [ "Examples.increment_ok", @@ -40,7 +40,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "bee807a7ce1681621e66c41aa8e46771" + "993e29095131ab0b38603b321efb63a0" ], [ "Examples.increment_ok", @@ -61,7 +61,7 @@ "typing_FStar.SL.Monotonic.Heap.points_to" ], 0, - "af44563676cb0b32cdf23b69b4675dec" + "9c31a077a3890357e15d74712c267bd9" ], [ "Examples.swap_ok", @@ -74,7 +74,7 @@ "true_interp" ], 0, - "a0c7a6b76e2237f200c9027b8a2bf8a9" + "c8a51b8b47a466a6800d0bd7215c3e04" ], [ "Examples.swap_ok", @@ -86,7 +86,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "ae3c361589e5587429e85494be64e438" + "c02a5d367fe92d0b82bacb538c06c0d2" ], [ "Examples.swap_ok", @@ -104,7 +104,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "da9b035fb3d31015a3868af9dfe0dd22" + "fbe588dc5d0e16731196c04696b7e167" ], [ "Examples.swap_ok", @@ -116,7 +116,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "91108d36bcc4c42eea237971f02f8c74" + "919beb0f62b682c6af8a64461b2141bc" ], [ "Examples.swap_ok", @@ -135,7 +135,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "93accffb6d6162a623135a386f7b34eb" + "c7adf0203758a1e53374610a4a6add96" ], [ "Examples.swap_ok", @@ -161,7 +161,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "a2b0c7870f93b1559e767472a0ded6da" + "035d761ba622bf149db0726a82d435b2" ], [ "Examples.swap_ok", @@ -180,7 +180,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "77aa327336bd875ee4524e37d21f5b8d" + "53657d7bbab9e146d34315018b7d8437" ], [ "Examples.swap_ok", @@ -201,7 +201,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "55d38b293a1950a5c7bb7c1efb77c54a" + "264e043fae3b505488002ab4cd5c4060" ], [ "Examples.swap_ok", @@ -222,7 +222,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "e4687864167186b1b38e854f7b7e2fc9" + "242b44912068ac1fa7622e0cedb0f5e9" ], [ "Examples.double_increment_ok", @@ -237,7 +237,7 @@ "unit_inversion", "unit_typing" ], 0, - "5140f977cd1eab92c9b90b49ec10dbe1" + "24e58e8b13457706dc0ef447ad0c636e" ], [ "Examples.double_increment_ok", @@ -252,7 +252,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "7e9dd07e8a8d1fbd6b36ce6158d11d11" + "ca638cd3e41828a41a01c5e9138b418a" ], [ "Examples.double_increment_ok", @@ -270,7 +270,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "5257f0d68317b0ffb65f1e17e10f7b03" + "c3e61769b6ac2b4fa098daaf4e0a2ffa" ], [ "Examples.double_increment_ok", @@ -289,7 +289,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "5847a669c054425051a343193b7303b7" + "c9634b17356e91b4d6763a47b5673d2c" ], [ "Examples.double_increment_ok", @@ -329,7 +329,7 @@ "typing_FStar.UInt64.v" ], 0, - "969658a6235e2efe840b3665429ca319" + "582b6aa8f8dd0663566c22019eb87d6c" ], [ "Examples.init_ok", @@ -369,7 +369,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "d55bc27a6315ac3e9a1d0da483790fe2" + "fefcfc56507ecde5427ab72915d347cc" ], [ "Examples.init_ok", @@ -407,7 +407,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "48f2224c1e26e3dc6e11a25a0afc010b" + "c7c97998293cf87f0264ef27f829395d" ], [ "Examples.copy_ok", @@ -423,7 +423,7 @@ "true_interp" ], 0, - "e6050ce8863dacd84d499c93fce7fc87" + "1f2d20e7d1823352f0242621a054514f" ], [ "Examples.copy_ok", @@ -438,7 +438,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "d2ee1aea9fd54b5e9a7004c60fb6e1e1" + "d6294e5c93c3ee818add94ef4bb99c3b" ], [ "Examples.copy_ok", @@ -456,7 +456,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "5e30d6b091c81d01ee7dad3e3901542c" + "6dde9ce40b5ee53dfc34d02bedb12c9b" ], [ "Examples.copy_ok", @@ -474,7 +474,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "a0a9f22f9012194d89e4077504eb021b" + "e60f708d355a293ee6961bb0838e1c03" ], [ "Examples.copy_ok", @@ -495,7 +495,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "5d3b22aabff9099b08bf05df653d71cc" + "064e17c07b53677247f19a229516303f" ], [ "Examples.copy_ok", @@ -513,7 +513,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "811d1fe84c961d2e9d4fc9ced1ef5e0b" + "e1e818ae08ba880ec96e69814066f7a1" ], [ "Examples.copy_ok", @@ -525,7 +525,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "2c1e276af33fc51d7ed8ce6af71780e2" + "49de80b4a20df978f9d61ab134c5cb05" ], [ "Examples.copy_ok", @@ -537,7 +537,7 @@ "refinement_interpretation_Examples_Tm_refine_27e663d45ab46f5b4e6a1f9a37782360" ], 0, - "4cd9dbfd392010f8eee51fe5e08922d6" + "eac1cedd99d7808ef246e0cc5eecb953" ], [ "Examples.write_ok", @@ -546,7 +546,7 @@ 1, [ "@query" ], 0, - "fb2ef98cff1850587c58966700ec4842" + "79838da13700fec768b98ead008fe714" ], [ "Examples.increment_ok", @@ -555,7 +555,7 @@ 1, [ "@query" ], 0, - "4943e94d0c26ed3847eb34fac940a921" + "fb8731edd402d38ab3cc11a2ddf77c71" ], [ "Examples.increment_ok", @@ -570,7 +570,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "675484e602bf6783d1e7625d4865ef66" + "6d18ce5870be0a6409d2028a4479ba5a" ], [ "Examples.increment_ok", @@ -591,7 +591,7 @@ "typing_FStar.SL.Monotonic.Heap.points_to" ], 0, - "deec094a9dd53a4527e2d1715fe84a9b" + "05dc649bbd076a23b2e2976d07f197d5" ], [ "Examples.swap_ok", @@ -604,7 +604,7 @@ "true_interp" ], 0, - "42b25cd3769d9f4895164a5c6d64c09b" + "2118960b1deec99f6c79b40b4e2c1861" ], [ "Examples.swap_ok", @@ -613,7 +613,7 @@ 1, [ "@query" ], 0, - "d419090d131e32cebdc1173a4bc4c7c1" + "eb9a4d2f5bc7c7c5b558f67528951558" ], [ "Examples.swap_ok", @@ -631,7 +631,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "72c04983f2671f3c20839775a7138255" + "3e9e585627985fa1eb9bb3e571c952c7" ], [ "Examples.swap_ok", @@ -643,7 +643,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "5a2899c5266612b43014e05d33553a7b" + "7f352b0a148b8cab3f8323c911728753" ], [ "Examples.swap_ok", @@ -662,7 +662,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "993c4904abc6ba742d2040adc8cff7f6" + "ce0b44232b586ecca53a3b04f6e514f2" ], [ "Examples.swap_ok", @@ -688,7 +688,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "1c036320fbf183f41f5f60c99cc4acaa" + "d62ca5983a558667743dd97f363b49cb" ], [ "Examples.swap_ok", @@ -707,7 +707,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "fd0aa48b55f7c99beba52bd142863510" + "4f486d29943c3cffb35a14fe777d6ea5" ], [ "Examples.swap_ok", @@ -728,7 +728,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "fbe119bffadb0104118936d0478e8df7" + "6e6387fd7e3e5440d5085d2e691177dc" ], [ "Examples.swap_ok", @@ -749,7 +749,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "d0e0a931782babd93ea2a53614116ad6" + "32003f8582a39dc9aa1eaf13ce53b8b3" ], [ "Examples.double_increment_ok", @@ -758,7 +758,7 @@ 1, [ "@query" ], 0, - "e59177ee1def68d19219979fe6f62199" + "c74f51daf6a2c517a7a7a9c7a04b6ee4" ], [ "Examples.double_increment_ok", @@ -773,7 +773,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "2bd0492e9a61b906ea99c693cd11598b" + "94da360a14fb81a27045f5f7bbe85cf6" ], [ "Examples.double_increment_ok", @@ -791,7 +791,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "bd90fa96a97a61b5ca0d679804ce4bdb" + "ee4df91994681e4ddb5842d9139439d2" ], [ "Examples.double_increment_ok", @@ -810,7 +810,7 @@ "typing_FStar.SL.Monotonic.Heap.get_next_addr" ], 0, - "03dd532f0c5425b0ed65bf233239a373" + "63791ddd9a5fae0bbe7571f9fe35509e" ], [ "Examples.double_increment_ok", @@ -850,7 +850,7 @@ "typing_FStar.UInt64.v" ], 0, - "4843973516e3c813e73025505c7599ad" + "fa6d234ed1876705c11c540a793f7df6" ], [ "Examples.init_ok", @@ -890,7 +890,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "2651086abd9002bca1b628505765d595" + "78520b58e300fb9c3ecf175cd6e995bb" ], [ "Examples.init_ok", @@ -928,7 +928,7 @@ "typing_FStar.UInt64.uint_to_t", "typing_Prims.pow2" ], 0, - "a47789a250ff80a1364840a55e2bb237" + "80216d5669fe748d4c2132c6089ac72c" ], [ "Examples.copy_ok", @@ -944,7 +944,7 @@ "true_interp" ], 0, - "df9b5426495283fe7f170982566cefc9" + "22df93959f2d2c1e97a458d280807326" ], [ "Examples.copy_ok", @@ -953,7 +953,7 @@ 1, [ "@query" ], 0, - "b08a0833a69c0f5460f893509ccdcc19" + "10dc7b3e110e9b9189189b7f645ecb37" ], [ "Examples.copy_ok", @@ -971,7 +971,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "25910747fc5f7d1af13f157b85142b51" + "d0cb137bd05992d0170c751fefa1feb9" ], [ "Examples.copy_ok", @@ -989,7 +989,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "322ad8f395ee2c417fb260183bdc5100" + "77a14e2b64216e96c5adc6296e490498" ], [ "Examples.copy_ok", @@ -1010,7 +1010,7 @@ "typing_FStar.SL.Monotonic.Heap.sel" ], 0, - "f4e7f2550832374c9710624a261ba394" + "fe111cf9211edbf2481fa8c5e324b0e5" ], [ "Examples.copy_ok", @@ -1028,7 +1028,7 @@ "typing_FStar.SL.Heap.trivial_preorder" ], 0, - "db994e2d44666a9226a5ba9f4e6ee81f" + "4fa3bd5bc4f7741d2b40d836bbb477f4" ], [ "Examples.copy_ok", @@ -1040,7 +1040,7 @@ "primitive_Prims.op_disEquality", "projection_inverse_BoxBool_proj_0" ], 0, - "9cb81b89a5729d56df1512ff60b14ac3" + "b47e146d7b9f2d8d1bbdfe60de7cdc2f" ], [ "Examples.copy_ok", @@ -1052,7 +1052,7 @@ "refinement_interpretation_Examples_Tm_refine_27e663d45ab46f5b4e6a1f9a37782360" ], 0, - "d824432101ab054713c9fbd659854d1b" + "1c7d565688e310389d0da1c777f45bac" ] ] ] \ No newline at end of file diff --git a/examples/seplogic/SL.Examples.fst.hints b/examples/seplogic/SL.Examples.fst.hints index 8eede0f301c..804de91e7e6 100644 --- a/examples/seplogic/SL.Examples.fst.hints +++ b/examples/seplogic/SL.Examples.fst.hints @@ -12,7 +12,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "228743b070cedc2840611d8626ec0062" + "da64178325735d6c619e349480fb7734" ], [ "SL.Examples.lemma_rw", @@ -21,7 +21,7 @@ 1, [ "@query", "typing_SL.Heap.op_Bar_Greater" ], 0, - "9168ba1936221879b499041a4078dd33" + "3a2c2daae73ae717dc164ef86c4314a1" ], [ "SL.Examples.lemma_bind", @@ -33,7 +33,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "a3d97e478ef7bcf1b34c995b534a1125" + "da50637201600714699dc6e70ff5e5d1" ], [ "SL.Examples.lemma_singleton_heap_procedure", @@ -46,7 +46,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "f4eb54f6cec6baf7be01579eb18456f8" + "8cb6cb8b56b66dc2717798af1361ad4b" ], [ "SL.Examples.lemma_procedure", @@ -55,7 +55,7 @@ 1, [ "@query" ], 0, - "ac1abf946f14d36da34a6737e2c11be7" + "68a5824c3a75c3f2ff762a0303fbf53b" ], [ "SL.Examples.lemma_pure_right", @@ -67,7 +67,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "080d54d776573325a670c92bd6e02e55" + "08ab793e0f5137432c056e72d73a66f6" ], [ "SL.Examples.lemma_rewrite_sep_comm", @@ -76,7 +76,7 @@ 1, [ "@query" ], 0, - "78aa2bb3be25112fad5f24a400f4482c" + "8814dbb31f3cd004b150d203f9ec8442" ], [ "SL.Examples.lemma_rewrite_sep_assoc1", @@ -85,7 +85,7 @@ 1, [ "@query", "lemma_SL.Heap.lemma_sep_assoc" ], 0, - "5a26df8e2de33575feb0094ce8eaf916" + "59295a0e34c97a6a1ae4c2ce9c8f5e70" ], [ "SL.Examples.lemma_rewrite_sep_assoc2", @@ -94,7 +94,7 @@ 1, [ "@query", "lemma_SL.Heap.lemma_sep_assoc" ], 0, - "053ae5ef18f430d140eaaec1cb8fedc7" + "af26001a891f591e9031063147d70ad3" ], [ "SL.Examples.lemma_rewrite_sep_assoc3", @@ -103,7 +103,7 @@ 1, [ "@query", "lemma_SL.Heap.lemma_sep_assoc" ], 0, - "0b2f62f1c707ba7907c6d096de6e2743" + "f3f8b79ee3bc1e9e9ac7019b8fe6613a" ], [ "SL.Examples.lemma_rewrite_sep_assoc4", @@ -112,7 +112,7 @@ 1, [ "@query", "lemma_SL.Heap.lemma_sep_assoc" ], 0, - "f85d73cdafd4cb403d72bbb619d101e8" + "086478178dd07de504146995fd4a7204" ], [ "SL.Examples.apply_lemmas", @@ -124,7 +124,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "deed58a5643e68206ca252115466e82e" + "d70917a3bb73e60d8d0b7ca257ee5a94" ], [ "SL.Examples.prelude", @@ -147,7 +147,7 @@ "typing_FStar.Tactics.Result.uu___is_Success", "unit_typing" ], 0, - "0b3076ad5adee9212401a44dc4b60ca6" + "8d6e0c7a5d6960716ff0c461999eceda" ], [ "SL.Examples.split_lem", @@ -159,7 +159,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "d46c48e50fc69c77aae733b8c9aa9a77" + "dfed68ac652670bdb740f444f978f600" ], [ "SL.Examples.write_read", @@ -171,7 +171,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_0139bf7052c09762f3fd33651746d3b5" ], 0, - "923f5e1927fa0ba95e90091d3d220d72" + "91bcc831387122631d8146ea80c821a5" ], [ "SL.Examples.write_read", @@ -199,7 +199,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "529bc2ed85bba7853bbfce703f2122e4" + "c2e39e8c62463902712912e61115d17a" ], [ "SL.Examples.write_read", @@ -224,7 +224,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "e051ff9c81254f0e7acd746bb2486aa5" + "507af2c402b6cd62c99f1b6de58626eb" ], [ "SL.Examples.swap", @@ -236,7 +236,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_c9caf63a45faa2fe57fd3bb4c51c320c" ], 0, - "7ae088855e51c61bed1daec5492dad00" + "8265fa27cfce4abe5d03f4e3e0153b86" ], [ "SL.Examples.swap", @@ -248,7 +248,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_c9caf63a45faa2fe57fd3bb4c51c320c" ], 0, - "fc0350d28c62656a48d64deab30e9408" + "a6993e8a018566925aba2483370debd2" ], [ "SL.Examples.swap", @@ -262,7 +262,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "bc117de922dabdd8e2e16db8c8ee4ff2" + "e768fe2537ee60394e846d3e663553e0" ], [ "SL.Examples.swap", @@ -276,7 +276,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "d1ac0cba6a7e79397bb8d6d66e20938b" + "5d86d74609c44284b173991cdec452c9" ], [ "SL.Examples.swap", @@ -288,7 +288,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_c9caf63a45faa2fe57fd3bb4c51c320c" ], 0, - "655d029e9faa35fc3b9ff9445b382976" + "25e9298106ac570b6d079f865edb8271" ], [ "SL.Examples.swap", @@ -316,7 +316,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "3c083a6281278cc3e7c56abd06732530" + "1a0d4df12adbc80c17fbe8afc902dfca" ], [ "SL.Examples.swap", @@ -350,7 +350,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "a85d1688c18d3f6191a6789e55c88911" + "5ee0d0378c545c210b0a229f49e2bfb3" ], [ "SL.Examples.incr", @@ -363,7 +363,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "f49191081cce15c4f14c31bbd47606df" + "56fbc9b40ce67348cd98e8aedff14d99" ], [ "SL.Examples.incr", @@ -376,7 +376,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Bar_Greater" ], 0, - "3e5b664f66f692a2b603b33d34d4e4f9" + "c686670eeb452f8423e32606b58e2d43" ], [ "SL.Examples.incr", @@ -393,7 +393,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "44906d295e2b9b5c755ae324ab97f840" + "256cecca77251c17285bfaed18eb474c" ], [ "SL.Examples.incr", @@ -411,7 +411,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "4c0908141db9d9a67e64a954351f95ff" + "ab7a1229648c35702d8d8808e0c8cb83" ], [ "SL.Examples.incr2", @@ -423,7 +423,7 @@ "lemma_SL.Heap.lemma_points_to_defined" ], 0, - "42e2bbd6fce962bde8d107f75418df25" + "547fd0274c58f95dc9f1efadde845bfc" ], [ "SL.Examples.incr2", @@ -440,7 +440,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "cf23b9a133f30a818d595cb1bec1c426" + "d188c6f315609fb7fc89bd4557a89c1c" ], [ "SL.Examples.incr2", @@ -460,7 +460,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "8c217daea89c900049861b41a2cba155" + "fb73b1947979b3876ef9e8e9e25f687c" ], [ "SL.Examples.rotate", @@ -475,7 +475,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "916eb4d2da7bf281f05d023dc081fa2e" + "fe9088770bcfe446fc58994bf1cf84f2" ], [ "SL.Examples.rotate", @@ -493,7 +493,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "d5e860b4bde2d25ce24293f69bcfba8b" + "d57051e20211e3f2ff5d5581b9ac0476" ], [ "SL.Examples.rotate", @@ -526,7 +526,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "fa4b718cc4d9219e0724b6d64e2c0fde" + "143bce6695139f8dbc0b9974e5285881" ], [ "SL.Examples.rotate", @@ -557,7 +557,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "ca34ef33fffc02e82f4d6cfd185ded21" + "e4e2c56be9626d103ce149b7c6b18fcd" ], [ "SL.Examples.rotate", @@ -586,7 +586,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "9f3f6792a623ead1dfc0200fe0654838" + "dc54f63da48a212fbe02c8546fdcb3e8" ], [ "SL.Examples.rotate", @@ -617,7 +617,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "08a96e0f60958d58eba80a29f7393213" + "d1a328e505fab3bc573c5e28cd415bab" ], [ "SL.Examples.rotate", @@ -648,7 +648,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "e78962ce008df3d8d994af3e94c2c4cf" + "451e5bcbdaadbede8e9dcb23ee508cc1" ], [ "SL.Examples.rotate", @@ -679,7 +679,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "052fe4ea2570d61cd55bbc5097800684" + "b70f4f03fb18be6262ba1dd9b0822289" ], [ "SL.Examples.rotate", @@ -716,7 +716,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "337ab7f2b17bf27f27ad956e57557b45" + "6fc39ff6ef32a1e970b44e6459692b56" ], [ "SL.Examples.lemma_inline_in_patterns_two", @@ -728,7 +728,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "0a7faa6f6f5b27af8ef7385b48e60945" + "d870c5c8921a8d587816e1373ba6e409" ], [ "SL.Examples.lemma_frame_out_empty_right", @@ -740,7 +740,7 @@ "lemma_SL.Heap.lemma_sep_unit" ], 0, - "cca26e9ff2527b35c9fd209499d704ed" + "d744f14d51fba65dc1bc1f6e045d0781" ], [ "SL.Examples.lemma_frame_out_empty_left", @@ -752,7 +752,7 @@ "lemma_SL.Heap.lemma_sep_unit", "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "9c25650ebd1b77e4a75995bef65e6929" + "3fa20e25d516c2d2f34b5ba273cf4a10" ], [ "SL.Examples.cond_test", @@ -764,7 +764,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_3e8850268c538ad9254730979b04971f" ], 0, - "b55f0793ffc0133dc6eabb8ea2670d1a" + "f0fad1021ae45d9976cc62a1ee76459e" ], [ "SL.Examples.cond_test", @@ -776,7 +776,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_3e8850268c538ad9254730979b04971f" ], 0, - "486b26f123e73d893c46984c8223c697" + "508f9a269ea514872fc2889f92a2fc2d" ], [ "SL.Examples.cond_test", @@ -788,7 +788,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_3e8850268c538ad9254730979b04971f" ], 0, - "92653e41729b31e433cb678c199fd80e" + "7c53212447e409430f03de3735bda45c" ], [ "SL.Examples.cond_test", @@ -800,7 +800,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_3e8850268c538ad9254730979b04971f" ], 0, - "6b5069ceab186895d098e319364658f1" + "7ed4a27004d5056d3c21c92585ce810b" ], [ "SL.Examples.cond_test", @@ -828,7 +828,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "31811b1367a94f9bc5935d5713e8ac79" + "24b6712cbc9f172f96d68d70f1af9181" ], [ "SL.Examples.cond_test", @@ -870,7 +870,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "4d47e6cc574589940989795631acba8c" + "590672cc73558585bccfd227364492c5" ], [ "SL.Examples.cond_test", @@ -882,7 +882,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_3e8850268c538ad9254730979b04971f" ], 0, - "3eca39094dbf738984661e34956f8f24" + "fd33ed1d52116a0effdc8b7a6f44af90" ], [ "SL.Examples.cond_test", @@ -896,7 +896,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "cec82b2ad4df31d32d05c3131962c831" + "ffdbb1e8cce5af9d62c3ff6bcf5fc924" ], [ "SL.Examples.cond_test", @@ -925,7 +925,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "978ae6e0b5b6b74a686296a3e89d63e9" + "5eb89002c1e3dae9cdd73774f6b8bb03" ], [ "SL.Examples.cond_test", @@ -954,7 +954,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "3c6cfbf539d4efb6674fdf95a07deef4" + "e9d41ebdb0da7fa84d0a857ce67c0cc3" ], [ "SL.Examples.cond_test", @@ -989,7 +989,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "156fceb9e8ccb07758a22638f6f6d9f0" + "201d2e1e0165bc294878ae5df8cf9491" ], [ "SL.Examples.cond_test", @@ -1021,7 +1021,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "aed674c2a5c7522d0c63e1fa1abe2490" + "2bbb4f1db9da631ca3d67c98fd664546" ], [ "SL.Examples.cond_test", @@ -1054,7 +1054,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "688cb1872815af5e359648104767624f" + "6859c92f50ad04a3f8665a629656d6b8" ], [ "SL.Examples.cond_test", @@ -1066,7 +1066,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_8a5eac184ae64109676f362e58afe491" ], 0, - "73c3afa95882a6d46eabad653b647761" + "250134500ec303db1cfa4d277d011ce5" ], [ "SL.Examples.valid", @@ -1084,7 +1084,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "e2982008cf52128d928f46dbe323491e" + "2c07d2d4a629bad8bc6da1d37c8f6e1f" ], [ "SL.Examples.__exists_elim_as_forall2", @@ -1093,12 +1093,12 @@ 1, [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", - "equation_Prims.squash", "l_quant_interp__7797", + "equation_Prims.squash", "l_quant_interp__7823", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5", "refinement_interpretation_SL.Examples_Tm_refine_7070d46f3c3cb717e23b2dabcbc4c12c" ], 0, - "86c2424254fcc1b5b3a11a736c4a115b" + "14347a62866774112bfac883d9691e06" ], [ "SL.Examples.__exists_elim_as_forall1", @@ -1107,12 +1107,12 @@ 1, [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", - "equation_Prims.squash", "l_quant_interp__7801", + "equation_Prims.squash", "l_quant_interp__7827", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5", "refinement_interpretation_SL.Examples_Tm_refine_d16de86ec5446f55c1622708945a0449" ], 0, - "66e1d213230b5abd1d436ea4a10e5859" + "442026a0ec796382652843cab57d426a" ], [ "SL.Examples.__elim_valid_without_match", @@ -1137,7 +1137,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "96b566c0a27f5f43b2bbca048c3cc9ff" + "ca10523cbdecf447d76c0dad4876a5de" ], [ "SL.Examples.lemma_frame_exact", @@ -1146,7 +1146,7 @@ 1, [ "@query" ], 0, - "ac98b0762962d818d307a83d9d62a71e" + "30c8210bb4ca5a9defb5fe405154d303" ], [ "SL.Examples.length", @@ -1155,7 +1155,7 @@ 1, [ "@query", "assumption_SepLogic.Heap.Emp_defined_axiom" ], 0, - "67ec650fc15ad446d23114391b9feedc" + "903dc316ea6242c89a8f9e22bc0ed0b6" ], [ "SL.Examples.length", @@ -1164,7 +1164,7 @@ 1, [ "@query", "assumption_SL.Heap.Emp_defined_axiom" ], 0, - "93138e9753bc5a7e9784cce9a56da58b" + "49421b8d2b668d6b2a349d1a351dcfaa" ], [ "SL.Examples.length", @@ -1177,7 +1177,7 @@ "lemma_SepLogic.Heap.lemma_sep_unit" ], 0, - "7bd5f210872510e994d63b6b7e9bdf1d" + "e7c0cb3b8e8ed9d4fde819dac891b37b" ], [ "SL.Examples.length", @@ -1189,7 +1189,7 @@ "function_token_typing_SL.Heap.emp", "lemma_SL.Heap.lemma_sep_unit" ], 0, - "9ff93f63527599aa5314f4b3b5263f2b" + "e5a341fe47fea181f9c21c1ee822d198" ], [ "SL.Examples.length", @@ -1206,7 +1206,7 @@ "projection_inverse_Prims.Nil_a" ], 0, - "22addabf724d550d0778d8ee124d0efc" + "1dcc9c8233f99ca712b3ced7114b2ee4" ], [ "SL.Examples.length", @@ -1219,7 +1219,7 @@ "projection_inverse_FStar.Pervasives.Native.None_a" ], 0, - "b390a8d21a5a6c217742be4bd5b5d2e2" + "3e3f9c336e0d478de73096367d187b5c" ], [ "SL.Examples.length", @@ -1232,7 +1232,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "e9ab72259e8d1cc3af2ba0340f620600" + "ebfd7bd80cbebb158802d88c03cad406" ], [ "SL.Examples.length", @@ -1247,7 +1247,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "49aae2e1afe3a9b97b1394fe1418dda3" + "4797dd783ad0d509549b01646288be27" ], [ "SL.Examples.length", @@ -1262,7 +1262,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "4f8106e5d62da9cf35147adf572f4b85" + "d7a2ef15f2859fdd8b8e63a3fa718b1e" ], [ "SL.Examples.length", @@ -1279,7 +1279,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "d1fc8c30bc05aa7a545fd911b3d1c654" + "5d9c4482aaf2ec9025dc2a2c879f7a43" ], [ "SL.Examples.length", @@ -1296,7 +1296,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "e77740c939e46255c957fa719a68420a" + "0ee42349af4093d66fad8c36f902b255" ], [ "SL.Examples.length", @@ -1313,7 +1313,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "7a0f46ef7d9d3ed978a2970723688c4d" + "2c79ec4c97627386459adea3b9b7429a" ], [ "SL.Examples.length", @@ -1330,7 +1330,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "4d1128eb51102bf59be40e8640052b2a" + "2cad323085153ad283a0b1572211ad94" ], [ "SL.Examples.length", @@ -1354,7 +1354,7 @@ "typing_SL.Heap.op_Bar_Greater", "unit_inversion", "unit_typing" ], 0, - "0b8cc6251d4ef2c00cf48686453fc93c" + "cd43bf3044b5966f8c7888407abefca9" ], [ "SL.Examples.length", @@ -1367,7 +1367,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_412e9f270f624237a204a51cd01783c1" ], 0, - "cdc8bc2967b7d045c16a8fc90fe10330" + "73e35bf8ee15b618a5d86d32338b110a" ], [ "SL.Examples.length", @@ -1391,7 +1391,7 @@ "typing_SL.Heap.op_Bar_Greater", "unit_inversion", "unit_typing" ], 0, - "94dd05112e2930828d664bb457401f32" + "62bf326cd6015f1ff8d91618dbe9b398" ], [ "SL.Examples.length", @@ -1415,7 +1415,7 @@ "typing_SL.Heap.op_Bar_Greater", "unit_inversion", "unit_typing" ], 0, - "316a0efdb674cb6e7ecf6a6ee57beec8" + "236a021abdaf4cb8c69d29e0b84b37ba" ], [ "SL.Examples.length", @@ -1452,7 +1452,7 @@ "unit_typing" ], 0, - "3caa677fba048e455e9d0a99315dd98a" + "8e4d555438cddb9bb1ed0ff6969eec14" ], [ "SL.Examples.length", @@ -1480,7 +1480,7 @@ "unit_typing" ], 0, - "755aa64bc6b1b8160de69f76e8ee0eb7" + "c1fbbc94254aecf5e17a99cd4ad3d56c" ], [ "SL.Examples.length", @@ -1508,7 +1508,7 @@ "unit_typing" ], 0, - "51966893135a9d2d36c0e74d22ac1359" + "a05e9f8b95e7a20b3e887dfdc8669be8" ], [ "SL.Examples.length", @@ -1537,7 +1537,7 @@ "unit_typing" ], 0, - "a7ac4a9e7911b76e88d8872dc5c3f0e5" + "4607bcd04e230c12b66a8f7feb17b0df" ], [ "SL.Examples.length", @@ -1566,7 +1566,7 @@ "unit_typing" ], 0, - "8448a362557b500bd949db63a00e8640" + "814d09cf7ce1cc6d096ee1277ffe8bbc" ], [ "SL.Examples.length", @@ -1595,7 +1595,7 @@ "unit_typing" ], 0, - "90a83ca4b193f8d056304c7fff91935e" + "7267f39d64315b42cdae17a9fa29eec2" ], [ "SL.Examples.length", @@ -1624,7 +1624,7 @@ "unit_typing" ], 0, - "4178600702778137ff6eff55a14d8285" + "d04be455a0788b1c1b4a5d0d04d30bf6" ], [ "SL.Examples.length", @@ -1653,7 +1653,7 @@ "unit_typing" ], 0, - "5e719b40b8a6586966fc6455fd0b0f82" + "7a05644f206dea0fe88e5845f9d64da7" ], [ "SL.Examples.length", @@ -1682,7 +1682,7 @@ "unit_typing" ], 0, - "7444f30a4e2af8bcd3299558cd0ad41b" + "40fa5c3ca23c0385ec6776ac1f140b7d" ], [ "SL.Examples.length", @@ -1711,7 +1711,7 @@ "unit_typing" ], 0, - "7f909668ddd7036117d6e261d79293e1" + "937511ed429fff9ce9eb3ec2b0b07998" ], [ "SL.Examples.length", @@ -1740,7 +1740,7 @@ "unit_typing" ], 0, - "b6deef93814cfce0c70f5283bd45dc7b" + "884db0238bfef94041c93347baaf7b84" ], [ "SL.Examples.length", @@ -1758,7 +1758,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some", "typing_SL.Heap.ref" ], 0, - "e8e7b20687f897d119b43c6c356c4f49" + "a68006dc4114345add5f15b6d02edcdf" ], [ "SL.Examples.length", @@ -1787,7 +1787,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "45d92e5156a5219cc04ebfe35d49647a" + "92bc040494c46b23692cba9f23d82b52" ], [ "SL.Examples.append", @@ -1799,7 +1799,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "0f35cb02660901627cb6402d48e16ac6" + "f242b0a37b4719fba8ab3a27b95a8b56" ], [ "SL.Examples.append", @@ -1811,7 +1811,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "7ae30189f99b590a13281895c5651350" + "a99428038798a860eac061b8d6073d2e" ], [ "SL.Examples.append", @@ -1823,7 +1823,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "a3a1848aa673fa5863837be7df5eee8f" + "57e2202b661a92dd5e416d3e187aebcc" ], [ "SL.Examples.append", @@ -1837,7 +1837,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "bbea8333a073fed3de48c6cbb7ff71cd" + "be40a1639eccad07bf22cf14063690fa" ], [ "SL.Examples.append", @@ -1869,7 +1869,7 @@ "function_token_typing_FStar.UInt32.n", "function_token_typing_SL.Heap.emp", "int_inversion", "int_typing", "kinding_SL.Examples.listcell@tok", "l_and-interp", - "l_quant_interp__7792", "lemma_SL.Heap.lemma_addrs_in_join", + "l_quant_interp__7818", "lemma_SL.Heap.lemma_addrs_in_join", "lemma_SL.Heap.lemma_sep_assoc", "lemma_SL.Heap.lemma_sep_comm", "lemma_SL.Heap.lemma_sep_defined", "lemma_SL.Heap.lemma_sep_unit", "proj_equation_FStar.Pervasives.Native.Some_v", @@ -1886,7 +1886,7 @@ "unit_typing" ], 0, - "350dfb1645e9cdd2156379ebace2080b" + "0aa6a1750e317a5166dbcff063e25918" ], [ "SL.Examples.append", @@ -1901,7 +1901,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_333995310cc67a2191c689eaa0bcbaa3" ], 0, - "75443ec74757bfc031b7fe1c4aa4a7d8" + "442daeff6459d8eebe851e9f8dbe10fa" ], [ "SL.Examples.append", @@ -1916,7 +1916,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_135a58b9e2191af079c261fa72d0209d" ], 0, - "be14d3850058a1f280ca2dcfaee03717" + "6297c747b48dff93f70f6f74ff350901" ], [ "SL.Examples.append", @@ -1928,7 +1928,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "944d17c2a6826f0a764917dae131bfe0" + "747316f13ee1ee18875540be0766cb42" ], [ "SL.Examples.append", @@ -1940,7 +1940,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "cc4f12c18d6df05928d55f6d10e0040d" + "0d9bb66b248b5a88973124e0599a7bfa" ], [ "SL.Examples.append", @@ -1958,7 +1958,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "4147598d39c0e7f08a6e3213f5f57873" + "42a6e562b48d9e7ed76a9a8b160ddfe8" ], [ "SL.Examples.append", @@ -1976,7 +1976,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "f15667341ee2421e03d47d02f33b225c" + "db07fe8ba1ffd9e1e1747332636f17a7" ], [ "SL.Examples.append", @@ -1994,7 +1994,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "94cdd4789d0cd1084cd065816dd4368f" + "780b5f95dd065398031dd37438241d65" ], [ "SL.Examples.append", @@ -2012,7 +2012,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "faed616392a74debb5e88b0c3e81d48e" + "ec810b9f7d8219a2add2c66be042e2c6" ], [ "SL.Examples.append", @@ -2030,7 +2030,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "6302bb56163d7ede5d2f360c2782107a" + "e69c52824ac35b9989c380e6ec31aafc" ], [ "SL.Examples.append", @@ -2052,7 +2052,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "3b40b5d589c9bee3cd9dce2b5e506a78" + "bba763a7955a6694ce4b921dc087c256" ], [ "SL.Examples.append", @@ -2080,7 +2080,7 @@ "unit_typing" ], 0, - "43235ea1b85008215f0de8de5b978025" + "e550d450a9d75ba7937b88f767c87010" ], [ "SL.Examples.append", @@ -2121,7 +2121,7 @@ "unit_typing" ], 0, - "2b388fb6c403671a722383061285edf9" + "4adc18b2879f4c535c961a07350b9c7e" ], [ "SL.Examples.append", @@ -2162,7 +2162,7 @@ "unit_typing" ], 0, - "0fd91441edf13b1356c23bf9b6d9cdab" + "a18b78f3f6b2edd24e3cb3597d31e160" ], [ "SL.Examples.append", @@ -2207,7 +2207,7 @@ "unit_typing" ], 0, - "83c50d987eaa7a05fa9c879f805a67a0" + "8a663601d68ed453bee5554b3118a7b0" ], [ "SL.Examples.append", @@ -2252,7 +2252,7 @@ "unit_typing" ], 0, - "eda5c9247f91c54682b2023b5c373c46" + "e44e2d523a47fcf60b360ce9583339cb" ], [ "SL.Examples.append", @@ -2297,7 +2297,7 @@ "unit_typing" ], 0, - "6dd2528a395b4057d91108cd0585545c" + "e5537507a9f79f30a223eddd4e140849" ], [ "SL.Examples.append", @@ -2342,7 +2342,7 @@ "unit_typing" ], 0, - "7d43165212bff1f2e5b854fada08dcbe" + "4a2c4cd079de6b527c57a286fc5b5369" ], [ "SL.Examples.append", @@ -2387,7 +2387,7 @@ "unit_typing" ], 0, - "88834299b544d58932de13a7789c5896" + "cf93a26cd4697c1882eb8ee69391b045" ], [ "SL.Examples.append", @@ -2432,7 +2432,7 @@ "unit_typing" ], 0, - "2baa815fab77554f7a5b96b415befa95" + "71c96bc021e697a8fa6b4c86b2449768" ], [ "SL.Examples.append", @@ -2477,7 +2477,7 @@ "unit_typing" ], 0, - "c284e08fc3223111ac0eb1e000ca525b" + "2333161e07810bea7ee64296675fb250" ], [ "SL.Examples.append", @@ -2522,7 +2522,7 @@ "unit_typing" ], 0, - "0cb0832a76aededfd5180583507446ad" + "5854c5ffe00a25e3e7f6b0fbdfbdade9" ], [ "SL.Examples.append", @@ -2567,7 +2567,7 @@ "unit_typing" ], 0, - "10fd8de1f14f3cb246a594e45624959a" + "075418ac39c3b888ba5cdeddddc9d7ac" ], [ "SL.Examples.append", @@ -2612,7 +2612,7 @@ "unit_typing" ], 0, - "701b1fa1878838d930988c638701b58f" + "1d999937765b9315dc84b1069130a1fe" ], [ "SL.Examples.append", @@ -2657,7 +2657,7 @@ "unit_typing" ], 0, - "79d6c47f3f38a11c750196dcd931a35e" + "1d32bf776603308a29da65107d75cb28" ], [ "SL.Examples.append", @@ -2702,7 +2702,7 @@ "unit_typing" ], 0, - "ae69b5fbebe35b635836120c899d3aaf" + "45f0bf28d7281d63bc1b8ffd675d7208" ], [ "SL.Examples.append", @@ -2741,7 +2741,7 @@ "function_token_typing_Prims.int", "function_token_typing_SL.Heap.emp", "int_inversion", "int_typing", "kinding_SL.Examples.listcell@tok", "l_and-interp", - "l_quant_interp__7792", "lemma_FStar.Set.disjoint_not_in_both", + "l_quant_interp__7818", "lemma_FStar.Set.disjoint_not_in_both", "lemma_FStar.Set.lemma_equal_elim", "lemma_FStar.Set.lemma_equal_intro", "lemma_FStar.Set.mem_intersect", "lemma_FStar.Set.mem_union", "lemma_SL.Heap.lemma_addrs_in_join", @@ -2775,7 +2775,7 @@ "unit_typing" ], 0, - "f339c6d62703d759391fa9f85500f62f" + "ea358197103f1e9fc2e1b3d9e050db94" ], [ "SL.Examples.append", @@ -2842,7 +2842,7 @@ "unit_typing" ], 0, - "05b48580229fe73ed7d0ae58e848d8ae" + "f973af5d635c3d77822000f689c0a85e" ], [ "SL.Examples.append", @@ -2860,7 +2860,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "3494284c37b80bc78273398df1b204d0" + "eea40522fbecf10fc1374074bb7fd5b7" ], [ "SL.Examples.append", @@ -2878,7 +2878,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "8cb444768044485b8eddf8531d43db74" + "47a16f9a1da4b5a802085cc7bff69cd5" ], [ "SL.Examples.append", @@ -2914,7 +2914,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "34549002924aaf4f3b0f5ff135365afe" + "ec08a721f0f30aeec500772197807974" ], [ "SL.Examples.append", @@ -2950,7 +2950,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "9e9b8dfcb5bf5750fefe8a020e81f1c4" + "74503a744f7ee3faa10ca2a5805e6a8f" ], [ "SL.Examples.append", @@ -3008,7 +3008,7 @@ "unit_typing" ], 0, - "324f9a8d42d7a7473755c50f2f0b0392" + "7f4df6b0beec6ad8aeb0dac559fcb097" ], [ "SL.Examples.append", @@ -3066,7 +3066,7 @@ "unit_typing" ], 0, - "d47d603e0560406051996c282ae3d5c9" + "b6839964c8dae580f3c579b095c555bf" ], [ "SL.Examples.append", @@ -3104,7 +3104,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "c953ae930284a06173baf09bfa79bc17" + "85517c8f1679ad5b38ebaf7bc5e96fa1" ], [ "SL.Examples.append", @@ -3142,7 +3142,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "03d4abaff962b86ce8e61c48fbb46d3d" + "680d0e041b1780a94436f28c7494f46c" ], [ "SL.Examples.append", @@ -3196,7 +3196,7 @@ "unit_typing" ], 0, - "894c15c3ba4e138995ffc8294730da9a" + "0e83ef888a3e36c2f37c7786ce946a56" ], [ "SL.Examples.append", @@ -3250,7 +3250,7 @@ "unit_typing" ], 0, - "398054517d585ecc272452c91ae9cf03" + "42f7e92033c68b01e0e4ccaae16e240f" ], [ "SL.Examples.append", @@ -3304,7 +3304,7 @@ "unit_typing" ], 0, - "859b8cf4c46d2f047576d0cd40bc55d3" + "dd20355a3fb47d09a1c27a2c8e46ff68" ], [ "SL.Examples.append", @@ -3358,7 +3358,7 @@ "unit_typing" ], 0, - "696d1b33b01fe5e37c66671b8a527a72" + "c87966f31de801c772456a30212f5053" ], [ "SL.Examples.append", @@ -3412,7 +3412,7 @@ "unit_typing" ], 0, - "6be662abe8fcf9ab99bf86823750157b" + "f833174a9ff71812ba0fc01356454979" ], [ "SL.Examples.append", @@ -3466,7 +3466,7 @@ "unit_typing" ], 0, - "189aee79dbfb3e3a499a0a05aa64823c" + "2b0c2c28c65e965728d7b092cc0c385d" ], [ "SL.Examples.append", @@ -3520,7 +3520,7 @@ "unit_typing" ], 0, - "98017f70fe33eca228e61be632a14c54" + "4439416fb6d78716c7df76162d97eed1" ], [ "SL.Examples.append", @@ -3574,7 +3574,7 @@ "unit_typing" ], 0, - "4694d7e7bd039a26c1cab0fb74f256a1" + "125626a6e23f05b8018837d07dbd8df4" ], [ "SL.Examples.append", @@ -3612,7 +3612,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "3f0e150255fb4494b4b9600bd5613b8f" + "d27cf6810d0d8c08fdb39de09f909767" ], [ "SL.Examples.append", @@ -3650,7 +3650,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "beb657482e661ca18706adfa3f54a638" + "6caf87c89186e0a4991860ab0d233809" ], [ "SL.Examples.append", @@ -3688,7 +3688,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "c3a98819a0981eb43693f398c4e654de" + "5edc62838bf5cbd893278af9d87b1a1e" ], [ "SL.Examples.append", @@ -3726,7 +3726,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "bf00019cc5acd25a8a4aaa120c2b8824" + "3f1da924b476eff0beae79c27a1e9df8" ], [ "SL.Examples.append", @@ -3764,7 +3764,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "e7839345b60e89322fc64a30f4df5b21" + "d835b1575b74981a9d801b62dff7e463" ], [ "SL.Examples.append", @@ -3782,7 +3782,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some", "typing_SL.Heap.ref" ], 0, - "4a1eed141f4efe31080f83d04f9772fd" + "5bb10435e93a90e07741e9a4fee11197" ], [ "SL.Examples.append", @@ -3800,7 +3800,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some", "typing_SL.Heap.ref" ], 0, - "c0cc7907fbbca35e78014de92afe57aa" + "b9ea4c0eb5e1fde130b8128716b28dd9" ], [ "SL.Examples.append", @@ -3837,7 +3837,7 @@ "function_token_typing_SL.Examples.null", "function_token_typing_SL.Heap.emp", "int_inversion", "kinding_SL.Examples.listcell@tok", "l_and-interp", - "l_quant_interp__7792", "lemma_FStar.Set.lemma_equal_elim", + "l_quant_interp__7818", "lemma_FStar.Set.lemma_equal_elim", "lemma_FStar.Set.lemma_equal_refl", "lemma_SL.Heap.lemma_addrs_in_join", "lemma_SL.Heap.lemma_addrs_in_points_to", @@ -3872,7 +3872,7 @@ "unit_inversion", "unit_typing" ], 0, - "e8229c8d87e952a2fc72ee3bf33f0e5c" + "47e3092692099d7e0a00a3d1119da567" ], [ "SL.Examples.lemma_apply_rewrite_assoc_mem1", @@ -3884,7 +3884,7 @@ "lemma_SL.Heap.lemma_sep_comm" ], 0, - "cb33071a465d1ed66a1f031fb2dc5154" + "bf5dd63cd5214460adb1759549390106" ], [ "SL.Examples.rev_append", @@ -3896,7 +3896,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "49704ed2937b56e2d5b0a534d3503296" + "7986b1575072a3ba754f06345d0b36d3" ], [ "SL.Examples.rev_append", @@ -3908,7 +3908,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "a1e70275976585657a0d417654844feb" + "f4e43c640c6d15a6209e115e6314383e" ], [ "SL.Examples.rev_append", @@ -3920,7 +3920,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "56014b5c3bc52c0e540cd7ee5b2fdede" + "ca23e7df3a8be5cfa8226322f0f0ca63" ], [ "SL.Examples.rev_append", @@ -3934,7 +3934,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_8002c79ae42ff92c4edc4d769192262d" ], 0, - "5fc3c6760bd7a0109840f2e95bacfcd6" + "709bce13f60268f0509e6bc816eeb806" ], [ "SL.Examples.rev_append", @@ -3965,9 +3965,9 @@ "fuel_guarded_inversion_Prims.list", "function_token_typing_FStar.UInt32.n", "function_token_typing_Prims.int", - "function_token_typing_SL.Heap.emp", "int_inversion", "int_typing", + "function_token_typing_SL.Heap.emp", "kinding_SL.Examples.listcell@tok", "l_and-interp", - "l_quant_interp__7792", "lemma_SL.Heap.lemma_addrs_in_join", + "l_quant_interp__7818", "lemma_SL.Heap.lemma_addrs_in_join", "lemma_SL.Heap.lemma_sep_assoc", "lemma_SL.Heap.lemma_sep_comm", "lemma_SL.Heap.lemma_sep_defined", "lemma_SL.Heap.lemma_sep_unit", "proj_equation_FStar.Pervasives.Native.Some_v", @@ -3985,7 +3985,7 @@ "unit_typing" ], 0, - "2bd950ae01a16aed74133ee1fa241696" + "5109294cf4545b02976c7c0d97867fe2" ], [ "SL.Examples.rev_append", @@ -4000,7 +4000,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_333995310cc67a2191c689eaa0bcbaa3" ], 0, - "71f4a48e7e3b557a0e7c8f1fba5f6526" + "30aab4de0e6f7e1d950d2e6fdbd3b610" ], [ "SL.Examples.rev_append", @@ -4015,7 +4015,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_135a58b9e2191af079c261fa72d0209d" ], 0, - "f77b926833f649db2b640c912efdabf7" + "353b5a5ee194586edef1fab61e8667ea" ], [ "SL.Examples.rev_append", @@ -4027,7 +4027,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "e4d7dd2277c7a7563c9125756c6b146d" + "b0f0268ca2f75d443943e74765a0b211" ], [ "SL.Examples.rev_append", @@ -4039,7 +4039,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_fe2aacf66542bf88fcf16f74c0c1bf03" ], 0, - "a2cb3ec32d72a82ae90a9f9d10d165a4" + "84a2551ebffc2d1551d61c44dddfacf4" ], [ "SL.Examples.rev_append", @@ -4057,7 +4057,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "efbf6e3f8e1fa67230065d720d80bdc3" + "e06ce063821152e3bb2588543db708f6" ], [ "SL.Examples.rev_append", @@ -4075,7 +4075,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "20b1c04b5cc6a3a2127f501d87fc300f" + "8bec1ca10b57c512593945e0244b22be" ], [ "SL.Examples.rev_append", @@ -4093,7 +4093,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "bb578ac5a1817f9d52556503b167b24c" + "0288d539089a60f03599efd20d3c4bbc" ], [ "SL.Examples.rev_append", @@ -4111,7 +4111,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "87ab81f8db2be2ae565e142e9c8db17f" + "6d917eafc71c83b23d93717aff013a27" ], [ "SL.Examples.rev_append", @@ -4129,7 +4129,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "c0279e78d7470cfdeb51cb5f7781c9ba" + "d426c869ecfc3adcd764d40337940ec3" ], [ "SL.Examples.rev_append", @@ -4163,7 +4163,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "98ce261936778863d21588f003ec3087" + "e868c2f947da2299bcec072a26f69b93" ], [ "SL.Examples.rev_append", @@ -4197,7 +4197,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "bb669dda8e3dd66dc8748cdc98b82eb0" + "5bb08cb28219880a8543f33c00587b8d" ], [ "SL.Examples.rev_append", @@ -4236,7 +4236,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "c805cb4ff42e8d99e0bdb31027d4dda1" + "e3573e5829723184014473396c994c93" ], [ "SL.Examples.rev_append", @@ -4249,7 +4249,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_412e9f270f624237a204a51cd01783c1" ], 0, - "7c4693c149767a1dc455796f47cfef9f" + "747205a902c6dd9cd98a75c86a6d8a97" ], [ "SL.Examples.rev_append", @@ -4281,7 +4281,7 @@ "function_token_typing_SL.Examples.null", "function_token_typing_SL.Heap.emp", "kinding_SL.Examples.listcell@tok", "l_and-interp", - "l_quant_interp__7792", "lemma_FStar.Set.lemma_equal_elim", + "l_quant_interp__7818", "lemma_FStar.Set.lemma_equal_elim", "lemma_FStar.Set.lemma_equal_intro", "lemma_FStar.Set.lemma_equal_refl", "lemma_FStar.Set.mem_empty", "lemma_FStar.Set.mem_intersect", "lemma_FStar.Set.mem_union", @@ -4313,7 +4313,7 @@ "unit_typing" ], 0, - "5a449a266d4c7fef20891f2eca96ff13" + "93e9c2a5e4b534516fa37e3100518ba7" ], [ "SL.Examples.rev_append", @@ -4332,7 +4332,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_b1a34bf5909291ee0006341a36798700" ], 0, - "9fa752172cf2596b29adad390a29d59e" + "9d13b9dd33cdc6f57c4693b6f1f1228c" ], [ "SL.Examples.rev_append", @@ -4351,7 +4351,7 @@ "refinement_interpretation_SL.Examples_Tm_refine_b1a34bf5909291ee0006341a36798700" ], 0, - "afe4a55955535a94f7f932a5dced0400" + "52ce42250d701fd69c12241d2fcc6845" ], [ "SL.Examples.rev_append", @@ -4372,7 +4372,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "559f97d2596bd510c09870dbb5814f2e" + "1c9e1cf8820559377ec0bda6759ab830" ], [ "SL.Examples.rev_append", @@ -4393,7 +4393,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "9dce435ee8eae8b00a619f6baa655f72" + "5797d5359baa08b3670c859ee8b1fdb9" ], [ "SL.Examples.rev_append", @@ -4414,7 +4414,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "b6a13417b0da39055481bfdf699f436e" + "3567be9062fb215546923d323f79c360" ], [ "SL.Examples.rev_append", @@ -4435,7 +4435,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "5a6a9855da6f0cfd8abd236416231295" + "d732a58e1aebe1ae96cc5f296a56fd8d" ], [ "SL.Examples.rev_append", @@ -4456,7 +4456,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "088f3a62032c0aa989f8fd1fe80f7092" + "5217015d364a29f5c9f042f209e597f6" ], [ "SL.Examples.rev_append", @@ -4477,7 +4477,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "410b1eb8d2382dfe1bc92e88ea92a2d8" + "39218ab104d6e64d4440d1d72b4ac964" ], [ "SL.Examples.rev_append", @@ -4498,7 +4498,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "724fbe45f8f6e8e62b70d8d37087a5e4" + "4b7ed253c01bcab3d212842d18fa39b4" ], [ "SL.Examples.rev_append", @@ -4520,7 +4520,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "33f2b1770627bb89412e2ef999061c21" + "e30f34ecfa986efb20e0690f8a7008ef" ], [ "SL.Examples.rev_append", @@ -4542,7 +4542,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "b2a7da80597a49f5d26071b32ce17ec0" + "7331e08bd04367e58c6e1f1a19c7abaa" ], [ "SL.Examples.rev_append", @@ -4560,7 +4560,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some", "typing_SL.Heap.ref" ], 0, - "b4bf0d7842b723fa005be40becbca806" + "68a6ea9d003129f36ae32e60e6edbc0f" ], [ "SL.Examples.rev_append", @@ -4621,7 +4621,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "f11e7e3a9976ef70f8332fa790a4f867" + "5f50dae1e3ad533b27c4085ca01325c0" ], [ "SL.Examples.equal_dom", @@ -4633,7 +4633,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "10602c3de62b074c3eaf34dab9498c1f" + "a573ac86d915b029881ee0c0e8426f06" ], [ "SL.Examples.rev", @@ -4670,7 +4670,7 @@ "typing_SL.Heap.addrs_in", "unit_inversion", "unit_typing" ], 0, - "8c9c3eaf7d01a33e9c30bf1a35c86d0d" + "0e9f1478ae5e612f83942fecfe4fd9b9" ] ] ] \ No newline at end of file diff --git a/examples/seplogic/SL.ExamplesAuto.fst.hints b/examples/seplogic/SL.ExamplesAuto.fst.hints index 88ab15dd2f6..2d9b35c5a08 100644 --- a/examples/seplogic/SL.ExamplesAuto.fst.hints +++ b/examples/seplogic/SL.ExamplesAuto.fst.hints @@ -11,7 +11,7 @@ "lemma_SL.Heap.lemma_sep_comm" ], 0, - "4a76ac9bc9a9028ad8a3ff4682e33ed6" + "1f0a4996a9c808412a5e7d416917dc10" ], [ "SL.ExamplesAuto.footprint_of", @@ -28,7 +28,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "function_token_typing_FStar.Reflection.Types.name", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -36,7 +36,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "ed03af1245545f62f7a53351eef718a7" + "98eb434cd7391ff97deecac3efe27bc4" ], [ "SL.ExamplesAuto.frame_wp_lemma", @@ -50,7 +50,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "88ed4a6c0cdac040c54666d55604d9fc" + "e515ca0d1e64f62aab8559ee858fc767" ], [ "SL.ExamplesAuto.ite_wp_lemma", @@ -63,7 +63,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "7d5cc5444d9ea181a5393215b8521ce0" + "7577ebbf199438164b21bdb12445276f" ], [ "SL.ExamplesAuto.if_then_else_wp_lemma", @@ -77,7 +77,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "5701ac4a96ff9d7126fe89a812e8c7c9" + "601a5705fb472fa6b870efde5a305546" ], [ "SL.ExamplesAuto.close_wp_lemma", @@ -87,11 +87,11 @@ [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", "equation_Prims.squash", "equation_SL.Effect.st_close_wp", - "l_quant_interp__19618", + "l_quant_interp__19670", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "751d202a1ac255680ef03dee11b10679" + "c0d3bab61cc47843f37393fa8d68d6bc" ], [ "SL.ExamplesAuto.assume_p_lemma", @@ -105,7 +105,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "4b205353462e9041c3448c696ec61c92" + "c78c08431440fd345650a05e691ad89d" ], [ "SL.ExamplesAuto.pointsto_to_string", @@ -120,7 +120,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "function_token_typing_FStar.Reflection.Types.name", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -128,7 +128,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "deb5805fab4ec52f523f9cf3ba3856ca" + "59c2a16fd85f67afb846cf7ed6f93cc0" ], [ "SL.ExamplesAuto.sort_sl_correct", @@ -146,7 +146,7 @@ "token_correspondence_CanonCommMonoid.sortWith" ], 0, - "8332cf3fb827824d885fe49a1d9e6dd0" + "abcd6fb07ec07dab255d1b42e9de16f3" ], [ "SL.ExamplesAuto.__proj__Frame__item__ta", @@ -160,7 +160,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_7b96c44bc1723c750211be32c4326057" ], 0, - "743e055070effe6ec7a6b05253d752c6" + "9fc99375d8b8f09df7a16a585684c300" ], [ "SL.ExamplesAuto.__proj__Frame__item__twp", @@ -174,7 +174,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_7b96c44bc1723c750211be32c4326057" ], 0, - "e30c57bce66a9547ace57d7ae9a1033a" + "26c8a261b921bf10259f11b04d92f775" ], [ "SL.ExamplesAuto.__proj__Frame__item__tpost", @@ -188,7 +188,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_7b96c44bc1723c750211be32c4326057" ], 0, - "9b0939473e9630db185c4a61dcc85e37" + "38c8a1ce2621aa1ccae677305373eedc" ], [ "SL.ExamplesAuto.__proj__Frame__item__tm", @@ -202,7 +202,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_7b96c44bc1723c750211be32c4326057" ], 0, - "3e134caa5a5c2aab1db1015bc3312aa3" + "c4f88f88b120f6e24ec99188bee2a252" ], [ "SL.ExamplesAuto.__proj__Unknown__item___0", @@ -216,7 +216,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_3eb8fee3b8fcd7b6207497a8ddf9490a" ], 0, - "7059cda264347d32cf11884f30a8172d" + "822c813547948344ffac2e8a0371849e" ], [ "SL.ExamplesAuto.peek_cmd", @@ -234,7 +234,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "function_token_typing_FStar.Reflection.Types.name", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -242,7 +242,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "04e3ddd81698b433e6eeae93c200ae24" + "15a1c9d32c1ac4d74751b87bbd47c059" ], [ "SL.ExamplesAuto.unfold_first_occurrence", @@ -254,7 +254,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "f2112fc495d983e53d9ab44965e1b827" + "8082fbf082d78fbd1684edec4dcb499a" ], [ "SL.ExamplesAuto.__tcut", @@ -267,7 +267,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "2be59c7cea33ed30127ba36931dd4a6e" + "b0b9f8d85aa63109b3708f1da7c1fe86" ], [ "SL.ExamplesAuto.sl", @@ -301,7 +301,7 @@ "typing_SL.ExamplesAuto.__proj__Unknown__item___0" ], 0, - "98d3e82f9b483a6b5f099f71fcfb8f76" + "ceadfb7821409a927274c2c40daf08c6" ], [ "SL.ExamplesAuto.__elim_exists_as_forall", @@ -310,12 +310,12 @@ 1, [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", - "equation_Prims.squash", "l_quant_interp__19857", + "equation_Prims.squash", "l_quant_interp__19909", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5", "refinement_interpretation_SL.ExamplesAuto_Tm_refine_d16de86ec5446f55c1622708945a0449" ], 0, - "17dcd2e31d9b6f8ff3864745fe288da3" + "f9972daa3b8cc8b49c49a9293bd63c29" ], [ "SL.ExamplesAuto.swap", @@ -347,7 +347,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "bfb9569b3766b91a0118d8d87018e14a" + "5c33e8b9f62f606570d8ad09b805f75f" ], [ "SL.ExamplesAuto.swap", @@ -376,7 +376,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "b8528f436427bab83500bbcf6a67cbdb" + "ff6cd4760749360a15abb1f8fabe00fb" ], [ "SL.ExamplesAuto.swap", @@ -405,7 +405,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "f184e7cf6133ad8ecefdaa9c70af5ea4" + "2abcd27a1b1acf84dba3817a14e8004c" ], [ "SL.ExamplesAuto.swap", @@ -435,7 +435,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "733b6d182cfadd5efef80eacb3dc6d34" + "916281b5d729c4fe8036f4691546bd91" ], [ "SL.ExamplesAuto.swap", @@ -465,7 +465,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "37e670d703ce98220960f38a52e173fc" + "f90c7c2d57ebef18a0dba8df580d6726" ], [ "SL.ExamplesAuto.swap", @@ -497,7 +497,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "2f97b3bc2361b9f4f6e89aaf154c34fd" + "8a38fa01edf7a8d80983e4604f8cb9bc" ], [ "SL.ExamplesAuto.swap", @@ -530,7 +530,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "d68d91eb4ec9cb428fc5444179c0511b" + "3cc2b4fa1c5c0c4a430d13eb1070e3fa" ], [ "SL.ExamplesAuto.swap", @@ -550,7 +550,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "2bc1c494ad905c1e18d0643741c9503a" + "41078baa8f57ef6898423a69bb53ed46" ], [ "SL.ExamplesAuto.swap", @@ -570,7 +570,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "5ecb7283bed2f30fdfbc635ae5a933af" + "0a232f16df5b1c2cfda084ab3454ec4c" ], [ "SL.ExamplesAuto.rotate", @@ -602,7 +602,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "645e8e63258146c0b120d0a02804bfbb" + "6203541a7371426e3c9aa53f45de4528" ], [ "SL.ExamplesAuto.rotate", @@ -639,7 +639,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "4ba760ef9d03bb87995f10f783f5ade2" + "e85fc0487a69db56c036e30e0700bc8d" ], [ "SL.ExamplesAuto.rotate", @@ -674,7 +674,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "8285ef427d84aeb17184eabdeac7194d" + "2d92f4fd5119c734c1b74461db00cb17" ], [ "SL.ExamplesAuto.rotate", @@ -694,7 +694,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "813f1f57cd5e40705f1a4ae54c055b3b" + "2a8e1bb4edbcdb8d24fc1cd7163d69d1" ], [ "SL.ExamplesAuto.rotate", @@ -714,7 +714,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "64a67d6a69c6ba5e28a6932ab909b6ef" + "2c367d88aee97082fd6912838b9f3ce0" ], [ "SL.ExamplesAuto.test", @@ -726,7 +726,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_8bfca1b807f3b95890cf7a960b4ff61e" ], 0, - "e7a857abb49681100eeb252170d6530b" + "008ea1dba0f794d6e106715b3a591c8f" ], [ "SL.ExamplesAuto.test", @@ -740,7 +740,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_8bfca1b807f3b95890cf7a960b4ff61e" ], 0, - "d0d4ddd5a651f1db6fca9b3ace41fdde" + "090d73d56ef9ddb3c60ef05d6599e135" ], [ "SL.ExamplesAuto.test", @@ -754,7 +754,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_8bfca1b807f3b95890cf7a960b4ff61e" ], 0, - "0b84b93663858ae48e5526eb446eb53f" + "15ef563ee9a52d7c428f6ce63dffafc4" ], [ "SL.ExamplesAuto.write_read", @@ -781,7 +781,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "5ced53479766b4c8f9d5720b45e81789" + "7d61ea4eef6b022324c1d4956158e232" ], [ "SL.ExamplesAuto.write_read", @@ -801,7 +801,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "38f9b6e4124675513f59da39c9fec6a1" + "8b2282f144518a4d1ca194f218f2748f" ], [ "SL.ExamplesAuto.write_read", @@ -821,7 +821,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "bb0d4bfbbef58d71ffd26240c13820b4" + "3119ed5d5d967404df673a1acc6ca441" ], [ "SL.ExamplesAuto.write_read", @@ -842,7 +842,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "3aff3feec006efc26bbc3203ca1d1d9c" + "2c45fbe4a5efcd57761f2c85cbc12316" ], [ "SL.ExamplesAuto.write_read", @@ -863,7 +863,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "81de33008d1e342c6024081c0c854ee6" + "0a996efa3a784f077d6f028c8cf34840" ], [ "SL.ExamplesAuto.read_write", @@ -895,7 +895,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "96cd86d0e62c2b40555fbac1b3201f83" + "e8e33f2f7e7539de8f57df498fcfa56c" ], [ "SL.ExamplesAuto.read_write", @@ -924,7 +924,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "1fbe6f5362edff8abb6814913c3d4116" + "6ab1842ad773fa03ff5c3a4a5a65cfcf" ], [ "SL.ExamplesAuto.read_write", @@ -953,7 +953,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "75b3165ccc301739f5a46080edd50f65" + "45ac5310dd059be50013142016304c69" ], [ "SL.ExamplesAuto.read_write", @@ -973,7 +973,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "ac4c5aeeaffe56402045fef1a6f97932" + "0acc486e8cb7324d38f99325ef01e28f" ], [ "SL.ExamplesAuto.read_write", @@ -993,7 +993,7 @@ "typing_SL.Heap.op_Bar_Greater" ], 0, - "e761e99cc268eee8ea05dbb07150a095" + "62238369537109163188ed6d5408848d" ], [ "SL.ExamplesAuto.cond_test", @@ -1005,7 +1005,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "6c65d925171fa4988c910a1c0544298c" + "16d4a66de9845dc6c7430fed29f59561" ], [ "SL.ExamplesAuto.cond_test", @@ -1030,7 +1030,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "fde5d65e9d523a48f06970ed91236850" + "bdb7e2a99e51e500f32460bf8d924438" ], [ "SL.ExamplesAuto.cond_test", @@ -1043,7 +1043,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_ef1494113268b111e11d71f440b8d0ec" ], 0, - "75b606be442eb723b524d91def72afed" + "e64bd5adadd20173a15b7dde5effdd64" ], [ "SL.ExamplesAuto.cond_test", @@ -1056,7 +1056,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_ef1494113268b111e11d71f440b8d0ec" ], 0, - "13eade6af4e3e004f57c595f7804c570" + "eb0bbb1e13732334011adefd295891ae" ], [ "SL.ExamplesAuto.cond_test", @@ -1081,7 +1081,7 @@ "typing_SL.Heap.addrs_in", "typing_SL.Heap.op_Bar_Greater" ], 0, - "d5fbf11cc421524c688cf11abaa485de" + "209a57ea3922cbb75f3b087e8ae72556" ], [ "SL.ExamplesAuto.cond_test", @@ -1094,7 +1094,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_ef1494113268b111e11d71f440b8d0ec" ], 0, - "0c260c9bfd10dfc4ca656f1c4fe95e91" + "d07403de8058a0ed87412035b9df4412" ], [ "SL.ExamplesAuto.cond_test", @@ -1107,7 +1107,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_ef1494113268b111e11d71f440b8d0ec" ], 0, - "6c194428d59d65ee1b7193868bac6bad" + "0dfd93c515aef34cc792b65867e31b09" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -1119,7 +1119,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "e19e349bb26e7f7722779c030f383256" + "7fcfeb3c34c6ad19915ffc74f49ba131" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -1152,7 +1152,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "efb838f44d71ab9f3711057e9fec0c77" + "6dbb4bf43ab8e784329dec06e0b84d57" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -1168,7 +1168,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "4e365bc20fd1472b81fefa2fdb768af2" + "fe6756686ae95e90da69b5148383c518" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -1184,7 +1184,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "926bea2894cfd3e16182c3daa3d54665" + "4ad9f7789189eec9dffdad02b967a088" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -1217,7 +1217,7 @@ "typing_SL.Heap.op_Less_Star_Greater" ], 0, - "7c52e91d222edcf277430315399acf21" + "b4f65488b3f4cf21b0668bf35dec0fc8" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -1230,7 +1230,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_f584ac7f9e02ea51fdd9f4acf0063cf9" ], 0, - "93d9996ec1e38e9b2e131ee37b88206b" + "8dc585f2289b31cacde6730ae97675da" ], [ "SL.ExamplesAuto.rotate_left_or_right", @@ -1243,7 +1243,7 @@ "refinement_interpretation_SL.ExamplesAuto_Tm_refine_f584ac7f9e02ea51fdd9f4acf0063cf9" ], 0, - "7fa52be39ceba3ad8eddc8ef67f68b3a" + "8929fb5cb21e502edbdb08d1e2ace87e" ] ] ] \ No newline at end of file diff --git a/examples/software_foundations/SfBasic.fst.hints b/examples/software_foundations/SfBasic.fst.hints index 7a59cc9205f..c0df2c9b6dd 100644 --- a/examples/software_foundations/SfBasic.fst.hints +++ b/examples/software_foundations/SfBasic.fst.hints @@ -229,7 +229,7 @@ "subterm_ordering_SfBasic.S", "typing_SfBasic.__proj__S__item___0" ], 0, - "deb7c6532ff56eaf381e73f0f47d9dfe" + "8d0b17e00b9b60dd491bb9ac2d81e7c7" ], [ "SfBasic.test_oddb1", @@ -301,7 +301,7 @@ "fuel_guarded_inversion_SfBasic.nat", "subterm_ordering_SfBasic.S" ], 0, - "01a58ecd4189dbd44baed2990aa51b31" + "b2bb140f5cb44dbafacbbc48c4e19396" ], [ "SfBasic.mult", @@ -315,7 +315,7 @@ "fuel_guarded_inversion_SfBasic.nat", "subterm_ordering_SfBasic.S" ], 0, - "4230a9c7c231e4c945ddd03f9935b0b5" + "52ca2387a34ca7ab81a08a1f6c6dbbbb" ], [ "SfBasic.test_mult1", @@ -364,7 +364,7 @@ "subterm_ordering_SfBasic.S", "typing_tok_SfBasic.O@tok" ], 0, - "7a6777beead01839d544a0118ef97594" + "a39adae0e7c05f793996e83fbfd57c23" ], [ "SfBasic.beq_nat", @@ -381,7 +381,7 @@ "subterm_ordering_SfBasic.S", "typing_tok_SfBasic.O@tok" ], 0, - "5ee0308533fcd6bd40e1a6eae4945af6" + "50ba1a96576455fdb31eaafc029e9596" ], [ "SfBasic.ble_nat", @@ -402,7 +402,7 @@ "subterm_ordering_SfBasic.S", "typing_tok_SfBasic.O@tok" ], 0, - "1604773cfce5e6980d86191fddc05492" + "29150f2cdf5e8c432b92be639d6865e2" ], [ "SfBasic.test_ble_nat1", @@ -874,7 +874,7 @@ "subterm_ordering_SfBasic.S", "typing_SfBasic.__proj__S__item___0" ], 0, - "2465560e9a341daafcaa97fcc0a882b3" + "a5ff3ef464d81c4e37eab69f8bd16953" ], [ "SfBasic.test_oddb1", @@ -906,7 +906,7 @@ "fuel_guarded_inversion_SfBasic.nat", "subterm_ordering_SfBasic.S" ], 0, - "9b3269731fe21ff04a3a18457cfbd0d5" + "8e5e5bc868c82e387e031a4e0213781f" ], [ "SfBasic.mult", @@ -920,7 +920,7 @@ "fuel_guarded_inversion_SfBasic.nat", "subterm_ordering_SfBasic.S" ], 0, - "43d0ec7e34690806020d3c7f19b3a666" + "b83fd4f52b52c613ea6ec704cc17b15c" ], [ "SfBasic.test_mult1", @@ -951,7 +951,7 @@ "typing_tok_SfBasic.O@tok" ], 0, - "a351d0de11f0a3ca0876963fb65472d4" + "bfe608bafa18e8a05501d840e83ca8b7" ], [ "SfBasic.beq_nat", @@ -967,7 +967,7 @@ "subterm_ordering_SfBasic.S", "typing_tok_SfBasic.O@tok" ], 0, - "01cca037cc56cb64420bb36a027f480e" + "84eb1506ab920908a6de91996956322d" ], [ "SfBasic.ble_nat", @@ -989,7 +989,7 @@ "typing_tok_SfBasic.O@tok" ], 0, - "b832c3a3dc24d3b4796528a2bf50dd7d" + "2adc244eeef837b2493125ce39ffe499" ], [ "SfBasic.test_ble_nat1", diff --git a/examples/software_foundations/SfLists.fst.hints b/examples/software_foundations/SfLists.fst.hints index b8cf7bffa7e..d720c939fd6 100644 --- a/examples/software_foundations/SfLists.fst.hints +++ b/examples/software_foundations/SfLists.fst.hints @@ -52,7 +52,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "3bea516fb205be0ba6858aa2c282b785" + "315489c062a67228457ee4673f86f89a" ], [ "SfLists.repeat", @@ -71,7 +71,7 @@ "well-founded-ordering-on-nat" ], 0, - "f075af583d73ce55b8e8bc3171f50fd3" + "fc2b8576e21a777837a25eafadec7083" ], [ "SfLists.app", @@ -86,7 +86,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "6f1349a2856e89329bebeb8818bd9c8b" + "85b399f516b4375b394a0df17b5ed96e" ], [ "SfLists.test_app1", @@ -433,7 +433,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "e1d494c080eaebb56c8073c39bf352ab" + "4ce0251a51cf1114d3cc41d6afdac66f" ], [ "SfLists.rev", @@ -448,7 +448,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "cf7de0b507ddba3bbe66628fe748708f" + "0af6355463d5ec359fc6782b744a6b12" ], [ "SfLists.length_snoc", @@ -590,7 +590,7 @@ "typing_SfLists.length", "well-founded-ordering-on-nat" ], 0, - "29c63f14f3659a2d2cca48156503ecd8" + "77fb5ae746d87e33891a2fbc738aa57b" ], [ "SfLists.foo3", @@ -630,7 +630,7 @@ "subterm_ordering_SfLists.Cons", "typing_tok_SfLists.Nil@tok" ], 0, - "a2b442ff04883ec41a3d226da0a6998b" + "e59b8f3b8538cce68fa12f60a7bbf2f9" ], [ "SfLists.foo4", @@ -834,7 +834,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "05304bdf2ed8dc845cbf6375db3da455" + "8e72753d59d60e081eefaf2cb48ff57e" ], [ "SfLists.app_cons", @@ -962,7 +962,7 @@ "subterm_ordering_SfLists.Cons", "typing_tok_SfLists.Nil@tok" ], 0, - "2c06f508272d3cd53f221a2c7b89750a" + "f23fe939105bc3cd55d12c2f5636f1e3" ], [ "SfLists.forallb", @@ -977,7 +977,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "6f734019eac1d0f25c26930c3e665fad" + "3b46eae71f7d4b3d25263f4955fbb14d" ], [ "SfLists.existsb", @@ -992,7 +992,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "4efa0b541ff022c0202dab4a8727ffeb" + "36e9f6477fa466b9de6e80417b8e2eee" ], [ "SfLists.existsb_existsb'", @@ -1086,7 +1086,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "6cef2008fab48a1a5f61962035e8278f" + "5ceea63746b1acb2206f0a7ac2018bbd" ], [ "SfLists.repeat", @@ -1104,7 +1104,7 @@ "well-founded-ordering-on-nat" ], 0, - "8480ba5a18b62a47e0f7e27b5905aa82" + "f53848b0adc6ead2e7cc13a748b53cca" ], [ "SfLists.app", @@ -1119,7 +1119,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "0f32f2185a11f48289e352baf65f60c6" + "6fe058520cb16f657b1bd0c87e23fc64" ], [ "SfLists.test_app1", @@ -1264,7 +1264,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "5f85b3d665e0b7bd6ed9f6d771884714" + "0eaa8448a0698e71401e04e1665e1ff8" ], [ "SfLists.rev", @@ -1279,7 +1279,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "2757424110a8a868bdd8b2d68f2b5849" + "e261477ca03775522399fb3bb468b3d9" ], [ "SfLists.length_snoc", @@ -1358,7 +1358,7 @@ "typing_SfLists.length", "well-founded-ordering-on-nat" ], 0, - "c0f90043de867f668b0f5894b8ecec8f" + "6761a4f68f2f1c5cdf3c81630e2d0dfa" ], [ "SfLists.foo3", @@ -1386,7 +1386,7 @@ "subterm_ordering_SfLists.Cons", "typing_tok_SfLists.Nil@tok" ], 0, - "6e80d399abb90e1b3299991dd8142a75" + "3c280d6eec1d0f98286cf7e2524daf66" ], [ "SfLists.foo4", @@ -1476,7 +1476,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "85cfec85782b2f252465a809569d06ad" + "e05af28ea432ff784d812bcb0edf7d28" ], [ "SfLists.app_cons", @@ -1527,7 +1527,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "0f268631c181e19a6e6d80982ba596ca" + "01a9b5dcbef2c388b2e51efb72ac97f9" ], [ "SfLists.existsb", @@ -1542,7 +1542,7 @@ "subterm_ordering_SfLists.Cons" ], 0, - "19720633b0af6d14f24ac3ea82a3e998" + "b7d1321707580a9a83a1468c8d69dce1" ], [ "SfLists.existsb_existsb'", diff --git a/examples/software_foundations/SfPoly.fst.hints b/examples/software_foundations/SfPoly.fst.hints index af340b91bac..d4d99ca2dbc 100644 --- a/examples/software_foundations/SfPoly.fst.hints +++ b/examples/software_foundations/SfPoly.fst.hints @@ -16,7 +16,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "2ff2fd753268c4d74f0cddd0f0ad02cf" + "4ca487fc786e6718c99acb5299ff601d" ], [ "SfPoly.test_length1", @@ -146,7 +146,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "9dd9a4e00a35b9d34fcfc7c041cb17ab" + "2c6cfc7a23211d207cd5f7a51d813806" ], [ "SfPoly.nil_app", @@ -238,7 +238,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "ec64ec8a1ca72decc05352fc8f25795c" + "cafe38fbe332fac4393b001389c4f26a" ], [ "SfPoly.snoc_with_append", @@ -277,7 +277,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "e6de4bc28cc48424fe8d448c17525d2f" + "fa0a7204988f78f48980aeeeb1b51062" ], [ "SfPoly.rev_snoc", @@ -342,7 +342,7 @@ "well-founded-ordering-on-nat" ], 0, - "956a822c6e32f01194142d9bba3fe4b5" + "00fca4336de412575181f71882b73e82" ], [ "SfPoly.combine", @@ -364,7 +364,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "96793358b399e85efd1cf61d97f839f4" + "cc986517313d529d3c7c8e4208a325c8" ], [ "SfPoly.index_option", @@ -385,7 +385,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "edc446458de725044ee515e2c363c01d" + "811478db84e17dd817442c33e60c5e28" ], [ "SfPoly.test_index_option1", @@ -505,7 +505,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "aaf44276ea55bd321456b8e60f23f670" + "9bb060fa2a99ef18533e370a2540bf2d" ], [ "SfPoly.test_prod_uncurry", @@ -581,7 +581,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "c776f7dcbd501bde7fd425ed2bd1aed1" + "cad3a11bd483e589491e3fc8957bb41b" ], [ "SfPoly.evenb", @@ -607,7 +607,7 @@ "well-founded-ordering-on-nat" ], 0, - "bf9db0d6a187ce50424e53aebca038b7" + "fddbdf7cbb510fbc2add3e6fa5f39688" ], [ "SfPoly.test_filter1", @@ -701,7 +701,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "eb360e49b20ade9eb63d538cac7c96f2" + "5a3bc7e90505054577c3ea13802ccdc7" ], [ "SfPoly.test_map1", @@ -895,7 +895,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "5a64bbc9bbb5e340ef05087f6f711078" + "847c6299d5c32c563acee61577d1aedc" ], [ "SfPoly.fold_example1", @@ -1340,7 +1340,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "2df1d95149cdd02e4475a8023c8e1188" + "fec95a3c11c80ad4e9ba5aaf74ee0889" ], [ "SfPoly.test_length1", @@ -1390,7 +1390,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "5de00daabfaa123e8db6ca21d82302f6" + "155965649973088d66f795d099bed470" ], [ "SfPoly.length_app", @@ -1413,7 +1413,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "4012b5d3428ef66c7f7d30d5aa9ecf38" + "1f6ff9ed104aad12e123162d3058222b" ], [ "SfPoly.rev", @@ -1427,7 +1427,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "61b975107a980b57e7a32840874c2dae" + "47fc512b59036efb5d029022f9af20e4" ], [ "SfPoly.repeat", @@ -1444,7 +1444,7 @@ "well-founded-ordering-on-nat" ], 0, - "ed11268278d17719fc022928ef1bd78b" + "00d10c2961d133f23889079559ea4efe" ], [ "SfPoly.combine", @@ -1466,7 +1466,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "d16e8bba1b5d04816c8ef5dffe75a757" + "d0555e72259027a6cba82a8187f61576" ], [ "SfPoly.index_option", @@ -1487,7 +1487,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "116720a29ad90696907d2f05ac8e70f1" + "e242b02613564fa621acdba332332cef" ], [ "SfPoly.test_index_option1", @@ -1549,7 +1549,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "87672219165b54162d4c2882da4047e3" + "9338b5e21479f1e1f9375f7b2ca6cb3d" ], [ "SfPoly.filter", @@ -1563,7 +1563,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "dedec6cac0db154f9b16bd23d0bbe695" + "34aacb1abd8286d6c604c2e8f18482d2" ], [ "SfPoly.evenb", @@ -1588,7 +1588,7 @@ "well-founded-ordering-on-nat" ], 0, - "299f41ee49008d4119c6204ecb3a542d" + "1bebcb549a5c79d537d56a28506e5bbe" ], [ "SfPoly.test_filter1", @@ -1630,7 +1630,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "2f6237c1dd66367d5c729de588dd52bd" + "1327d38ffcc8940b3711088aca77d09d" ], [ "SfPoly.test_map1", @@ -1699,7 +1699,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "ccef07c429b53d82db9d4c450d3b66ba" + "508f503d35731534e7754a34d3d13c69" ], [ "SfPoly.fold_example1", diff --git a/examples/tactics/Alt.fst.hints b/examples/tactics/Alt.fst.hints index beadeff4ad1..29ff8b8c8b2 100644 --- a/examples/tactics/Alt.fst.hints +++ b/examples/tactics/Alt.fst.hints @@ -11,7 +11,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "3c48606786ab0cfabda56fc4f7dacaaa" + "988fa2a63b022324009f11429125219d" ], [ "Alt.uu___64", @@ -23,7 +23,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "0672f6f7e56f5b16e0581cca747a8f47" + "14caa441a6c539a07321d6ec36256026" ], [ "Alt.uu___64", @@ -35,7 +35,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "4ced8e6df1460ab5b765ae4086322133" + "8da6351bb528fa4b32248b96fbccca88" ], [ "Alt.uu___64", @@ -47,7 +47,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "e1ec5cc52c4ef4df5cbaa44a4121a4a9" + "543b9b236bdd0d142c15be7650dc4615" ] ] ] \ No newline at end of file diff --git a/examples/tactics/AnnoyingVCs.fst.hints b/examples/tactics/AnnoyingVCs.fst.hints index c30248144d1..2680dd601a4 100644 --- a/examples/tactics/AnnoyingVCs.fst.hints +++ b/examples/tactics/AnnoyingVCs.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "true_interp" ], 0, - "f379a79960d847a46227d2655ba3229e" + "672ab7637b45353e1e6f38f240339cbe" ], [ "AnnoyingVCs.test2", @@ -17,7 +17,7 @@ 1, [ "@query", "true_interp" ], 0, - "42d52e898e283a7ba1f6e7e7a634eb97" + "9f60dcd21b4ca5a256160cb6b22d54c3" ], [ "AnnoyingVCs.test2", @@ -26,7 +26,7 @@ 1, [ "@query", "true_interp" ], 0, - "49cc5d322bd6c06f02b5af26cc5304a9" + "92263ad6f857f79025d078d0f176f235" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Arith.fst.hints b/examples/tactics/Arith.fst.hints index cbd4742b5d4..ed898eb75bc 100644 --- a/examples/tactics/Arith.fst.hints +++ b/examples/tactics/Arith.fst.hints @@ -12,7 +12,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "3d3944f75be03338e480c6365dd41f37" + "8d1d22ba665b4edb0e6cfba4e4fc6771" ], [ "Arith.lem1", @@ -30,7 +30,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "4822235636175f10a27368524c6cf01e" + "082ac98653246413fd32425a9ee63ee0" ], [ "Arith.lem1", @@ -43,7 +43,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "a3710a5c0c95dfc006479172ac050fe1" + "cc4d8bd271dbfcc882fae085a9cbb9c8" ], [ "Arith.lem2", @@ -56,7 +56,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "a9edf51596f12412136f787f2a235739" + "bde278709e446382502bba74d4295544" ], [ "Arith.lem2", @@ -74,7 +74,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "13dc0fe2f2190c0b7753c67932a8a895" + "ad013f6989cbf8a8cd458093d9bfbbb8" ], [ "Arith.lem3", @@ -89,7 +89,7 @@ "projection_inverse_Prims.Cons_tl", "true_interp" ], 0, - "53ffd45b67425d054cf929c266a18f65" + "7cfc713c5c0617496da61ffe3239e816" ], [ "Arith.lem3", @@ -114,7 +114,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "66f2a326ee3f72e62d7beba671b535e2" + "46fcc68be2a7147cb8fa0adeba00fd12" ], [ "Arith.lem3", @@ -129,7 +129,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "fdd72dea884399e244d7cc954163c375" + "848d430e33692f52db994aead69ca481" ], [ "Arith.lem4", @@ -144,7 +144,7 @@ "projection_inverse_Prims.Cons_tl", "true_interp" ], 0, - "f7a0a1fc58bb373d90c169cddbb08e98" + "cd92a301c1c8cee9e9d19b2fd684c368" ], [ "Arith.lem4", @@ -162,7 +162,7 @@ "unit_inversion", "unit_typing" ], 0, - "9c8eebd16a0439942c309ae95c65f11e" + "ce950a3020b3ac2b9d1a491331554ea0" ], [ "Arith.lem4", @@ -173,11 +173,11 @@ "@MaxIFuel_assumption", "@query", "Prims_interpretation_Tm_arrow_f82c3fb9ac6610efb97620a59b378092", "equation_Prims.l_Forall", "equation_Prims.squash", "int_inversion", - "l_quant_interp__7992", + "l_quant_interp__8018", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "f1b6554e064aa3336b14b947e011d8a5" + "7df7dec81dd92171ce92cec0fd404d50" ], [ "Arith.lem4", @@ -202,7 +202,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "d01e37c8feb567fcea14d9a0021255a1" + "e4f269bbf59b553017c9e4f8ca5e65b5" ], [ "Arith.lem4", @@ -211,12 +211,12 @@ 1, [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", - "equation_Prims.squash", "int_typing", "l_quant_interp__8008", + "equation_Prims.squash", "int_typing", "l_quant_interp__8034", "projection_inverse_BoxInt_proj_0", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "d18f8d904d656182cb99f97ae85c1c6e" + "5388f338bd86f47a2adaca5843383a26" ], [ "Arith.lem0", @@ -229,7 +229,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "e3e281c006ddf1fc9281dfffe1caf316" + "ff300d9fb69084c0c5a96f1364edd032" ], [ "Arith.lem1", @@ -247,7 +247,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "1a885fe5ac09742d405557024f224521" + "5183be31c09b8bc62bdc3f1e04877785" ], [ "Arith.lem1", @@ -260,7 +260,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "59feac92a1175c50385aa0d2a904e590" + "04c9bc6c23c71783d4a653f4a8d37367" ], [ "Arith.lem2", @@ -273,7 +273,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "dfe008f9159771071073b77ff902d5cf" + "f570333f124ee02d93a9ea07f535339d" ], [ "Arith.lem2", @@ -291,7 +291,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "af9cf8a7043e382a3ca6ae0b9fec4a53" + "8cb26e4534faf6199fd9b9edac6ed1d5" ], [ "Arith.lem3", @@ -306,7 +306,7 @@ "projection_inverse_Prims.Cons_tl", "true_interp" ], 0, - "e53ae92547ded2875df29486a5e56f2e" + "631c1e7ab1f170219c5324093eb8ac95" ], [ "Arith.lem3", @@ -331,7 +331,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "f9151039ab3acb5e1d1327bd6bf8fef1" + "d20674a52a4d04a62721a45a799a137f" ], [ "Arith.lem3", @@ -346,7 +346,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "5694950685458d7db0b2b662b48f118f" + "8119cf2d465b39aba365f1d4ca0e1f27" ], [ "Arith.lem4", @@ -361,7 +361,7 @@ "projection_inverse_Prims.Cons_tl", "true_interp" ], 0, - "aa8eb56f02c8ccab367cefc9e79a63b9" + "9786082e4d3b08735bdb7d6dd06ad24b" ], [ "Arith.lem4", @@ -379,7 +379,7 @@ "unit_inversion", "unit_typing" ], 0, - "897972275b91236a74416cf716dca52d" + "1b0aaeee12654313f28e9c2d14dfce37" ], [ "Arith.lem4", @@ -390,11 +390,11 @@ "@MaxIFuel_assumption", "@query", "Prims_interpretation_Tm_arrow_f82c3fb9ac6610efb97620a59b378092", "equation_Prims.l_Forall", "equation_Prims.squash", "int_inversion", - "l_quant_interp__8058", + "l_quant_interp__8084", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "b0623b89a6132813cd286b89df9e4a04" + "e3fbdd86d054e3c691633c465a50ca04" ], [ "Arith.lem4", @@ -419,7 +419,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "e155151db3aef0ae475a42ec4d7f27a9" + "49176d97f7fba437cc4c04a0a5974a1c" ], [ "Arith.lem4", @@ -428,12 +428,12 @@ 1, [ "@MaxIFuel_assumption", "@query", "equation_Prims.l_Forall", - "equation_Prims.squash", "int_typing", "l_quant_interp__8074", + "equation_Prims.squash", "int_typing", "l_quant_interp__8100", "projection_inverse_BoxInt_proj_0", "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "ddcbac92f2e03d2d4e15ee800bb40d5e" + "73e224850025fdb400ebd2a8bac26327" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Bane.Lib.fst.hints b/examples/tactics/Bane.Lib.fst.hints index 96d04c63b0f..081ece14f01 100644 --- a/examples/tactics/Bane.Lib.fst.hints +++ b/examples/tactics/Bane.Lib.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "c7b89e03f78a30734186691bb95ef566" + "6f4b431d85e09bd8e4eb30acb140f46a" ], [ "Bane.Lib.repeat_or_fail", @@ -26,7 +26,7 @@ "lemma_FStar.Pervasives.invertOption", "unit_typing" ], 0, - "cffd41ba219194e3baf15cb4a8101eaf" + "a8c607439b0c0c2f59f00c761c951542" ], [ "Bane.Lib.big_phi", @@ -35,7 +35,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "15acc813adea4175eab1566fbf5c7f66" + "9562c0932f75475f94b023a393cae630" ], [ "Bane.Lib.repeat_or_fail", @@ -53,7 +53,7 @@ "lemma_FStar.Pervasives.invertOption", "unit_typing" ], 0, - "2ae3a42a52a28a6048530b5236b72b47" + "6a40dae31566b02f00227ead83ce0f94" ], [ "Bane.Lib.mytac", @@ -70,7 +70,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "53fab848f1d6205828a26b0e271997ed" + "bc5f7640873eaae7a6bb2d48eca0dd40" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Bug1252.fst.hints b/examples/tactics/Bug1252.fst.hints index 87f496cdcb3..e911eb5d1e5 100644 --- a/examples/tactics/Bug1252.fst.hints +++ b/examples/tactics/Bug1252.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "function_token_typing_Bug1252.p1" ], 0, - "0f9368fcef506b5090b9adfa1ed1482b" + "dc82dd5e8c5c98a47f16288dbfc8084e" ], [ "Bug1252.f", @@ -17,7 +17,7 @@ 1, [ "@query", "function_token_typing_Bug1252.p1" ], 0, - "3ef623a0a295a6867dcf00b06be5551d" + "f3a8c5b3e997ea6df73e894d57b2df2d" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Bug1256.fst.hints b/examples/tactics/Bug1256.fst.hints index bc37b523df0..ecec9e7cd5d 100644 --- a/examples/tactics/Bug1256.fst.hints +++ b/examples/tactics/Bug1256.fst.hints @@ -16,7 +16,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "3d42f0d34eb90685ddb2a1a25d6f2e9c" + "26a177166f32a167d118b3fd1123cee3" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Bug1270.fst.hints b/examples/tactics/Bug1270.fst.hints index be66d1974bd..1b69e41aad8 100644 --- a/examples/tactics/Bug1270.fst.hints +++ b/examples/tactics/Bug1270.fst.hints @@ -16,7 +16,7 @@ "typing_FStar.Reflection.Basic.binders_of_env" ], 0, - "d896565e5f49e53b1dde5cb7c9b96c52" + "d6d318d5d0fe33de5cfce80c10dbf1fa" ], [ "Bug1270.test", @@ -33,7 +33,7 @@ "typing_FStar.Reflection.Basic.binders_of_env" ], 0, - "fc5189e20e2c5a8fea76b31c96008dbe" + "3cbb4a75d0183405b5f2e5797a8a4c55" ], [ "Bug1270.test", @@ -50,7 +50,7 @@ "typing_FStar.Reflection.Basic.binders_of_env" ], 0, - "ae0473045c8b9ed84b8257b68108d381" + "fc777f7d6b7536588be8aa1b41715fd0" ], [ "Bug1270.test", @@ -67,7 +67,7 @@ "typing_FStar.Reflection.Basic.binders_of_env" ], 0, - "100943c8cb3657d739fc85e894e5bc70" + "e3c5968a7ddbbe5ba2f99d2c333b4890" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Bug1299.fst.hints b/examples/tactics/Bug1299.fst.hints index 279eabe56ba..dbbdd1ededa 100644 --- a/examples/tactics/Bug1299.fst.hints +++ b/examples/tactics/Bug1299.fst.hints @@ -26,7 +26,7 @@ "unit_typing" ], 0, - "d2d376b62705cbe4db013145a35357a0" + "d25359fcedfd712b36dc8eb3e2f86f33" ], [ "Bug1299.should_fail", @@ -53,7 +53,7 @@ "unit_typing" ], 0, - "851c885a23c1b7feb248e65443b56df6" + "a718f6c646071a22d8cc18c219c9cf2d" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Canon.fst.hints b/examples/tactics/Canon.fst.hints index d96ea17a459..b78fa60567c 100644 --- a/examples/tactics/Canon.fst.hints +++ b/examples/tactics/Canon.fst.hints @@ -11,7 +11,7 @@ "primitive_Prims.op_Multiply", "projection_inverse_BoxInt_proj_0" ], 0, - "37c29756c265dc8747211a74bc49ef99" + "023895de6cb4a5297e2ec71be604457f" ], [ "Canon.lem8", @@ -20,7 +20,7 @@ 1, [ "@query", "true_interp" ], 0, - "ba2d84f35d6e0a9149d23ebc8565bf5a" + "5fb8eee760e254c160a63a70ce94e779" ], [ "Canon.lem9", @@ -29,7 +29,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int", "true_interp" ], 0, - "3b62b6777916b4ba37f6e9372bb7a8c9" + "c5f90abde258538dcfe5776a57de0a84" ], [ "Canon.check_canon", @@ -46,7 +46,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "89e1b963e20c3df60e1be5f6bb3c1d06" + "00f0058dfb110aafe93a41a183964cd8" ], [ "Canon.lem1", @@ -58,7 +58,7 @@ "primitive_Prims.op_Multiply", "projection_inverse_BoxInt_proj_0" ], 0, - "32f33a0c3a3e440c85e4cbb183f22b0c" + "b4a2d4b242b24cb8846fbdaf49984f48" ], [ "Canon.lem8", @@ -67,7 +67,7 @@ 1, [ "@query", "true_interp" ], 0, - "5693c50b5bd8228ae8fa5e7a2c6a03e1" + "1813b3835b2ef6ffd9cbc4c7c0c961f7" ], [ "Canon.lem9", @@ -76,7 +76,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int", "true_interp" ], 0, - "519efc11da8a25d0cd01abad9d2a7229" + "5f384d085da7ce90e6e1a73830f64484" ] ] ] \ No newline at end of file diff --git a/examples/tactics/CanonCommMonoid.fst.hints b/examples/tactics/CanonCommMonoid.fst.hints index 01a364978db..88a3bec1045 100644 --- a/examples/tactics/CanonCommMonoid.fst.hints +++ b/examples/tactics/CanonCommMonoid.fst.hints @@ -11,7 +11,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "18010c4fa7117cec5ed8bb45c8643bad" + "b0e1267b5ca79ba005426ca61e4fcabc" ], [ "CanonCommMonoid.exp", @@ -24,7 +24,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "00777d24200d4d5727d8c816d2b07215" + "183bf6d8f20537a2b4230a2b9ce0f98b" ], [ "CanonCommMonoid.__proj__Var__item___0", @@ -38,7 +38,7 @@ "refinement_interpretation_CanonCommMonoid_Tm_refine_0ce029e55357168c7b2f4890c83d006f" ], 0, - "07adf4dd91d8448be54b7dcf7fb6e588" + "0b04d7f98997fe900b9b4aa0f1e8bef3" ], [ "CanonCommMonoid.__proj__Mult__item___0", @@ -52,7 +52,7 @@ "refinement_interpretation_CanonCommMonoid_Tm_refine_81ce976ce6cdc1820c6b0b8dcaaaa29c" ], 0, - "40dd9d1b17f7d49ec1c80fc9ec3c6406" + "2dbcce548e6f6de61dc6b7543f30fea2" ], [ "CanonCommMonoid.__proj__Mult__item___1", @@ -66,7 +66,7 @@ "refinement_interpretation_CanonCommMonoid_Tm_refine_81ce976ce6cdc1820c6b0b8dcaaaa29c" ], 0, - "9123fd0f392bcc0e2b5ff4183ef2690c" + "a6bfabb3b67efce45077fa3cb0309a08" ], [ "CanonCommMonoid.exp_to_string", @@ -83,7 +83,7 @@ "subterm_ordering_CanonCommMonoid.Mult" ], 0, - "b7af6c93ebd47ecec33ce9c16afae04d" + "72f03cd147713ecf5e93a68266c0e58e" ], [ "CanonCommMonoid.mdenote", @@ -105,7 +105,7 @@ "subterm_ordering_CanonCommMonoid.Mult" ], 0, - "a478d722e8ce49550ade1b3a7de3a4fd" + "44de2487148385d67450495d11fec468" ], [ "CanonCommMonoid.xsdenote", @@ -126,7 +126,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "54564f3a4900a43283bbaf3c760152cc" + "bf14d6465e6ae63004898067d71b0514" ], [ "CanonCommMonoid.flatten", @@ -143,7 +143,7 @@ "subterm_ordering_CanonCommMonoid.Mult" ], 0, - "180ebe0dea9fa19553f1624de399de0f" + "b2fd32e7466d1d124511ae190d3823d1" ], [ "CanonCommMonoid.flatten_correct_aux", @@ -182,7 +182,7 @@ "unit_typing" ], 0, - "b90ed038a91ae604a071169c610f12e8" + "07ce8e539bad3d81d20df71d28a5034e" ], [ "CanonCommMonoid.flatten_correct", @@ -225,7 +225,7 @@ "subterm_ordering_CanonCommMonoid.Mult" ], 0, - "0694b0fa40f27b9400c705441344f376" + "22254b496347bc75f28cf246fe94cad5" ], [ "CanonCommMonoid.apply_swap_aux_correct", @@ -280,7 +280,7 @@ "unit_typing" ], 0, - "a7d5705cf7841e7b6ecfa97f84026c91" + "294fea53bfe3aa37f15fa998045a67f0" ], [ "CanonCommMonoid.apply_swap_aux_correct", @@ -335,7 +335,7 @@ "unit_typing" ], 0, - "98273efdd79f78e61c7fc3da9d4be86a" + "b043d7a3569d92fedaa6d85f31a5fe28" ], [ "CanonCommMonoid.apply_swap_correct", @@ -362,7 +362,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "af19f0f28c202567bf3837a2f9d6aae4" + "aebdb91fa098d199b2f8939fb084365f" ], [ "CanonCommMonoid.apply_swaps_correct", @@ -391,7 +391,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.length" ], 0, - "0a53952e17e285b0ee057aabee1e7d11" + "c0b1ee334c6aa1b5adf5b32b33ea8159" ], [ "CanonCommMonoid.permute_via_swaps_correct_aux", @@ -404,7 +404,7 @@ "refinement_interpretation_CanonCommMonoid_Tm_refine_ef576a15b66f69e4ba5235543526c6d8" ], 0, - "4f5a7668527a91b29e00ef9e4509fc1b" + "80cb7b7fed4c0df2db6ce40e864f22c8" ], [ "CanonCommMonoid.sort", @@ -413,7 +413,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "b62438ebdc3c29cb078aeb8fb49bc050" + "fe67fbc09ef4db27a815ab6582c5851e" ], [ "CanonCommMonoid.sort_via_swaps", @@ -436,7 +436,7 @@ "unit_typing" ], 0, - "bb970490229abaca0ddb37443111f2e0" + "5e66e492f0b2d81c0549340080cb77f0" ], [ "CanonCommMonoid.sortWith_via_swaps", @@ -459,7 +459,7 @@ "token_correspondence_FStar.List.Tot.Base.sortWith" ], 0, - "03a5b98c462ca5583072182f99e630cc" + "68f63b639d758b778feb2954c0ed0466" ], [ "CanonCommMonoid.canon_correct", @@ -468,7 +468,7 @@ 1, [ "@query", "equation_CanonCommMonoid.canon" ], 0, - "179ae82d0c9a0fc72d3de60bad766763" + "1f794daccff48d8e094bd9b760ef0193" ], [ "CanonCommMonoid.monoid_reflect", @@ -481,7 +481,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "7d07293d5a9a956123d4b26c6468dfd8" + "b389497b5ce386ac6210a514e749de51" ], [ "CanonCommMonoid.where_aux", @@ -500,7 +500,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "9d35414b3734c9db3518cd17128223ad" + "b7370642053d1ce2bf46efef753e3c0d" ], [ "CanonCommMonoid.reification_aux", @@ -532,7 +532,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "ea6eb02aaa03f9c5a029a06b49890ba9" + "3a2ecb0a12cc0d77049bcce0e078a8f5" ], [ "CanonCommMonoid.term_mem", @@ -547,7 +547,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "51eea268164be7618acf3af3da3caef5" + "5e659549f70aca7bd71577b33d0e66b7" ], [ "CanonCommMonoid.quote_list", @@ -559,7 +559,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "b2185218581f42b65d20cfa7595dda13" + "9b6e3c8efdfa0e0b90f31b63b7af484f" ], [ "CanonCommMonoid.quote_exp", @@ -574,7 +574,7 @@ "fuel_guarded_inversion_CanonCommMonoid.exp" ], 0, - "01151b56927ef413651d304d3906f54c" + "456252b3fdfcf293d1d5e495ad979027" ], [ "CanonCommMonoid.const_compare", @@ -597,7 +597,7 @@ "typing_CanonCommMonoid.select_extra" ], 0, - "e44ffc25c0dac0ec8036defee9a1e8c5" + "17796affa1e747d02534e74bcc03347c" ], [ "CanonCommMonoid.lem1", @@ -615,7 +615,7 @@ "token_correspondence_CanonCommMonoid.sortWith", "true_interp" ], 0, - "fff3f96fb175e10fc4ad9eae5091c151" + "9ace7b7736a1781b1e049f22c51d1a0c" ], [ "CanonCommMonoid.lem1", @@ -633,7 +633,7 @@ "token_correspondence_CanonCommMonoid.sortWith", "true_interp" ], 0, - "73c6a728c98ad1feff7bfbcb510e34b8" + "a4754ea3ed27dbc39c7919e76ea02655" ], [ "CanonCommMonoid.lem1", @@ -651,7 +651,7 @@ "token_correspondence_CanonCommMonoid.sortWith" ], 0, - "48d376f6f1e5d1296eccc9c90787cdec" + "0974b81fe38951ba66d15e8922a291ca" ], [ "CanonCommMonoid.special_compare", @@ -674,7 +674,7 @@ "typing_CanonCommMonoid.select_extra" ], 0, - "3cb6df1b42209a051a2c193b9ab67701" + "985e42306ef5dfa97a36c1cc88093912" ], [ "CanonCommMonoid.special_first_correct", @@ -692,7 +692,7 @@ "token_correspondence_CanonCommMonoid.sortWith" ], 0, - "6f88a20490a6c15f2775cffa82782162" + "7656c6c25dce6a9c1b0e59e6c0933860" ], [ "CanonCommMonoid.dump", @@ -709,7 +709,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "f9e8932ce2ec94ec63838e7303f68bdd" + "80aab4e234ba3b8e63358ad6ca25d320" ], [ "CanonCommMonoid.var", @@ -721,7 +721,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "19108cc98b136d4cf7c45dd40686367e" + "b070a66cd0d5fe93e5cee1673f572a14" ], [ "CanonCommMonoid.exp", @@ -734,7 +734,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "ca3e4f6173f6fbbd884f913ded9f19e0" + "f51d678f73cbdd62f0c084c8ff6aa654" ], [ "CanonCommMonoid.__proj__Var__item___0", @@ -748,7 +748,7 @@ "refinement_interpretation_CanonCommMonoid_Tm_refine_0ce029e55357168c7b2f4890c83d006f" ], 0, - "025dee8b8c491e062f3892297bbc9d89" + "f2d5671c4576787f1bfc4170135e00b7" ], [ "CanonCommMonoid.__proj__Mult__item___0", @@ -762,7 +762,7 @@ "refinement_interpretation_CanonCommMonoid_Tm_refine_81ce976ce6cdc1820c6b0b8dcaaaa29c" ], 0, - "e4350c7ff6207a5e5c233d88e93694b8" + "b24c4f667e43ff6de490ddd38e44b4b3" ], [ "CanonCommMonoid.__proj__Mult__item___1", @@ -776,7 +776,7 @@ "refinement_interpretation_CanonCommMonoid_Tm_refine_81ce976ce6cdc1820c6b0b8dcaaaa29c" ], 0, - "deba6f0d96c7fcbb25277e2732050380" + "1368ad023a69ebd31d54ee4f24e53f71" ], [ "CanonCommMonoid.exp_to_string", @@ -793,7 +793,7 @@ "subterm_ordering_CanonCommMonoid.Mult" ], 0, - "6d73be5b244faabdd4b3c8b2bcacb81a" + "1eefe41ad37d44fdf35964af16417071" ], [ "CanonCommMonoid.mdenote", @@ -815,7 +815,7 @@ "subterm_ordering_CanonCommMonoid.Mult" ], 0, - "ce381194754012afbbb86af942c6898a" + "ef0cdd09feecb7da5ac41f8a418337b2" ], [ "CanonCommMonoid.xsdenote", @@ -836,7 +836,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "c679c1b76e3b4629789966a8a5f3b9e2" + "c39dd345a1449e92e8db8354f81836c1" ], [ "CanonCommMonoid.flatten", @@ -853,7 +853,7 @@ "subterm_ordering_CanonCommMonoid.Mult" ], 0, - "fcc9cbca668e8b5f93430d71192245db" + "8264c8a67e94026ace6585c597bc50bb" ], [ "CanonCommMonoid.apply_swap_aux_correct", @@ -870,7 +870,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "6f587b11a0aa7dc5490cce0cc266d545" + "c4588ed64dcd793dd86cb0127e1f197f" ], [ "CanonCommMonoid.apply_swap_correct", @@ -887,7 +887,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "113db37bf37307df7085eb3acd4aab21" + "abececb16dddff2d4feaee7af0bfaa9b" ], [ "CanonCommMonoid.sort", @@ -896,7 +896,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "ecb9dccb1cfe7768ddf78e46eeef1ecf" + "f3aa0fbe282f47d14c4b1326b7fcfac8" ], [ "CanonCommMonoid.monoid_reflect", @@ -909,7 +909,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "bcf8544f4b06152198b1f4d6fbca497b" + "0c7fd381b2578a0b9a5de9e6e12cd73b" ], [ "CanonCommMonoid.where_aux", @@ -928,7 +928,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "ddb08f1a7d97259c0dbbb97b398b9fb4" + "8fed499695410281f78e8f328289083c" ], [ "CanonCommMonoid.reification_aux", @@ -960,7 +960,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "1f1b2b114d450bc76b5fcd8109796079" + "df5697770a2bec4efcef3ea2caea2f40" ], [ "CanonCommMonoid.term_mem", @@ -975,7 +975,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "e9676f5de6aac4e7773d6e046b4a8894" + "700a812ff7c6bab0021106775caf0916" ], [ "CanonCommMonoid.quote_list", @@ -987,7 +987,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "52bc33d3fbc23a914beefa565c31553a" + "fcc6e8f8245d16f4ab6f571a8f616894" ], [ "CanonCommMonoid.quote_exp", @@ -1002,7 +1002,7 @@ "fuel_guarded_inversion_CanonCommMonoid.exp" ], 0, - "13cd0c4526623399d66c98569b2dfb88" + "62da946dbc643cca7da92114c74907b6" ], [ "CanonCommMonoid.const_compare", @@ -1025,7 +1025,7 @@ "typing_CanonCommMonoid.select_extra" ], 0, - "720379352270d1c3f3e338d4056e364f" + "fc71357f7d2aeeeb0b98f4dc6fef35c5" ], [ "CanonCommMonoid.lem1", @@ -1043,7 +1043,7 @@ "token_correspondence_CanonCommMonoid.sortWith" ], 0, - "3e6db4cbd8e700f20e0acf4a8519d732" + "7b8e2fd0efea92aab18a94abbe115266" ], [ "CanonCommMonoid.lem1", @@ -1061,7 +1061,7 @@ "token_correspondence_CanonCommMonoid.sortWith", "true_interp" ], 0, - "eca83875c6533ff6c8946ce02dae9463" + "b98bb401ab189c421b95c5497053e1d0" ], [ "CanonCommMonoid.lem1", @@ -1079,7 +1079,7 @@ "token_correspondence_CanonCommMonoid.sortWith" ], 0, - "c8bd2d6f620bc1a9e382063f5c39d6cb" + "aa8a16e59b1ab3b3e983261b2ac49b1e" ], [ "CanonCommMonoid.special_compare", @@ -1102,7 +1102,7 @@ "typing_CanonCommMonoid.select_extra" ], 0, - "c2b24115a5fd379589ee39650265012c" + "8fcc3988d8afd8bb61d77970aef3a49d" ] ] ] \ No newline at end of file diff --git a/examples/tactics/CanonCommMonoidSimple.fst.hints b/examples/tactics/CanonCommMonoidSimple.fst.hints index db1c5ec7aa8..b93f0063733 100644 --- a/examples/tactics/CanonCommMonoidSimple.fst.hints +++ b/examples/tactics/CanonCommMonoidSimple.fst.hints @@ -11,7 +11,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "24a7e82a357b096f4d2844a32e18bcf7" + "913baa47e15d0c0d8d6501dc2121ea89" ], [ "CanonCommMonoidSimple.exp", @@ -24,7 +24,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "bcceeba840af07f825f79ad4213c02c3" + "24bbbe6d70ccd4764f5a80e236a23ebf" ], [ "CanonCommMonoidSimple.__proj__Mult__item___0", @@ -38,7 +38,7 @@ "refinement_interpretation_CanonCommMonoidSimple_Tm_refine_d0cb6fb0a7f85b663ad72d6b65621a44" ], 0, - "d0f5664cd1ba4cdb588968bf2178820c" + "846bd2a23156151f47f78abfdf04ced8" ], [ "CanonCommMonoidSimple.__proj__Mult__item___1", @@ -52,7 +52,7 @@ "refinement_interpretation_CanonCommMonoidSimple_Tm_refine_d0cb6fb0a7f85b663ad72d6b65621a44" ], 0, - "fcda00ed40109061545e800180778493" + "010279fe65f0eb5da6b3121be60d5925" ], [ "CanonCommMonoidSimple.__proj__Atom__item___0", @@ -66,7 +66,7 @@ "refinement_interpretation_CanonCommMonoidSimple_Tm_refine_2ec30caafbd2bbfa6d777747c6ae9795" ], 0, - "03e38eb35215825c9d4563b521c2fbb9" + "72fe18bad44ede8f058260356b8d8531" ], [ "CanonCommMonoidSimple.exp_to_string", @@ -86,7 +86,7 @@ "typing_tok_CanonCommMonoidSimple.Unit@tok" ], 0, - "8708c0340707ad2e4b79f2bc0d279b6b" + "f92d3cb55f23606a0271564d1970372f" ], [ "CanonCommMonoidSimple.mdenote", @@ -112,7 +112,7 @@ "typing_tok_CanonCommMonoidSimple.Unit@tok" ], 0, - "8711fcab114cf888f61f6fbe4b3f3fbc" + "eed0dcde40971449f20f567f617dd477" ], [ "CanonCommMonoidSimple.xsdenote", @@ -134,7 +134,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "5799ea7ec6831843d29ca2074bc577ea" + "7111dd2f2773c40ef8b70702f79d9e51" ], [ "CanonCommMonoidSimple.flatten", @@ -154,7 +154,7 @@ "typing_tok_CanonCommMonoidSimple.Unit@tok" ], 0, - "3cf486d04f388d69ff41ea576d67841d" + "e9cc54e30d48c8c93baf0b2a0f5c3333" ], [ "CanonCommMonoidSimple.flatten_correct_aux", @@ -193,7 +193,7 @@ "unit_typing" ], 0, - "a85687021c1902ce4ba299f78f958b14" + "3d328151372c9d5270f055421735f945" ], [ "CanonCommMonoidSimple.flatten_correct", @@ -243,7 +243,7 @@ "typing_tok_CanonCommMonoidSimple.Unit@tok" ], 0, - "27b7cfdb1388aabd0cde28ec9b71c897" + "9906ba1b0558d085a64aceb22b1de11a" ], [ "CanonCommMonoidSimple.apply_swap_aux", @@ -281,7 +281,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "03b036f5cd9ac4b634a3aa0993dd5a50" + "83d627f7f224f4ac8f3eb019c24e7779" ], [ "CanonCommMonoidSimple.apply_swap_aux", @@ -318,7 +318,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "fe21a54c10c0a3a8554c7ba8c9eab52e" + "e9b59dccea1796991f3c1b2697b5b4d6" ], [ "CanonCommMonoidSimple.apply_swap_aux_correct", @@ -373,7 +373,7 @@ "unit_typing" ], 0, - "e46443ca4debe133e51677b488d19fdf" + "d5029a08bfbfdf6b14d8137357d963a1" ], [ "CanonCommMonoidSimple.apply_swap_aux_correct", @@ -428,7 +428,7 @@ "unit_typing" ], 0, - "7e6dc3466e98bde9e5c12e9dc916b8fe" + "cec3c9b30fc4d84388e57ce5a8111da6" ], [ "CanonCommMonoidSimple.apply_swap_correct", @@ -456,7 +456,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "1dc19d2ca5e199884252f90071d3be6e" + "a5379b7e47f28ca411b76f64e93bb840" ], [ "CanonCommMonoidSimple.apply_swaps", @@ -480,7 +480,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.length" ], 0, - "8c787a0bd636ae039bd708c25548c777" + "a10bcdfd68cc78f606c593a5f8f96074" ], [ "CanonCommMonoidSimple.apply_swaps_correct", @@ -511,7 +511,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.length" ], 0, - "7e2b08d5a1638613ae57e778e6fce557" + "0e97d36f1b19eafa6f4b025d6df29636" ], [ "CanonCommMonoidSimple.permute_via_swaps_correct_aux", @@ -524,7 +524,7 @@ "refinement_interpretation_CanonCommMonoidSimple_Tm_refine_b71f46c8bbd6ccd8641f89fd35bf370f" ], 0, - "f7cc0bb13c97687bfdbe7aef35a558e0" + "e665dd8a18467cbf182c9f0deea418ff" ], [ "CanonCommMonoidSimple.sort", @@ -533,7 +533,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "a3882d10ac106b180ebebbeca0b21f69" + "d7d34961a65c075bff5dbdb9dd697db5" ], [ "CanonCommMonoidSimple.sort_via_swaps", @@ -553,7 +553,7 @@ "token_correspondence_FStar.List.Tot.Base.sortWith", "true_interp" ], 0, - "c85bf10e080c35d9f6c4bd4159ecad3d" + "e59f07e1c516f6eeae3ddca0ba7a38c1" ], [ "CanonCommMonoidSimple.canon_correct", @@ -562,7 +562,7 @@ 1, [ "@query", "equation_CanonCommMonoidSimple.canon" ], 0, - "e148df0c0c6de151f8007d39d9c4faae" + "6cbf8b9712b46b627a32d90beff09209" ], [ "CanonCommMonoidSimple.monoid_reflect_orig", @@ -571,7 +571,7 @@ 1, [ "@query" ], 0, - "a9a25f03fcbd886009028121420324ec" + "783fac07811abadc41765251c36d4691" ], [ "CanonCommMonoidSimple.monoid_reflect", @@ -584,7 +584,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "2095e90d99b97e994800059ce3607287" + "0bdeb58f7da9799da67003783f016edf" ], [ "CanonCommMonoidSimple.where_aux", @@ -603,7 +603,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "bcca96efd5f2a32099212beed9afdd27" + "9005dbb0ff86211856d8d9c796869ca9" ], [ "CanonCommMonoidSimple.reification_aux", @@ -623,7 +623,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "6afebe66ba020959d29b72ef8cf5af60" + "c35e8c699154a35b51daeaee0d87386f" ], [ "CanonCommMonoidSimple.dump", @@ -640,7 +640,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "2f9c66a15e16f75bff614532b423cf01" + "07b89cf1d96315ce84114346fae36029" ], [ "CanonCommMonoidSimple.atom", @@ -652,7 +652,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "6348c47e78cbd7196e325d97eef969e7" + "6774dc9925f5c7d8d40ab7b63cdf9390" ], [ "CanonCommMonoidSimple.exp", @@ -665,7 +665,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "8d68719bdd6a142e50ad5b319907cfe4" + "48a81072f673f3d1d5b013fa4225e305" ], [ "CanonCommMonoidSimple.__proj__Mult__item___0", @@ -679,7 +679,7 @@ "refinement_interpretation_CanonCommMonoidSimple_Tm_refine_d0cb6fb0a7f85b663ad72d6b65621a44" ], 0, - "6f0f3dd2bb09f4c16abc85894526bbcd" + "06787ffaa5c0ade83cb293153a461965" ], [ "CanonCommMonoidSimple.__proj__Mult__item___1", @@ -693,7 +693,7 @@ "refinement_interpretation_CanonCommMonoidSimple_Tm_refine_d0cb6fb0a7f85b663ad72d6b65621a44" ], 0, - "8cc3880c18aff56d6f52d8d7e6919061" + "0e79f27df43c67316ab5efc92cff5b16" ], [ "CanonCommMonoidSimple.__proj__Atom__item___0", @@ -707,7 +707,7 @@ "refinement_interpretation_CanonCommMonoidSimple_Tm_refine_2ec30caafbd2bbfa6d777747c6ae9795" ], 0, - "0d10bb4980ac4db3e24070612e57f01d" + "e820eeae966d990560ada5d5052276ae" ], [ "CanonCommMonoidSimple.exp_to_string", @@ -727,7 +727,7 @@ "typing_tok_CanonCommMonoidSimple.Unit@tok" ], 0, - "5724b45041e043356ea87bf1adbea081" + "3e041ab9453e6f4e57e976ffba72d6df" ], [ "CanonCommMonoidSimple.mdenote", @@ -753,7 +753,7 @@ "typing_tok_CanonCommMonoidSimple.Unit@tok" ], 0, - "cb2051cfd352b9f3121e66a5a40c9033" + "006a4d3180e7d41eb4fdd27d863b8a7f" ], [ "CanonCommMonoidSimple.xsdenote", @@ -775,7 +775,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "c5512ead8063a237528eff194b1b9da0" + "7bc6355b0d88f05e349d84af53397842" ], [ "CanonCommMonoidSimple.flatten", @@ -795,7 +795,7 @@ "typing_tok_CanonCommMonoidSimple.Unit@tok" ], 0, - "d183301ad205b99111487200eada90d5" + "45a86ed46c178bc634252f03187dc326" ], [ "CanonCommMonoidSimple.apply_swap_aux", @@ -811,7 +811,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "6a4d8cb5080fa61a9972b076bab0e592" + "1fe62adb47454541ae961e222685fe40" ], [ "CanonCommMonoidSimple.apply_swap_aux", @@ -848,7 +848,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "cc7ce52cc6ff92983369b04349749ffa" + "2fb2d1e7df1d2ee3909ba4a1a4e60c87" ], [ "CanonCommMonoidSimple.apply_swap_aux_correct", @@ -865,7 +865,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "739ee9395539f276fa97046192f286a8" + "dbd860cc8ce95e955460286bb9842e1f" ], [ "CanonCommMonoidSimple.apply_swap_correct", @@ -883,7 +883,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "a0ea02e7b1cc6c140121fb058a9eced9" + "4427156899777e071d198f2e0b87a558" ], [ "CanonCommMonoidSimple.apply_swaps", @@ -914,7 +914,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "a6799455f8640bceb530611f719619fb" + "8235765fe46a672c285314e6e6943677" ], [ "CanonCommMonoidSimple.sort", @@ -923,7 +923,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "28649cba8ece8011ba19a6d8ec387902" + "7b63222452113914ae03eb4842eed19f" ], [ "CanonCommMonoidSimple.monoid_reflect", @@ -936,7 +936,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "ef3a7e1cffd3b48d9be2d5f0b36c30a4" + "26ff4e51bb17bb9ec071e381bfb3a0d3" ], [ "CanonCommMonoidSimple.where_aux", @@ -955,7 +955,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "c41e0e4f288c42dd5fc22cd1d984b2d6" + "42e8e9527daf2b0bc8c837ea0661a4a6" ], [ "CanonCommMonoidSimple.reification_aux", @@ -975,7 +975,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "128caf87518336bc07169164d7b1cbad" + "c8158bb3f99b798b4676a2964d1b3a89" ] ] ] \ No newline at end of file diff --git a/examples/tactics/CanonCommSemiring.fst.hints b/examples/tactics/CanonCommSemiring.fst.hints index 54a2351ad75..d5f54d57b6d 100755 --- a/examples/tactics/CanonCommSemiring.fst.hints +++ b/examples/tactics/CanonCommSemiring.fst.hints @@ -13,7 +13,7 @@ "projection_inverse_CanonCommSemiring.CR_cm_mult" ], 0, - "4d80fe8003778bef14c5cbdf376e233e" + "c7a9a437557a774631a47500b465c990" ], [ "CanonCommSemiring.distribute_right", @@ -22,7 +22,7 @@ 1, [ "@query" ], 0, - "ab6c8a6cc6421042fd0692b6d5b6a9fb" + "bf29c7a825d26ea9b7bf98baf603543c" ], [ "CanonCommSemiring.int_cr", @@ -47,7 +47,7 @@ "token_correspondence_Prims.op_Multiply" ], 0, - "12cd749887c7e126e22366d511835a52" + "df4c376774e74e9e3dbbf8e7c8631b47" ], [ "CanonCommSemiring.exp", @@ -60,7 +60,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "d2b150d254f4c6a0d58ebb454cde490f" + "31f91d8e8ac846ab763b168f60b88879" ], [ "CanonCommSemiring.__proj__Var__item___0", @@ -74,7 +74,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_8b689800a5c7de58fa5eb3a86d8f2b39" ], 0, - "a3def09ec0099b80f26ad80712d4cccb" + "b9db7c7da227a87a17348102e463dfa4" ], [ "CanonCommSemiring.__proj__Add__item___0", @@ -88,7 +88,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_f7b11b9e2e3b3ea1b294881eaa75b765" ], 0, - "f14717e65170bec12174c5446865d3c4" + "d30527995bf021ebbd548224a3e6c1fd" ], [ "CanonCommSemiring.__proj__Add__item___1", @@ -102,7 +102,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_f7b11b9e2e3b3ea1b294881eaa75b765" ], 0, - "40cc98eb85c44b1179d730bb6a20bee8" + "8f430347d9821224309cb7743f6388d2" ], [ "CanonCommSemiring.__proj__Mult__item___0", @@ -116,7 +116,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_7ebec51792cf922a19b62c9c71962f29" ], 0, - "98e47d5b8bc8f71dd301b281945e1b72" + "050c8afe344c9432caa4011a19294817" ], [ "CanonCommSemiring.__proj__Mult__item___1", @@ -130,7 +130,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_7ebec51792cf922a19b62c9c71962f29" ], 0, - "8e687ac4c99432e239ed3595da8cb53b" + "719193f4edc5834065ad79dc88a9df5b" ], [ "CanonCommSemiring.exp_to_string", @@ -148,7 +148,7 @@ "subterm_ordering_CanonCommSemiring.Mult" ], 0, - "366bcfcb1967f0e00572e4bd3d3a7be9" + "c0fbf18c0755f212ac166236a1f42388" ], [ "CanonCommSemiring.quote_exp", @@ -163,7 +163,7 @@ "fuel_guarded_inversion_CanonCommSemiring.exp" ], 0, - "847a9a6e3925135284ae325d57428c4d" + "8c98473c841d0bed885cbb4e8f098517" ], [ "CanonCommSemiring.rdenote", @@ -186,7 +186,7 @@ "subterm_ordering_CanonCommSemiring.Mult" ], 0, - "69391bf87a77ea867ca81e9768536872" + "5adcadd981fd3924fc0ced2fdcd34f2d" ], [ "CanonCommSemiring.sum_of_products", @@ -195,7 +195,7 @@ 1, [ "@query", "assumption_CanonCommMonoid.exp__uu___haseq" ], 0, - "3794a03e1805bb80b107c972e09570af" + "65d17ffaf912bce03034106667eec5ce" ], [ "CanonCommSemiring.__proj__Product__item___0", @@ -209,7 +209,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_c9c5705ff62947a3a85bf808488463d7" ], 0, - "9910168fe6fbf30ecb76ccd88b052d5d" + "d2d62a4e6180b308a242944279b52364" ], [ "CanonCommSemiring.__proj__Sum__item___0", @@ -223,7 +223,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_c4b343140a7f62b6023c700d9c444ae3" ], 0, - "1642c0299f2d8a957e7107834c93d660" + "e0f9ad7eae192cee3c9b82c646be2a9d" ], [ "CanonCommSemiring.__proj__Sum__item___1", @@ -237,7 +237,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_c4b343140a7f62b6023c700d9c444ae3" ], 0, - "11dc12e7bc5177994faedc97a32e79dd" + "578003db9dac7d6c13f9d87cecb2f918" ], [ "CanonCommSemiring.sum_denote", @@ -258,7 +258,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "4d1bf33159bae7020b952068da29d0eb" + "90dafb3bed7d6e43b322ce041697b72f" ], [ "CanonCommSemiring.multiply_sums", @@ -283,7 +283,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "85a8e0fe0bec75b0a3ec9b457c74eb11" + "5d99fc60258f898c5fef91d347c72e12" ], [ "CanonCommSemiring.exp_to_sum", @@ -301,7 +301,7 @@ "subterm_ordering_CanonCommSemiring.Mult" ], 0, - "c7663a6d6d619391aaabfa55d9dc0be8" + "0849b95c64022ee7a17ba1774cf1173f" ], [ "CanonCommSemiring.multiply_sums_correct", @@ -349,7 +349,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "829cc60c8e453b48cecc5214e8df2db9" + "d769faf73fa55ddc722d494e99d10f87" ], [ "CanonCommSemiring.exp_to_sum_correct", @@ -399,7 +399,7 @@ "subterm_ordering_CanonCommSemiring.Mult" ], 0, - "b6cb336ad0c49b29b8bee5cdaa5f1c0c" + "9dc914c5b61f079138d4cfa295f5336a" ], [ "CanonCommSemiring.cdenote", @@ -420,7 +420,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "b64cda94b0220cebdf3d173049b0d6c7" + "e903f6e4e746f992c0640155608ebdc3" ], [ "CanonCommSemiring.cdenote_correct", @@ -453,7 +453,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "dc19169b1722f95beb908b72458aaf00" + "b88c330aa36b7ed1a3bee90dad574567" ], [ "CanonCommSemiring.canon_correct", @@ -462,7 +462,7 @@ 1, [ "@query" ], 0, - "ba0c7f6c15f814d7752aeadfc0da480f" + "4d7b405cf31bddeb27e6a023fe17574c" ], [ "CanonCommSemiring.semiring_reflect", @@ -475,7 +475,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "02c9c8605b7bcdbd323ee998d31afe99" + "e5210904c3c3608ddb9362359d8e61a4" ], [ "CanonCommSemiring.make_fvar", @@ -497,7 +497,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "ab59800c2251f5e7789a662f2e679c72" + "86105b55e420eb63a8235fd45fa5c2f1" ], [ "CanonCommSemiring.is_not_const", @@ -514,7 +514,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "function_token_typing_FStar.Reflection.Types.name", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -522,7 +522,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "31bd470f83cbfea07336d1377413770e" + "b01b27e678275365d8f6a256ba68a8fc" ], [ "CanonCommSemiring.const_last_correct", @@ -540,7 +540,7 @@ "token_correspondence_CanonCommMonoid.sortWith" ], 0, - "108d221a172cace9b26fcfff8196280c" + "a86ff5c140917bbd19a63099811a266e" ], [ "CanonCommSemiring.lem0", @@ -553,7 +553,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "52ed1cdd81aa81c5d886155e16c76dbc" + "cf00154ae09429965df29ea46dd33d1a" ], [ "CanonCommSemiring.lemma_poly_multiply", @@ -568,7 +568,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "6464fb6200403b73bce911a5cf8ba531" + "57abf4c73f583ffbe8df028b5046b341" ], [ "CanonCommSemiring.modulo_addition_lemma", @@ -577,7 +577,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "485a1a5b2235ebaf221bc196bf84f2b8" + "a4c01a0b82bafc5080fa6d2a106e1005" ], [ "CanonCommSemiring.lemma_div_mod", @@ -589,7 +589,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "8f6a22394cc90b42e8e3a5617b6e8213" + "d10c0f6fb3774dcda614a07120780bfd" ], [ "CanonCommSemiring.lemma_poly_multiply", @@ -603,7 +603,7 @@ "projection_inverse_BoxInt_proj_0", "true_interp" ], 0, - "425aabf7c15e8356534532df400f6f23" + "7a4721f32cb7fc06e2889e2e0e0580fd" ], [ "CanonCommSemiring.lemma_poly_multiply", @@ -616,7 +616,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "df3c58cd9fe87e2a3eb76e7b51de2157" + "722d073dba337be0a5592453036ca196" ], [ "CanonCommSemiring.lemma_poly_reduce", @@ -635,7 +635,7 @@ "unit_typing" ], 0, - "c814a79e7714b2b5401d832209c4e155" + "ab745bf7a63bac6c39e41e5d31620488" ], [ "CanonCommSemiring.lemma_poly_reduce", @@ -649,7 +649,7 @@ "projection_inverse_BoxInt_proj_0", "true_interp" ], 0, - "2ff265aa956e36d8007b4fe1989d7225" + "812fff97e5dd6068ba3ab8108b347b09" ], [ "CanonCommSemiring.lemma_poly_reduce", @@ -662,7 +662,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "ad091cc25564b5bc96ca3faece2cae05" + "625f8acb6d168a8bc23afcadb5176a53" ], [ "CanonCommSemiring.ddump", @@ -679,7 +679,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "71563fb41ba92976e0ad8ea9f2ca9066" + "cfe1a0b1d04832cdaacf02f3ec28aca1" ], [ "CanonCommSemiring.__proj__CR__item__distribute", @@ -693,7 +693,7 @@ "projection_inverse_CanonCommSemiring.CR_cm_mult" ], 0, - "3a4734c3c8f3b907a953acc2c2ef4bd9" + "ed1b63268bc4342ad850eff739322750" ], [ "CanonCommSemiring.distribute_right", @@ -702,7 +702,7 @@ 1, [ "@query" ], 0, - "e513a768d1c064a0f0147fa4d7d36c8c" + "3d4eef7c3fc35eaf4bb884966aebe04e" ], [ "CanonCommSemiring.int_cr", @@ -727,7 +727,7 @@ "token_correspondence_Prims.op_Multiply" ], 0, - "98657fb30fbbd43f8c66518a600cf679" + "617b0c87f2828e9a391d6dbc8da67151" ], [ "CanonCommSemiring.exp", @@ -740,7 +740,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "51e33310207efeba76be1bf61d6c2ed2" + "b332b74b971b343f853d41b2a20fd96e" ], [ "CanonCommSemiring.__proj__Var__item___0", @@ -754,7 +754,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_8b689800a5c7de58fa5eb3a86d8f2b39" ], 0, - "2d8a5a725562098459b71d33e447e166" + "d7f7e2082c20668cc1bd09e28701b796" ], [ "CanonCommSemiring.__proj__Add__item___0", @@ -768,7 +768,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_f7b11b9e2e3b3ea1b294881eaa75b765" ], 0, - "c3dcf30eea16773b00a07860ad187816" + "2345301ae95c55d47e5820a053976209" ], [ "CanonCommSemiring.__proj__Add__item___1", @@ -782,7 +782,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_f7b11b9e2e3b3ea1b294881eaa75b765" ], 0, - "13ca1aa14bf931254b1426ded2938e39" + "c89061f434dc3a712db991be067081e8" ], [ "CanonCommSemiring.__proj__Mult__item___0", @@ -796,7 +796,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_7ebec51792cf922a19b62c9c71962f29" ], 0, - "aa2b7764302f80d1e85b3fc05e944da5" + "1ec541717e96a07fac29aae3be4d7303" ], [ "CanonCommSemiring.__proj__Mult__item___1", @@ -810,7 +810,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_7ebec51792cf922a19b62c9c71962f29" ], 0, - "e26d9a19145db097a4dd9bd82a86c10e" + "a71c96e1e44612bc4599edd4f93c8345" ], [ "CanonCommSemiring.exp_to_string", @@ -828,7 +828,7 @@ "subterm_ordering_CanonCommSemiring.Mult" ], 0, - "d95c184f305c21199d23785212826794" + "474a40a47f7a8d06848cd2bb53b6853b" ], [ "CanonCommSemiring.quote_exp", @@ -843,7 +843,7 @@ "fuel_guarded_inversion_CanonCommSemiring.exp" ], 0, - "aaf8af7b1c8478bdc2d31c03ce870fad" + "6acf791d4cd90d85f0d3499b87ec4178" ], [ "CanonCommSemiring.rdenote", @@ -866,7 +866,7 @@ "subterm_ordering_CanonCommSemiring.Mult" ], 0, - "05d68c6c304397454edd1908f5d39bf5" + "e76c9400456b7633362d331655b4c28a" ], [ "CanonCommSemiring.sum_of_products", @@ -875,7 +875,7 @@ 1, [ "@query", "assumption_CanonCommMonoid.exp__uu___haseq" ], 0, - "9d56bc1ecee91be88a4de58aa8de4417" + "4b8c63233e5e3199469ee72f5e88fd27" ], [ "CanonCommSemiring.__proj__Product__item___0", @@ -889,7 +889,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_c9c5705ff62947a3a85bf808488463d7" ], 0, - "ae2c828560a620eafc763fc2652227e6" + "78167c277884b500e51f3e5e2ceab13e" ], [ "CanonCommSemiring.__proj__Sum__item___0", @@ -903,7 +903,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_c4b343140a7f62b6023c700d9c444ae3" ], 0, - "8359295464c17db0e53d87bffbf5d888" + "fbfc470f13c3f595354be2a15cc31a21" ], [ "CanonCommSemiring.__proj__Sum__item___1", @@ -917,7 +917,7 @@ "refinement_interpretation_CanonCommSemiring_Tm_refine_c4b343140a7f62b6023c700d9c444ae3" ], 0, - "0357904eb37b5bb36591b0605e1324b0" + "a78eb0ab6e963c282571938027a998f7" ], [ "CanonCommSemiring.sum_denote", @@ -938,7 +938,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "77b4a08399662c87d844e8233508852c" + "7c56ce103d69d04dc89520087966a35d" ], [ "CanonCommSemiring.multiply_sums", @@ -963,7 +963,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "605f939762fc5edd57ac2a6623f164df" + "610f96e74ff4ec80e9d6ac68e5a5754c" ], [ "CanonCommSemiring.exp_to_sum", @@ -981,7 +981,7 @@ "subterm_ordering_CanonCommSemiring.Mult" ], 0, - "ff5f4ec9b505c5a7d111fbb094d1a0d2" + "77327e8dcc895949c51ad3ca0dd2adf0" ], [ "CanonCommSemiring.cdenote", @@ -1002,7 +1002,7 @@ "subterm_ordering_CanonCommSemiring.Sum" ], 0, - "aaadf275aa86911fa31dda6901efd21a" + "5fc060def19b49fddfe18ca812ad6b27" ], [ "CanonCommSemiring.semiring_reflect", @@ -1015,7 +1015,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "34e11953017bd6fc3da858f9caddc810" + "2a4f41b75fefdd1d05db2cc0295bf38b" ], [ "CanonCommSemiring.make_fvar", @@ -1037,7 +1037,7 @@ "typing_FStar.Pervasives.Native.uu___is_Some" ], 0, - "d4ca65b5ccc1017b5ae2c648c0e99724" + "45498d88b30c175ad2d595fe79a7ccf2" ], [ "CanonCommSemiring.is_not_const", @@ -1054,7 +1054,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "function_token_typing_FStar.Reflection.Types.name", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", @@ -1062,7 +1062,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "e0e7e94e180dac783f9a0d326c5386ba" + "6a6ff7435fa97fc5c5d938cced27415c" ], [ "CanonCommSemiring.lem0", @@ -1075,7 +1075,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "92a456ab27615db44da289f8a9dfda68" + "def37348327780c364c17d09a074caba" ], [ "CanonCommSemiring.modulo_addition_lemma", @@ -1088,7 +1088,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "710ccdf24115b8471c2801fe7f8cf836" + "bdd77cac081f6e7533527864ce8668bc" ], [ "CanonCommSemiring.lemma_div_mod", @@ -1100,7 +1100,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "d027c793f4b4c3523526d69b7e2c4517" + "ce3ccbfb3e0866e3aa0e9f248579e4f2" ], [ "CanonCommSemiring.lemma_poly_multiply", @@ -1115,7 +1115,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "e620dc8a4186953335c5ff1a0aab00bd" + "2d28bf7af86e63706e9b42a52dbaca3c" ], [ "CanonCommSemiring.lemma_poly_reduce", @@ -1134,7 +1134,7 @@ "unit_typing" ], 0, - "46a9fa83567ac7a6a35651ed584a6b1d" + "b7a4b4c334cc5c6866b0fc330d41a6a5" ] ] ] \ No newline at end of file diff --git a/examples/tactics/CanonCommSwaps.fst.hints b/examples/tactics/CanonCommSwaps.fst.hints index d446cf17cfa..e8f745d452d 100644 --- a/examples/tactics/CanonCommSwaps.fst.hints +++ b/examples/tactics/CanonCommSwaps.fst.hints @@ -74,7 +74,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "112d9d2ada2d2442a963cb54ad8480bb" + "c8496c8704bfa5dd517b5c3fdfe62817" ], [ "CanonCommSwaps.apply_swaps", @@ -98,7 +98,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.length" ], 0, - "bd04d12b4c8ab8baaab80c7f41d1854c" + "73af305ab03d7020f5f45fac401d7719" ], [ "CanonCommSwaps.extend_equal_counts", @@ -291,7 +291,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "244e6e9e3cda572f40438c10cfdf6364" + "f3d69a1073f8b1ba755fe61e02b385b7" ], [ "CanonCommSwaps.swap_to_front", @@ -337,7 +337,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "71428de7b8088ff56e82d2a761f0e2b6" + "e29d47a0fb8615e0c3eb1f2e0f6c8967" ], [ "CanonCommSwaps.equal_counts_implies_swaps", @@ -376,7 +376,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "d56beceaa2d39ef597089b6580f2ac43" + "a879e8a9b6d20f4354a4e2053169feb7" ], [ "CanonCommSwaps.apply_swap_aux", @@ -429,7 +429,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "eb76ee4c4c8867947cc04d383c9c9f87" + "2260c1dcb81f8e9bf5ede5800abdec74" ], [ "CanonCommSwaps.apply_swaps", @@ -454,7 +454,7 @@ "subterm_ordering_Prims.Cons", "typing_FStar.List.Tot.Base.length" ], 0, - "97ddfb3db17870dfdefa077cb6ffe175" + "7c5a26aae0fdc346646ca97a9d1aaa70" ], [ "CanonCommSwaps.append_swaps", @@ -535,7 +535,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "5cc2d8d210a7b3674031b7fa603edeaf" + "36b104d107a5c4adba65db39e539ea7b" ], [ "CanonCommSwaps.swap_to_front", @@ -581,7 +581,7 @@ "token_correspondence_FStar.List.Tot.Base.length.fuel_instrumented" ], 0, - "8909871e410b9bc05ef18aad0a61b844" + "7f0aa69b932b52dcac6a6f427639f565" ], [ "CanonCommSwaps.equal_counts_implies_swaps", @@ -620,7 +620,7 @@ "typing_FStar.List.Tot.Base.length" ], 0, - "a7622cfff6489df7f54fbb7f8d5afe56" + "228e0e1246916e132fef7e259292d6a4" ] ] ] \ No newline at end of file diff --git a/examples/tactics/CanonMonoid.fst.hints b/examples/tactics/CanonMonoid.fst.hints index 2dbe1a46baf..e91dde53cb1 100644 --- a/examples/tactics/CanonMonoid.fst.hints +++ b/examples/tactics/CanonMonoid.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "eb4e6b194455381bb83b002a11bc7636" + "8b98a164656a7cba1c54b5787506b715" ], [ "CanonMonoid.__proj__Var__item___0", @@ -21,7 +21,7 @@ "refinement_interpretation_CanonMonoid_Tm_refine_3aa12bf376c0a044f35aca70ccec3774" ], 0, - "3f03eb1de09d6cdc0bd95b4785564d3c" + "ca86aa8daf5ac8722ac7c40bdf9acf25" ], [ "CanonMonoid.__proj__Mult__item___0", @@ -34,7 +34,7 @@ "refinement_interpretation_CanonMonoid_Tm_refine_1a92faa5d804af3a0048eaa96d6d9c4e" ], 0, - "1c27f88156d2944707ed124914674861" + "1051bc8d6ed3c71647c99c1eea113352" ], [ "CanonMonoid.__proj__Mult__item___1", @@ -47,7 +47,7 @@ "refinement_interpretation_CanonMonoid_Tm_refine_1a92faa5d804af3a0048eaa96d6d9c4e" ], 0, - "568997d0f3709d6f7bebbf82f082bd36" + "88179e79fb6f312c7c56511539c41170" ], [ "CanonMonoid.exp_to_string", @@ -63,7 +63,7 @@ "subterm_ordering_CanonMonoid.Mult" ], 0, - "d18c7b7325c61a585a31d67d6600bfe5" + "fea6cf3beb830a8d921c3c267556f9bb" ], [ "CanonMonoid.mdenote", @@ -83,7 +83,7 @@ "subterm_ordering_CanonMonoid.Mult" ], 0, - "f5e0edd735dd87d450b8ca067f769f32" + "a88fca3900a5ca3a8aae09969224e7c4" ], [ "CanonMonoid.mldenote", @@ -101,7 +101,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "89565f75880217e2757ea4dcb3e4ab6d" + "4714e4970a68504de27d9955dcf7de48" ], [ "CanonMonoid.flatten", @@ -117,7 +117,7 @@ "subterm_ordering_CanonMonoid.Mult" ], 0, - "3de1cb1b0022bb525715ba6368cd4a8d" + "baf5300d47f86fb4311dc3ad05aa8643" ], [ "CanonMonoid.flatten_correct_aux", @@ -160,7 +160,7 @@ "typing_CanonMonoid.mldenote", "unit_typing" ], 0, - "1949c31983aee7d8b9b2c0cb778e8a8e" + "aac27d4c2e8bc746d31ff96cf8c6d153" ], [ "CanonMonoid.flatten_correct", @@ -199,7 +199,7 @@ "subterm_ordering_CanonMonoid.Mult" ], 0, - "14b451c5f592c25faccfe829f68668ac" + "4c644cdda7b6f6050c5e8af861a26384" ], [ "CanonMonoid.monoid_reflect", @@ -212,7 +212,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "52d763fce5351a32130ffcb145cc9685" + "cbf7946a907af33aa5d0f4fe9dde1f33" ], [ "CanonMonoid.dump", @@ -229,7 +229,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "8956747877bfbf811d4087516e13efdb" + "f0895a3b5b6f2061de761c781829c0f7" ], [ "CanonMonoid.exp", @@ -238,7 +238,7 @@ 1, [ "@query" ], 0, - "ff033f142399cfc2a6d758e85fd49f71" + "ea19a084631f029e07ebf4584a4a8a8a" ], [ "CanonMonoid.__proj__Var__item___0", @@ -251,7 +251,7 @@ "refinement_interpretation_CanonMonoid_Tm_refine_3aa12bf376c0a044f35aca70ccec3774" ], 0, - "fd3e3d64e225f23fff08da38e6c39bf1" + "efaef4747e6f33f6cb3d36cbf7ee0919" ], [ "CanonMonoid.__proj__Mult__item___0", @@ -264,7 +264,7 @@ "refinement_interpretation_CanonMonoid_Tm_refine_1a92faa5d804af3a0048eaa96d6d9c4e" ], 0, - "6d7b8217ecd3e2e45d72cc6057d8664c" + "1216d9546f38d9ec3f84274f2ed92791" ], [ "CanonMonoid.__proj__Mult__item___1", @@ -277,7 +277,7 @@ "refinement_interpretation_CanonMonoid_Tm_refine_1a92faa5d804af3a0048eaa96d6d9c4e" ], 0, - "a00020fa30f3f651274214a81cd78f7e" + "5c74f81a436600fad0d80cbfbcf196b2" ], [ "CanonMonoid.exp_to_string", @@ -293,7 +293,7 @@ "subterm_ordering_CanonMonoid.Mult" ], 0, - "703e1660e4f70a99622963cae903d05e" + "eab16f2f66a38b6672e400f098683317" ], [ "CanonMonoid.mdenote", @@ -313,7 +313,7 @@ "subterm_ordering_CanonMonoid.Mult" ], 0, - "7628e189cfe0b8d4097e7568f57abcce" + "4ef75822ef9666b3a17d4460f71c40ed" ], [ "CanonMonoid.mldenote", @@ -331,7 +331,7 @@ "projection_inverse_Prims.Cons_tl", "subterm_ordering_Prims.Cons" ], 0, - "103bc8046e5372509a7434dd499814f1" + "1bc35b21343bab7b61b166c03b98eb8a" ], [ "CanonMonoid.flatten", @@ -347,7 +347,7 @@ "subterm_ordering_CanonMonoid.Mult" ], 0, - "768e0296a8dbf71b546a42df0fd089d6" + "fd7da641bc66516532005acfe6f914cc" ], [ "CanonMonoid.monoid_reflect", @@ -360,7 +360,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "47e9ddd104e2ff43e1aed32b48db02ad" + "25b2e2068ebc28ab92eaf04165b68c48" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Cases.fst.hints b/examples/tactics/Cases.fst.hints index 61df61f4b32..858d2d1cf7b 100644 --- a/examples/tactics/Cases.fst.hints +++ b/examples/tactics/Cases.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "true_interp" ], 0, - "96609fb104861b388d2bf2f80065a09c" + "dd06d04a532eb7edf16f1e056005e951" ], [ "Cases.test_cases_unsquash", @@ -17,7 +17,7 @@ 1, [ "@query", "true_interp" ], 0, - "6ead1fbb8a5c4443728e2f41910e75fd" + "a93954e95027e31205b476989b5ae9c6" ], [ "Cases.test_cases_bool", @@ -26,7 +26,7 @@ 1, [ "@query", "true_interp" ], 0, - "1a37e8f5b6b0bae8eaff7ebcf2e8cd56" + "743106ba4855d42775957a2c8d81bd23" ], [ "Cases.test_cases_bool_2", @@ -35,7 +35,7 @@ 1, [ "@query", "true_interp" ], 0, - "4552e5cec88ccb5efd940a3a9f1ed0c1" + "934ed529cc6e687279daf51030ac2479" ], [ "Cases.test_cases_bool_2", @@ -44,7 +44,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "d1e056aa7c761f52094e43891787c134" + "4b9f80f13c8d35404048ea29a5f148e0" ], [ "Cases.test_cases_bool_2", @@ -58,7 +58,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "1bd6c85b6f9055b8a7f59970311c76f2" + "d61a5ea779ffb61a050eb671c7ca868c" ], [ "Cases.test_cases_bool_2", @@ -72,7 +72,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "5453097f3a89088408c4c7c01e36d045" + "572c82d03ee5095aefc3d97767a353e0" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Change.fst.hints b/examples/tactics/Change.fst.hints index d04e7fc4d57..7173ab3e3a8 100644 --- a/examples/tactics/Change.fst.hints +++ b/examples/tactics/Change.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "equation_Change.id" ], 0, - "b6b7f302b6aaaff8d71b0f783cf1fafc" + "fd72a538cf29722e9b92ab72a64f2c32" ], [ "Change.uu___64", @@ -17,7 +17,7 @@ 1, [ "@query", "equation_Change.id" ], 0, - "d08e387c466918bc8bbbe7c3b6893fab" + "115ab3df3fa44c6fa9f6120a9573d625" ], [ "Change.uu___63", @@ -26,7 +26,7 @@ 1, [ "@query", "equation_Change.id" ], 0, - "91b841cbf8bf05efc6cd38ec43458678" + "b946ad45ee5a7722bab94aa4586301aa" ], [ "Change.uu___64", @@ -35,7 +35,7 @@ 1, [ "@query", "equation_Change.id" ], 0, - "8a62175b112f20f244082a8ae960884a" + "9460296dd9ab473b8b4d1b583900bcbb" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Clear.fst.hints b/examples/tactics/Clear.fst.hints index f2b27079ac0..0c495326fa8 100644 --- a/examples/tactics/Clear.fst.hints +++ b/examples/tactics/Clear.fst.hints @@ -16,7 +16,7 @@ "true_interp", "unit_typing" ], 0, - "7577b5a119b61f10865eedf090c262c0" + "05dbbb2c0304691ebd941a83900aaaa1" ], [ "Clear.l2", @@ -33,7 +33,7 @@ "true_interp", "unit_typing" ], 0, - "88aa2d34b24dbd208da9f6b41cc675d6" + "b346278a39dcc17b7a0d94919958563b" ], [ "Clear.l2", @@ -46,7 +46,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "282405bc8d1f381a8e10e2ece1e2734b" + "37b0e3c8e3944426007509cea6fbba61" ], [ "Clear.l2", @@ -62,7 +62,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "unit_typing" ], 0, - "3addbf8373e962a7ca6a9f98a645d910" + "3a339bdf423168a9ad24e73f43203a09" ], [ "Clear.l2", @@ -79,7 +79,7 @@ "true_interp", "unit_typing" ], 0, - "0ed4014613f5346d46f793d1b076ce15" + "9003bc5962e92a4e6e788f135bd49240" ], [ "Clear.l2", @@ -92,7 +92,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "5d7fb36f30516238e9e48baab19475a3" + "b246689872f15ee9beae842ca267a1a4" ] ] ] \ No newline at end of file diff --git a/examples/tactics/DeltaDepth.fst.hints b/examples/tactics/DeltaDepth.fst.hints index 34476ecb94f..d9352b95d65 100644 --- a/examples/tactics/DeltaDepth.fst.hints +++ b/examples/tactics/DeltaDepth.fst.hints @@ -10,7 +10,7 @@ "@query", "assumption_Prims.HasEq_bool", "assumption_Prims.HasEq_int" ], 0, - "bfefefbd66c3b55e3df165eaf12c489a" + "8b46db1a0d742ed82f7761f156221b6d" ], [ "DeltaDepth.__proj__A__item___0", @@ -23,7 +23,7 @@ "refinement_interpretation_DeltaDepth_Tm_refine_5e57589849c6497f93798a0ea15a1df2" ], 0, - "dce474f6b89e6fd15909b7c08e0a56f1" + "4f6f959eba5939ddeb0277a7bc8ebb0d" ], [ "DeltaDepth.__proj__B__item___0", @@ -36,7 +36,7 @@ "refinement_interpretation_DeltaDepth_Tm_refine_90c35950d1e7f0a820470167e5c76674" ], 0, - "d103606efbd5c5a1d54781c2ba0a5db1" + "522024d11be8e33c114cd5d3ceca0d83" ], [ "DeltaDepth.m", @@ -49,7 +49,7 @@ "projection_inverse_DeltaDepth.A__0" ], 0, - "e95488fa750841365f5aee955350b61b" + "724b2bbf45116b061bedc58292b47011" ], [ "DeltaDepth.t", @@ -60,7 +60,7 @@ "@query", "assumption_Prims.HasEq_bool", "assumption_Prims.HasEq_int" ], 0, - "e0e09cbb2282e31a0660a0e5d04605d9" + "95a1ee36810152fd1e08479c3945a0af" ], [ "DeltaDepth.__proj__A__item___0", @@ -73,7 +73,7 @@ "refinement_interpretation_DeltaDepth_Tm_refine_5e57589849c6497f93798a0ea15a1df2" ], 0, - "d81d1f1ed2111aa7c75436cbe5441bb3" + "34af671d5a5dd3872f141469c80bf7a5" ], [ "DeltaDepth.__proj__B__item___0", @@ -86,7 +86,7 @@ "refinement_interpretation_DeltaDepth_Tm_refine_90c35950d1e7f0a820470167e5c76674" ], 0, - "9c6bb8d79b97c7ddfb1648611d1d280e" + "549bae54c6552e28e3a2769c66eac49d" ], [ "DeltaDepth.m", @@ -99,7 +99,7 @@ "projection_inverse_DeltaDepth.A__0" ], 0, - "d6eaa9c63c013b22296467f4a6e63596" + "117575a381d8462b97827321e74057bb" ] ] ] \ No newline at end of file diff --git a/examples/tactics/DependentSynth.fst.hints b/examples/tactics/DependentSynth.fst.hints index a1b0576a3c7..5125b85bda7 100644 --- a/examples/tactics/DependentSynth.fst.hints +++ b/examples/tactics/DependentSynth.fst.hints @@ -11,7 +11,7 @@ "equation_DependentSynth.myty", "int_typing", "unit_typing" ], 0, - "04db54c4ce16221b5482cbecb391fdd1" + "e0485ae0b91a2911bc978071789e9db8" ], [ "DependentSynth.f", @@ -23,7 +23,7 @@ "equation_DependentSynth.myty", "int_typing", "unit_typing" ], 0, - "74672c3102e611cdbfe55c5d4e23771c" + "109255473799bb48f910fb6bd959a7c0" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Destruct.fst.hints b/examples/tactics/Destruct.fst.hints index 5ba6c0fd9eb..14e1d6342b3 100644 --- a/examples/tactics/Destruct.fst.hints +++ b/examples/tactics/Destruct.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "f74f9b25693e43595c4184787401c5b9" + "8114613e0baba8cdc66635c521e2c859" ], [ "Destruct.uu___64", @@ -17,7 +17,7 @@ 1, [ "@query" ], 0, - "31717518b4f8bf3db0c80e35d130cd88" + "8986f700b31c5d84e3ce8d86944a28fb" ], [ "Destruct.uu___65", @@ -26,7 +26,7 @@ 1, [ "@query" ], 0, - "5dbe52a767e8ffa51745b8602578c738" + "239d3b0cd498bb17c9379729fc85d972" ], [ "Destruct.t2", @@ -48,7 +48,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "420fdaec714a167cec360a788c54a272" + "ff7c8d988dac0fc3448f51ea21e6f5ec" ], [ "Destruct.__proj__A2__item___0", @@ -61,7 +61,7 @@ "refinement_interpretation_Destruct_Tm_refine_15d80be637ca75d5c418364229a1bb22" ], 0, - "b69600c35c35b7bb77a0630e73110972" + "5e541db18b035c98c70295bbd2f41b9d" ], [ "Destruct.__proj__B2__item___0", @@ -74,7 +74,7 @@ "refinement_interpretation_Destruct_Tm_refine_cb5b47cb8fe6a6ad9ef550685a5d6a5d" ], 0, - "34411cf47ea0aa14d606e5ba470e6810" + "43ef6a5da1839a4d7fddea967b49121e" ], [ "Destruct.__proj__C2__item___0", @@ -87,7 +87,7 @@ "refinement_interpretation_Destruct_Tm_refine_42019ac1942b4ff52b545bc4be0e0841" ], 0, - "d44c061034169555b39585d7241f0534" + "07eeca6cb8591f3ff2fc4aa98ac34487" ], [ "Destruct.__proj__C2__item___1", @@ -100,7 +100,7 @@ "refinement_interpretation_Destruct_Tm_refine_42019ac1942b4ff52b545bc4be0e0841" ], 0, - "d5efc2e00e96455aa428c6a9ec6ea0b1" + "426433c36d6dc333ed5da93946407b45" ], [ "Destruct.__proj__C2__item___2", @@ -113,7 +113,7 @@ "refinement_interpretation_Destruct_Tm_refine_42019ac1942b4ff52b545bc4be0e0841" ], 0, - "d700fbea0e0e61c5ff16bd1800d9ef3b" + "16a0c990a46e26f1dc41118062084f23" ], [ "Destruct.uu___66", @@ -122,7 +122,7 @@ 1, [ "@query" ], 0, - "58bf5cc789fc7d26cfb675f9f51927ae" + "ee642d4ad2388c1c9d89d638b34e10ed" ], [ "Destruct.uu___67", @@ -134,7 +134,7 @@ "projection_inverse_Destruct.A3_i" ], 0, - "12e21aa66460a3ed3523ce51e74444c8" + "2f044ed147ad11a3f87b3a545a7c8c3f" ], [ "Destruct.uu___68", @@ -147,7 +147,7 @@ "projection_inverse_Destruct.B3_i" ], 0, - "e0be690d5bcca79efae1f3eb7b1a7b7b" + "6565f2a7695d1892e7607710f7b7b1d6" ], [ "Destruct.t3", @@ -169,7 +169,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "ff983107303675b45f2f53205bd30594" + "f295d1c2fd4b20b75bb3f390bfe5635f" ], [ "Destruct.__proj__B3__item___0", @@ -182,7 +182,7 @@ "refinement_interpretation_Destruct_Tm_refine_09dde35c659cf7f75ce8e59a37558929" ], 0, - "8395964844c0bb0aafeca34f433bb111" + "10d0ebb98c30cb0d2facdbc3e5d40718" ], [ "Destruct.__proj__C3__item___0", @@ -195,7 +195,7 @@ "refinement_interpretation_Destruct_Tm_refine_11b50967a69485f0d567e8d70b8ffdc0" ], 0, - "5897a281458cd184cbd4921c11bd9f05" + "9ca37158aee380f13b0d05002b188ffe" ], [ "Destruct.__proj__C3__item___1", @@ -208,7 +208,7 @@ "refinement_interpretation_Destruct_Tm_refine_11b50967a69485f0d567e8d70b8ffdc0" ], 0, - "aed5b8f723bb4b518e3bbb973c381bbf" + "d1f4a7ad3082aa5bd04a58b2e8e7b3af" ], [ "Destruct.uu___69", @@ -222,7 +222,7 @@ "projection_inverse_Destruct.C3_i" ], 0, - "cdaa084cb14780582400280d896b1e4f" + "b41827192dc0d4abfb9ee770690f5f6f" ], [ "Destruct.uu___70", @@ -231,7 +231,7 @@ 1, [ "@query" ], 0, - "a05a435d422bf024f250eae8a27384b3" + "a32a8f60610424bc8ce8ebdb4f21e908" ], [ "Destruct.uu___71", @@ -240,7 +240,7 @@ 1, [ "@query" ], 0, - "7a4e14dd2d3a96498510bd51f27159bf" + "6a814fe4a4c75bd99acad8196d7999bc" ], [ "Destruct.t4", @@ -260,7 +260,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "356d0ba975eb8fc64695d92feb76c207" + "7948ca7755510c975deaac36ffff9d93" ], [ "Destruct.__proj__A4__item___0", @@ -273,7 +273,7 @@ "refinement_interpretation_Destruct_Tm_refine_56ba732a08a46e2a006cb7cd49c61bb2" ], 0, - "04791cbc1bb229485bc7ea5a8e6d6883" + "b36ec6bb1ed9a64b1348b3cb67db6d41" ], [ "Destruct.__proj__B4__item___0", @@ -286,7 +286,7 @@ "refinement_interpretation_Destruct_Tm_refine_316b60465156994faf26a3b05c39e34a" ], 0, - "c848dbb0e161f2a4ae432d91a63ad6be" + "22d7d1a5dc7982309e53746149fd3b05" ], [ "Destruct.__proj__C4__item___0", @@ -299,7 +299,7 @@ "refinement_interpretation_Destruct_Tm_refine_bb2e13b75ca87847a19e6c915787a293" ], 0, - "029a033d1fe94bd5d192237f11e65a5b" + "4b46d46ef6eb8e67b0aa30aacaec511a" ], [ "Destruct.__proj__C4__item___1", @@ -312,7 +312,7 @@ "refinement_interpretation_Destruct_Tm_refine_bb2e13b75ca87847a19e6c915787a293" ], 0, - "9a84972079d968cf41189cd185ab234d" + "4d3f8e8d5f9445ce3d2d347f3268c2f5" ], [ "Destruct.__proj__C4__item___2", @@ -325,7 +325,7 @@ "refinement_interpretation_Destruct_Tm_refine_bb2e13b75ca87847a19e6c915787a293" ], 0, - "a4291954813ecd779ec8cbfcb5aa4454" + "78e54486502557ec9e071142fea56f35" ], [ "Destruct.uu___72", @@ -334,7 +334,7 @@ 1, [ "@query" ], 0, - "d4116967b07d698900bdeb6122b57ed0" + "6b72f57e592ea2dbea3fd599f5bd7c4a" ], [ "Destruct.uu___73", @@ -343,7 +343,7 @@ 1, [ "@query" ], 0, - "ea6bc173afa00c3ee9aa74b59d30a54a" + "2d31a984138845ec8b79a1b12313c97e" ], [ "Destruct.uu___74", @@ -352,7 +352,7 @@ 1, [ "@query" ], 0, - "a53aa8386948cfe1d9fbf562221be29f" + "bd22f802153ea94f459522c965ec67d8" ], [ "Destruct.vec", @@ -365,7 +365,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "8bff6c5b26d7234cc2f923c8c8672483" + "6d42522098589671440896226e9695de" ], [ "Destruct.vec", @@ -381,7 +381,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "04df3d1a815b4a840cd9ee36a24996a5" + "e7fa6b323b520a5a92ed0cf6c5ca81fa" ], [ "Destruct.__proj__VCons__item__n", @@ -394,7 +394,7 @@ "refinement_interpretation_Destruct_Tm_refine_30dcdfe3f7fdaa373efe7d0f17e40dc2" ], 0, - "6cee2be2ae1f508bd2c2862e579b8644" + "b7d410caff21dfd129e3974689a7a251" ], [ "Destruct.__proj__VCons__item___1", @@ -407,7 +407,7 @@ "refinement_interpretation_Destruct_Tm_refine_30dcdfe3f7fdaa373efe7d0f17e40dc2" ], 0, - "08622275f95dd97cdf7b46f6e03f9975" + "508b3914c5261b5672d3b0f1fda2e466" ], [ "Destruct.__proj__VCons__item___2", @@ -424,7 +424,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "d5b6b16a078a945a4517af8d4aec6b44" + "81b092f527ee6aba7ba10e2626aa8ff5" ], [ "Destruct.uu___75", @@ -433,7 +433,7 @@ 1, [ "@query" ], 0, - "9a64f3ca4fa1d3541f31b20b76516c20" + "f3ac5bdc92a61cfdaa9b3583b553e11e" ], [ "Destruct.uu___76", @@ -442,7 +442,7 @@ 1, [ "@query" ], 0, - "03a570ca5ff29274263da9ecbf78c7a7" + "84ac83c5ede5f9654b47055683010e9e" ], [ "Destruct.uu___77", @@ -451,7 +451,7 @@ 1, [ "@query" ], 0, - "0eccc59dc0cea9a86c2d0d46778cf129" + "f98e645bdf945e7bc4996df9867ec5ee" ], [ "Destruct.fin", @@ -464,7 +464,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "67a83bf6617cb8977f3bc2810b7d29a9" + "a90f9be75e39fb5ae521f87e55109331" ], [ "Destruct.fin", @@ -479,7 +479,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "cfe5c2d335aa688ab70baed6430149d0" + "305d92072b3892bedbb602bd18b16465" ], [ "Destruct.__proj__Z__item__n", @@ -492,7 +492,7 @@ "refinement_interpretation_Destruct_Tm_refine_091244a5b42f3d992595a20613c09453" ], 0, - "eae36eb7a4fa5cdbb490affecae78f31" + "79b090a478e9caf2c08b79f3430f4a75" ], [ "Destruct.__proj__S__item__n", @@ -505,7 +505,7 @@ "refinement_interpretation_Destruct_Tm_refine_409191d6e26cee56f95ecac12bcba703" ], 0, - "e325bcb508c3d60db185a7fe8e3da84a" + "1359e8e10c2ce743d29ba5befda21e15" ], [ "Destruct.__proj__S__item___1", @@ -521,7 +521,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "181f131fa166dc01bf03fb6b5a87a90e" + "280fa523960692aa4cd39b1871435777" ], [ "Destruct.decr2", @@ -537,7 +537,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "ff8c28fab5daa0f6c85ca2be65b16d92" + "f9fdd16e33ff1ba721eee9ecb9bde9e9" ], [ "Destruct.decr2", @@ -550,7 +550,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "02391667d1f07bf8b9154e7cace340d4" + "c7ab21d6d49acf358db563974d2acb22" ], [ "Destruct.intros'", @@ -568,7 +568,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "b0b2cbfa6a26bb2fc5583f665851e43a" + "af3c5ab978db02570eb21c8c6df3f339" ], [ "Destruct.destruct", @@ -586,7 +586,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "36abb4a2c6da7a1bdc02586278e21fca" + "55974719f8b2729b7b2ea06997371648" ], [ "Destruct.f1", @@ -599,7 +599,7 @@ "fuel_guarded_inversion_Destruct.t1" ], 0, - "166bc2472cccd8c53d1e7d5e8dfc362f" + "0a949434166156c328db7fd1d24fd0bb" ], [ "Destruct.uu___63", @@ -608,7 +608,7 @@ 1, [ "@query" ], 0, - "6f1730243e1116ca7398811cd3175fed" + "299df6f83532b667b93658bde41a8cc5" ], [ "Destruct.uu___64", @@ -617,7 +617,7 @@ 1, [ "@query" ], 0, - "5f1215c6fd03daaa38c798d0e447ae23" + "47db4bdb375f6a477ddc48a469e34694" ], [ "Destruct.uu___65", @@ -626,7 +626,7 @@ 1, [ "@query" ], 0, - "30508c2829a8c25dfc6c435f7a329212" + "b1af6a29c5ebfabbeabbe9f9bf98eff8" ], [ "Destruct.t2", @@ -648,7 +648,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "3a436da1236d900b586e54fb00da49ed" + "f1140b6ddd2e131a8c646a45ae92233d" ], [ "Destruct.__proj__A2__item___0", @@ -661,7 +661,7 @@ "refinement_interpretation_Destruct_Tm_refine_15d80be637ca75d5c418364229a1bb22" ], 0, - "a92309e365690002005c38a935af26ed" + "0d36f1edb84666677c8eab7d84da1e0a" ], [ "Destruct.__proj__B2__item___0", @@ -674,7 +674,7 @@ "refinement_interpretation_Destruct_Tm_refine_cb5b47cb8fe6a6ad9ef550685a5d6a5d" ], 0, - "184cc49657073eff4d62ed438a6eb244" + "a6ba63fd9f7dc8117d207df0fd12871b" ], [ "Destruct.__proj__C2__item___0", @@ -687,7 +687,7 @@ "refinement_interpretation_Destruct_Tm_refine_42019ac1942b4ff52b545bc4be0e0841" ], 0, - "d3a6c47b64d629a45cd63b82075b06c6" + "2f8faecd121ab4c44ab84e089c4e047a" ], [ "Destruct.__proj__C2__item___1", @@ -700,7 +700,7 @@ "refinement_interpretation_Destruct_Tm_refine_42019ac1942b4ff52b545bc4be0e0841" ], 0, - "b7f4f18fea57b852697fa42ba3a14daf" + "dc39ef4c0102a7d93244f0565ecc9648" ], [ "Destruct.__proj__C2__item___2", @@ -713,7 +713,7 @@ "refinement_interpretation_Destruct_Tm_refine_42019ac1942b4ff52b545bc4be0e0841" ], 0, - "f85a2d4994d8e361a6d9dd7527b38abc" + "e67828958e80ad092864a34317250e38" ], [ "Destruct.f2", @@ -726,7 +726,7 @@ "fuel_guarded_inversion_Destruct.t2" ], 0, - "95634abc05393c136f56352a53794e4a" + "07163fd97bc643008e182ad022b66007" ], [ "Destruct.uu___66", @@ -735,7 +735,7 @@ 1, [ "@query" ], 0, - "4925793f6d59fdf211d71eed0869876f" + "8fd74cc4fd88853add6152b7c8fce0f6" ], [ "Destruct.uu___67", @@ -744,7 +744,7 @@ 1, [ "@query" ], 0, - "27a7f10c7a6a9e5611f3b5aa6df9aa7c" + "618dc2e9f0e0b01c0e71fcc78891b7f0" ], [ "Destruct.uu___68", @@ -753,7 +753,7 @@ 1, [ "@query" ], 0, - "532c3adebf81423f5969303ad7a82df8" + "cc9be70e1d0286873067cc3dffa51c92" ], [ "Destruct.t3", @@ -775,7 +775,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "1ec689a0b5cdf91787ee23174fe9cb27" + "d4481b59df1935190b4f374ec86ef18d" ], [ "Destruct.__proj__B3__item___0", @@ -788,7 +788,7 @@ "refinement_interpretation_Destruct_Tm_refine_09dde35c659cf7f75ce8e59a37558929" ], 0, - "b5effd98bfbb9187fb3fc0f6e7cf38da" + "819d50a2ea794c7a1829b47587096d36" ], [ "Destruct.__proj__C3__item___0", @@ -801,7 +801,7 @@ "refinement_interpretation_Destruct_Tm_refine_11b50967a69485f0d567e8d70b8ffdc0" ], 0, - "de231668c043db99274d48e667544116" + "4834f3aa04665c22cd1550fbca81d675" ], [ "Destruct.__proj__C3__item___1", @@ -814,7 +814,7 @@ "refinement_interpretation_Destruct_Tm_refine_11b50967a69485f0d567e8d70b8ffdc0" ], 0, - "78921794f8516a15a73ab9d2dea99369" + "d42aa492ffa4b33b6c4c5901f6c5f7ff" ], [ "Destruct.f3", @@ -827,7 +827,7 @@ "fuel_guarded_inversion_Destruct.t3" ], 0, - "07de2bbd70996b775ac4297a01b4f076" + "e8076963230f60c82653dbaa2c4f332f" ], [ "Destruct.uu___69", @@ -836,7 +836,7 @@ 1, [ "@query" ], 0, - "34c92af9107c6deb8e478571f5442072" + "9269415d1d9f21619cf885b5a2825d4c" ], [ "Destruct.uu___70", @@ -845,7 +845,7 @@ 1, [ "@query" ], 0, - "5eca3267002a634596d78cfecfdfaa3b" + "bd1799f0b5c5ac164346621508a2abea" ], [ "Destruct.uu___71", @@ -854,7 +854,7 @@ 1, [ "@query" ], 0, - "7b23ec95adcf12d4d36a4eab118fd864" + "6e74f983c1bc8de8206b3f157ae7c980" ], [ "Destruct.t4", @@ -874,7 +874,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "5cdfac83c2322f57db8def90b63c059c" + "006dc857239ae2dfbbfda0826f5df528" ], [ "Destruct.__proj__A4__item___0", @@ -887,7 +887,7 @@ "refinement_interpretation_Destruct_Tm_refine_56ba732a08a46e2a006cb7cd49c61bb2" ], 0, - "f13847831f3a114ef2dfc119ce2eb5a9" + "22bb28efb14166a617835d5d65ba63e7" ], [ "Destruct.__proj__B4__item___0", @@ -900,7 +900,7 @@ "refinement_interpretation_Destruct_Tm_refine_316b60465156994faf26a3b05c39e34a" ], 0, - "23472c7fc79acc2c41b485b88eecc5d9" + "4c6a882e6dc5cc87d789a08787572fe8" ], [ "Destruct.__proj__C4__item___0", @@ -913,7 +913,7 @@ "refinement_interpretation_Destruct_Tm_refine_bb2e13b75ca87847a19e6c915787a293" ], 0, - "0197dbff2d8a8f48971786ac9b718b18" + "ed5f119785a0bc48a798dfc806c4b40e" ], [ "Destruct.__proj__C4__item___1", @@ -926,7 +926,7 @@ "refinement_interpretation_Destruct_Tm_refine_bb2e13b75ca87847a19e6c915787a293" ], 0, - "97fd96f679f86830775ee0bb80576dd5" + "0ef3e19a08283da924ad2665c8ac0b9c" ], [ "Destruct.__proj__C4__item___2", @@ -939,7 +939,7 @@ "refinement_interpretation_Destruct_Tm_refine_bb2e13b75ca87847a19e6c915787a293" ], 0, - "e115ae83ffefce11afc73ea19dbb4bdf" + "4ceca80eb51d2b518fef17d557407cf4" ], [ "Destruct.f4", @@ -952,7 +952,7 @@ "fuel_guarded_inversion_Destruct.t4" ], 0, - "70521444239ec94244cf08b8f1e9aa5a" + "2c2d5925a8e23c86142c9e67e51d09eb" ], [ "Destruct.uu___72", @@ -961,7 +961,7 @@ 1, [ "@query" ], 0, - "d657ac2739a8e611ff91404013295bba" + "62783352f6d8d46e49382eedcd654512" ], [ "Destruct.uu___73", @@ -970,7 +970,7 @@ 1, [ "@query" ], 0, - "e3fb5c95ec5d2f9661895d81996c0b3f" + "01094e2a62998613af28ef8c38f5ab7c" ], [ "Destruct.uu___74", @@ -979,7 +979,7 @@ 1, [ "@query" ], 0, - "2157d1bccf67bc6f8b54582b90f02da6" + "0400ea99626934b29c7b0718f5db01d4" ], [ "Destruct.vec", @@ -992,7 +992,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "2d71154b1472480e6de60cda4d9752a3" + "07151afeb94f203f860aa6b44625cc76" ], [ "Destruct.vec", @@ -1008,7 +1008,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "f0e952dbd0eeb5a9d03c550f1c1932f0" + "a1e696f3ed950dbb3452285d1bced000" ], [ "Destruct.__proj__VCons__item__n", @@ -1021,7 +1021,7 @@ "refinement_interpretation_Destruct_Tm_refine_30dcdfe3f7fdaa373efe7d0f17e40dc2" ], 0, - "8df8b704ce2bf239ce3448e32d4746e7" + "31ed0022f144e649cc7566b096e6248a" ], [ "Destruct.__proj__VCons__item___1", @@ -1034,7 +1034,7 @@ "refinement_interpretation_Destruct_Tm_refine_30dcdfe3f7fdaa373efe7d0f17e40dc2" ], 0, - "b08d14f55a2e4c2e450bda96fd6eef3c" + "be9752bd9597db74f3a8ae7030aa95ac" ], [ "Destruct.__proj__VCons__item___2", @@ -1051,7 +1051,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "be651635981cacb8d451c762b13d88be" + "0fcca7b3d225577bdfcc729c1574b43b" ], [ "Destruct.vlen", @@ -1063,7 +1063,7 @@ "disc_equation_Destruct.VNil", "fuel_guarded_inversion_Destruct.vec" ], 0, - "3d5811bab545ed3b92f70d65cfdf727b" + "21feedbb344eeee80f93ea81b7a16f89" ], [ "Destruct.uu___75", @@ -1072,7 +1072,7 @@ 1, [ "@query" ], 0, - "f43523fa478d338191e5150344c4c428" + "ec9118fe849bf354b63a1c747d5a2139" ], [ "Destruct.uu___76", @@ -1081,7 +1081,7 @@ 1, [ "@query" ], 0, - "f495807519ea5b093298898a67c9eb3d" + "9f6f618bb26642b9d0395dc785191a86" ], [ "Destruct.uu___77", @@ -1090,7 +1090,7 @@ 1, [ "@query" ], 0, - "d486302bf67f23e3dfa117c2891a7493" + "f8dfff260bcb901a6913922152182b99" ], [ "Destruct.fin", @@ -1103,7 +1103,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "5bc48413f05b6a303db05c7330455970" + "9aec783d286d08677e10316ef04e61cf" ], [ "Destruct.fin", @@ -1118,7 +1118,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "2bdb13312498fe396374d1d54d797740" + "194fdfdd98aeeb2c6dcbec2ed6b9ea1d" ], [ "Destruct.__proj__Z__item__n", @@ -1131,7 +1131,7 @@ "refinement_interpretation_Destruct_Tm_refine_091244a5b42f3d992595a20613c09453" ], 0, - "b94e28ec5f27d13a9adace67c40a8b97" + "1b0e9ab16903af982083ae9b97c45636" ], [ "Destruct.__proj__S__item__n", @@ -1144,7 +1144,7 @@ "refinement_interpretation_Destruct_Tm_refine_409191d6e26cee56f95ecac12bcba703" ], 0, - "6bd8dcf2bf4bec6beaf2b44d7ebd8b63" + "b5ba849b29158d8b9568ae508c517305" ], [ "Destruct.__proj__S__item___1", @@ -1160,7 +1160,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "0d27de589ec3f4fedc9e8e09e17f2c05" + "c2a39515eedadad3d8c56ac7c6b3561b" ], [ "Destruct.decr2", @@ -1173,7 +1173,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "d9a1ce83c297637f9f06846cd0061313" + "888c94c8e5254172d5c54a347b74c826" ], [ "Destruct.decr2", @@ -1191,7 +1191,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "000cedb55aee57b3002fa94ef6b06952" + "20a3ae7e845461e4e0945b6af68055f7" ], [ "Destruct.decr2", @@ -1204,7 +1204,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "d1604b891eb084366a18164c6b317de7" + "3256857b7ad2be3ae0e00ae1b80b6038" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Easy.fst.hints b/examples/tactics/Easy.fst.hints index 0666e2af5e5..9bf98945dc0 100644 --- a/examples/tactics/Easy.fst.hints +++ b/examples/tactics/Easy.fst.hints @@ -11,7 +11,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "bd1eb595bcb06171a2d681a9235e7362" + "29461a50ebf84eeff43d70c1f3a5468b" ], [ "Easy.plus_assoc", @@ -23,7 +23,7 @@ "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0" ], 0, - "80ce6e56869aa025f12da94559f2ddc1" + "8cdfb820bdb8e57b54637151322e8877" ], [ "Easy.plus_comm", @@ -35,7 +35,7 @@ "primitive_Prims.op_Addition" ], 0, - "ab89bc817f12be0b6f2e7f8948dec523" + "440ba0ef1c4220b2e707e375dd84c1f6" ], [ "Easy.easy_fill", @@ -56,7 +56,7 @@ "typing_FStar.Tactics.Result.uu___is_Success" ], 0, - "7c3dff675095f3705675d451cd885e64" + "4840a1976e7888a6010017ba8796de66" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Even.fst.hints b/examples/tactics/Even.fst.hints index 31081e01b87..f029ceb8042 100644 --- a/examples/tactics/Even.fst.hints +++ b/examples/tactics/Even.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "76e0fb0ccad8cf158cdfdb2b9469e198" + "e7663c8a370888490a16fa189ac48c50" ], [ "Even.__proj__S__item___0", @@ -21,7 +21,7 @@ "refinement_interpretation_Even_Tm_refine_bb628da1f7d40b6a048cba9503380f5d" ], 0, - "fcfee50c4fa782e3d83877f36a886224" + "2851fa89d5c2053d2c27951aac1f0db0" ], [ "Even.nat2unary", @@ -37,7 +37,7 @@ "well-founded-ordering-on-nat" ], 0, - "a5a4db4f551a1652dd66745758873b92" + "e006e8dade5f4b31398aef9c94c01282" ], [ "Even.even", @@ -46,7 +46,7 @@ 1, [ "@query", "assumption_Even.unat__uu___haseq" ], 0, - "77a1d8baa3792353c3885230d533be21" + "1cc3eefdb5e6bfb8c2c956a62ab00fac" ], [ "Even.__proj__Even_SS__item__n", @@ -59,7 +59,7 @@ "refinement_interpretation_Even_Tm_refine_54b3fdb8b64a7b5a7f1535a28234d0d5" ], 0, - "8487849d7a17ce8c3c4a1956c62f2c2e" + "a8ba3fcd0facceb42c6762ca8716c086" ], [ "Even.__proj__Even_SS__item___1", @@ -73,7 +73,7 @@ "refinement_interpretation_Even_Tm_refine_54b3fdb8b64a7b5a7f1535a28234d0d5" ], 0, - "ad367a533d5f33b8e3f327a08bb11b19" + "9499ed335dc5f8333738464c540d837a" ], [ "Even.unat", @@ -82,7 +82,7 @@ 1, [ "@query" ], 0, - "864eb1496e9823afc632d0d9368153ec" + "c3095482f1fed08b9ac8eb5a3273d056" ], [ "Even.__proj__S__item___0", @@ -95,7 +95,7 @@ "refinement_interpretation_Even_Tm_refine_bb628da1f7d40b6a048cba9503380f5d" ], 0, - "3ede28491b4040540fd75a9ce5b98d6d" + "4d0546f7d8390f2830fba1d8099a5c51" ], [ "Even.nat2unary", @@ -111,7 +111,7 @@ "well-founded-ordering-on-nat" ], 0, - "c22a399de962bc8a45a72d722912fa08" + "4fadcee84e8846a99b85208baa1e8280" ], [ "Even.even", @@ -120,7 +120,7 @@ 1, [ "@query", "assumption_Even.unat__uu___haseq" ], 0, - "0ff778a869fc1d4eacb6aed02b4447d4" + "5656e1bfc6e468066c2cc9ecc616c532" ], [ "Even.__proj__Even_SS__item__n", @@ -133,7 +133,7 @@ "refinement_interpretation_Even_Tm_refine_54b3fdb8b64a7b5a7f1535a28234d0d5" ], 0, - "5ace0b856a76c07720c7829588d8783e" + "0b64a577715df93e519c0d38ea32d1c2" ], [ "Even.__proj__Even_SS__item___1", @@ -147,7 +147,7 @@ "refinement_interpretation_Even_Tm_refine_54b3fdb8b64a7b5a7f1535a28234d0d5" ], 0, - "2840f85b82f30d3d82a38e3fcefb9498" + "7e2d7c36ce6116ae12ca9f993ee3b83f" ], [ "Even.prove_even", @@ -166,7 +166,7 @@ "typing_FStar.Tactics.Result.uu___is_Success", "unit_typing" ], 0, - "b9aad9a2af50fd6fced0c1da4604d826" + "081523c1dcb43725c327b4ea1843d2c8" ] ] ] \ No newline at end of file diff --git a/examples/tactics/FailFlow.fst.hints b/examples/tactics/FailFlow.fst.hints index c3de4dd6dd1..0b59fc71059 100644 --- a/examples/tactics/FailFlow.fst.hints +++ b/examples/tactics/FailFlow.fst.hints @@ -1,29 +1 @@ -[ - "v\u0012\u0013ٜ\u000fJ\u0012\"{", - [ - [ - "FailFlow.fail_flow", - 1, - 2, - 1, - [ - "@query", "disc_equation_FStar.Tactics.Result.Failed", - "projection_inverse_BoxBool_proj_0" - ], - 0, - "484950c5a361468fa00015bde88e1038" - ], - [ - "FailFlow.fail_flow", - 2, - 2, - 1, - [ - "@query", "disc_equation_FStar.Tactics.Result.Failed", - "projection_inverse_BoxBool_proj_0" - ], - 0, - "b151a453eacfee437e26a3bfadc553d5" - ] - ] -] \ No newline at end of file +[ "ON\nk\u0019^\u0006lx\u0001", [] ] \ No newline at end of file diff --git a/examples/tactics/Fresh.fst.hints b/examples/tactics/Fresh.fst.hints index c8d7101f212..4fd026ec905 100644 --- a/examples/tactics/Fresh.fst.hints +++ b/examples/tactics/Fresh.fst.hints @@ -14,7 +14,7 @@ "function_token_typing_FStar.UInt32.n" ], 0, - "ec2e923ed0717bd0cc5d01b35dfbcbc6" + "691241a344a173d024df5136793c0155" ], [ "Fresh.uu___63", @@ -29,7 +29,7 @@ "function_token_typing_FStar.UInt32.n", "true_interp" ], 0, - "97281dd81948c8fd946df978d3192fab" + "9bd6ca1a416f2755bd2ef2b013fa934b" ], [ "Fresh.uu___63", @@ -44,7 +44,7 @@ "function_token_typing_FStar.UInt32.n" ], 0, - "fd56adb9cbcf41d28bba1e9fc292ee09" + "b495b4c51f79304d543bd8e2213bb3d3" ], [ "Fresh.uu___63", @@ -59,7 +59,7 @@ "function_token_typing_FStar.UInt32.n", "true_interp" ], 0, - "be9ded8e521328bfc6dc00c4e35d653b" + "6575f6013417257a4807a6a142306971" ] ] ] \ No newline at end of file diff --git a/examples/tactics/GRewrite.fst.hints b/examples/tactics/GRewrite.fst.hints index a6c00e5c030..9ecdf3c0358 100644 --- a/examples/tactics/GRewrite.fst.hints +++ b/examples/tactics/GRewrite.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "f99fe5b265355dd123e565faa95a8775" + "78c45a01f3de53038bb1416b834ed0b5" ], [ "GRewrite.test_grewrite2", @@ -17,7 +17,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "9dd713238cb094a01474c9990f53e5ea" + "e5e48b3b3aa9001bd80e29bcdc881525" ], [ "GRewrite.test_grewrite2", @@ -26,7 +26,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "9694a6dc4a33e077bce20f1e64dbf6c0" + "476bc428e1127077bd75d1ee8f5c1c71" ], [ "GRewrite.test_grewrite2", @@ -38,7 +38,7 @@ "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0" ], 0, - "81f9ac7ea31259c9e2a565650c96e089" + "30979ab1044ecc78ce1bd2bbb00b7b52" ], [ "GRewrite.test_grewrite4", @@ -47,7 +47,7 @@ 1, [ "@query", "eq2-interp", "equation_Prims.eq2" ], 0, - "b5636864052de9a159528acb2b140014" + "76e752079b99452c6e2f0445920f07df" ], [ "GRewrite.test_grewrite5", @@ -61,7 +61,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "30fd0931918e1d78a48064c601a95b5a" + "4cb7b874e67da55e1d5f0d58756338a8" ], [ "GRewrite.test_term_eq", @@ -70,7 +70,7 @@ 1, [ "@query", "true_interp" ], 0, - "76bb432710621cb1a08eba796eb053e1" + "aabe395017d8cf6f099c1130d2c62926" ], [ "GRewrite.test_grewrite2", @@ -79,7 +79,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "8f0ebd28240de0348042ac257767a667" + "ffde7083bea42a09d70882c88e591587" ], [ "GRewrite.test_grewrite2", @@ -88,7 +88,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "99d86ef7ce1a522f40ce9166928e9c1d" + "edbf0df38261121d2b875c438ad29cad" ], [ "GRewrite.test_grewrite2", @@ -97,7 +97,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "5e4948a7a354c50eaa4126df99cef0be" + "b34916ff8680343533a8814f8c65d335" ], [ "GRewrite.test_grewrite2", @@ -109,7 +109,7 @@ "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0" ], 0, - "9674c4eb28f527da2d02c48ce298b2f9" + "73e63c88729721b9275305a991e7d43a" ], [ "GRewrite.test_grewrite4", @@ -118,7 +118,7 @@ 1, [ "@query", "eq2-interp", "equation_Prims.eq2" ], 0, - "6845a7c1da6722d4f189b30c99af4d35" + "e6820d267ae935bb8d56f8b8e60f1e91" ], [ "GRewrite.test_grewrite5", @@ -132,7 +132,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "c132b458da888765884f6675e5214dd0" + "3b7b0af607ffc045bc448ad1c3d21434" ], [ "GRewrite.test_term_eq", @@ -141,7 +141,7 @@ 1, [ "@query", "true_interp" ], 0, - "fae190ae2115f0cd5144c0d3cb4b74ed" + "52f5aa5fb67e70260284cdfb2abad16c" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Goals.fst.hints b/examples/tactics/Goals.fst.hints index 82e5ebafbe2..9e1628de98a 100644 --- a/examples/tactics/Goals.fst.hints +++ b/examples/tactics/Goals.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query" ], 0, - "5c8be07d4a4a43d50d2c81df6705c89d" + "d86481029c3cc03af3b09bafdc35e36e" ], [ "Goals.elim", @@ -20,7 +20,7 @@ "refinement_interpretation_Goals_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "e633fef4e738b82ac0f4568977a264a2" + "f625a8de3741d8f52270f3ddcdb65503" ], [ "Goals.intro_sq", @@ -29,7 +29,7 @@ 1, [ "@query" ], 0, - "b69224425b5a547e354baf4f8591f36a" + "f6c73e3dccdcab9d91882bbb97679d8c" ], [ "Goals.elim", @@ -41,7 +41,7 @@ "refinement_interpretation_Goals_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "8eaa475527d0e382ae328025ef488909" + "fedc489310025c1cc2843f85f7bdc1d2" ] ] ] \ No newline at end of file diff --git a/examples/tactics/HoleBy.fst.hints b/examples/tactics/HoleBy.fst.hints index 08db3657450..ad7b55a79a0 100644 --- a/examples/tactics/HoleBy.fst.hints +++ b/examples/tactics/HoleBy.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "equation_HoleBy.x" ], 0, - "6396f4c1763eb653430cea3b73342505" + "bb9983eaa183945b18fe7da04164f931" ], [ "HoleBy.lem2", @@ -17,7 +17,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "b9397087aed67b430d97a786caa5b389" + "72a264fa7b293f072f48d5c56f56fc20" ], [ "HoleBy.uu___63", @@ -26,7 +26,7 @@ 1, [ "@query", "equation_HoleBy.x" ], 0, - "c79d1de4fc33d46c5d15d07c5484b563" + "653aa9b8719b32cdb27be2adeca76081" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Imp.fst.hints b/examples/tactics/Imp.fst.hints index 54e1d4dc577..5a25ccbf520 100644 --- a/examples/tactics/Imp.fst.hints +++ b/examples/tactics/Imp.fst.hints @@ -12,7 +12,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "8563844446f971419d06262eaeba1431" + "49440e177f64e1e2baa6be17ef51b8f8" ], [ "Imp.__proj__Add__item___0", @@ -25,7 +25,7 @@ "refinement_interpretation_Imp_Tm_refine_e6ce28c4b80443ebde698de45d7d9ff5" ], 0, - "605bb09f65754e7bef779a942e13ab3c" + "d877c0367f13487d19cae4bcede91d9c" ], [ "Imp.__proj__Add__item___1", @@ -38,7 +38,7 @@ "refinement_interpretation_Imp_Tm_refine_e6ce28c4b80443ebde698de45d7d9ff5" ], 0, - "57575136dcdda28a60caa3eddd809f62" + "b65989e30f85480c7f32786daaeafce6" ], [ "Imp.__proj__Add__item___2", @@ -51,7 +51,7 @@ "refinement_interpretation_Imp_Tm_refine_e6ce28c4b80443ebde698de45d7d9ff5" ], 0, - "b26c1cd1a183143a7800bac54dab48cb" + "9ac2cfa3028b10643e8b53ade8d65069" ], [ "Imp.__proj__Sub__item___0", @@ -64,7 +64,7 @@ "refinement_interpretation_Imp_Tm_refine_6a21b5ee6f026c7c16d0946bc061a6f1" ], 0, - "b5c1d7bc05f489f74407c393bafc6789" + "bf9b7d2c966966f7f79ebbeccee47499" ], [ "Imp.__proj__Sub__item___1", @@ -77,7 +77,7 @@ "refinement_interpretation_Imp_Tm_refine_6a21b5ee6f026c7c16d0946bc061a6f1" ], 0, - "51d261677efec3f4b997b57f59969155" + "f2a42346e4edbf2c6bdfc30d4bf8d236" ], [ "Imp.__proj__Sub__item___2", @@ -90,7 +90,7 @@ "refinement_interpretation_Imp_Tm_refine_6a21b5ee6f026c7c16d0946bc061a6f1" ], 0, - "55e0dd6668f2db34a1e5405bfdd2121d" + "87c010e3f952fd073659af20715fe65d" ], [ "Imp.__proj__Mul__item___0", @@ -103,7 +103,7 @@ "refinement_interpretation_Imp_Tm_refine_eba13340a4747cc74a458556f1746952" ], 0, - "9dac6e688ad17b65d321505da14ae133" + "439728f5af0ebc8399c20969b5611ac9" ], [ "Imp.__proj__Mul__item___1", @@ -116,7 +116,7 @@ "refinement_interpretation_Imp_Tm_refine_eba13340a4747cc74a458556f1746952" ], 0, - "b3e5ac7b8ed0b29de7d3a7d3ec7f5a74" + "b0b68a569f0b661eccfd8f7ed880ea2f" ], [ "Imp.__proj__Mul__item___2", @@ -129,7 +129,7 @@ "refinement_interpretation_Imp_Tm_refine_eba13340a4747cc74a458556f1746952" ], 0, - "e3ac5496ec9d99259dcce1621f4ca230" + "7796f5fa78cd4966fcd9773f7e7ef6ea" ], [ "Imp.__proj__Const__item___0", @@ -142,7 +142,7 @@ "refinement_interpretation_Imp_Tm_refine_01ac0c7f58b13b9a9cb14230122b0e7a" ], 0, - "60d90ab3058cb7731be86108a40014a5" + "f823d35c46f99c864086fdb274d69df3" ], [ "Imp.__proj__Const__item___1", @@ -155,7 +155,7 @@ "refinement_interpretation_Imp_Tm_refine_01ac0c7f58b13b9a9cb14230122b0e7a" ], 0, - "68b6f521dfa477bf1270881075582e26" + "37a9dec1c677c8537de3a73e5941f9e4" ], [ "Imp.size", @@ -170,7 +170,7 @@ "fuel_guarded_inversion_Imp.inst" ], 0, - "ef64e7c8d706a948629ed3b2ebc64bf8" + "2f5b545d11aba5c4db4e1bb741760d6b" ], [ "Imp.size", @@ -188,7 +188,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "0ef0509d3d38370bcfc01a1551b9a022" + "3676233e4ff93d7a3413dd85b4103252" ], [ "Imp.override", @@ -197,7 +197,7 @@ 1, [ "@query", "assumption_Imp.reg__uu___haseq" ], 0, - "5c9cc47c3469ca0dc33ddf21fdc01a57" + "0506fa355bba0b32d8019b43359c04a8" ], [ "Imp.eval'", @@ -212,7 +212,7 @@ "fuel_guarded_inversion_Imp.inst" ], 0, - "7d2598ca6f29a5190f57947de4455a98" + "a50474aeeb941d01790c0e897136fab8" ], [ "Imp.uu___68", @@ -221,7 +221,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "67570561444c8bad4be584a95345dc53" + "8862d8155947a22aa098d55c029dc7b2" ], [ "Imp.uu___69", @@ -230,7 +230,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "c15f2eab4b7546e94b742e752cbb1c28" + "ead44bb6894eeef6e4877a56f780162e" ], [ "Imp.uu___70", @@ -239,7 +239,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "c1cd0b949c70ad30c3488713f0e0ed6c" + "70b5e6fe67b0dce0bebb6501325fb204" ], [ "Imp.uu___71", @@ -248,7 +248,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "0c4ad907d8abf10cf25a89c3afcfc81d" + "571e5ff24153dd2e4cdf216c9e81a39b" ], [ "Imp.uu___72", @@ -257,7 +257,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "8ad86e2cd7aa285d5952bffb90df25e0" + "7c3b65a9c8c957c53df3e01b193b9897" ], [ "Imp.uu___73", @@ -266,7 +266,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "fe6ef93236d782c310bd3d6e5ad9741c" + "892d4378ebc9979d81397deac003d21f" ], [ "Imp.uu___74", @@ -275,7 +275,7 @@ 1, [ "@query" ], 0, - "1521a3b14fbaf944cc8f17248af7b3d7" + "bc4101a49b771d0fc301b4a3c6567078" ], [ "Imp.uu___81", @@ -284,7 +284,7 @@ 1, [ "@query" ], 0, - "60577b4518bde73ca86f812287936611" + "4ea1752d18656609eae4611b27eade03" ], [ "Imp.uu___82", @@ -293,7 +293,7 @@ 1, [ "@query" ], 0, - "8fea3c400ef37c6cf5dc36e94b0f89e0" + "441f09a98bfb613e511bbc59d3f8e7b8" ], [ "Imp.uu___83", @@ -302,7 +302,7 @@ 1, [ "@query" ], 0, - "d50c9c9e5314ad9c6eb3975b193b40f0" + "f73a4adb0e50c7e1019926539c3a70a0" ], [ "Imp.uu___84", @@ -311,7 +311,7 @@ 1, [ "@query" ], 0, - "7649d6ff8f7bb0c596a08e762cc4ee93" + "cf9fc97d699902d54015fbffb4e63026" ], [ "Imp.uu___85", @@ -323,7 +323,7 @@ "primitive_Prims.op_Multiply", "projection_inverse_BoxInt_proj_0" ], 0, - "c1a2b2c563ba626a5791f0d02032d60e" + "137d50a128d174ea958c7c79d812b027" ], [ "Imp.uu___86", @@ -335,7 +335,7 @@ "primitive_Prims.op_Multiply", "projection_inverse_BoxInt_proj_0" ], 0, - "5bfe259ab1a40ee77a4c99b2e91e4431" + "00f9ba04df2098d46a27052479e72427" ], [ "Imp.uu___87", @@ -347,7 +347,7 @@ "primitive_Prims.op_Multiply", "projection_inverse_BoxInt_proj_0" ], 0, - "e315039176476e522c0e48652e0fdcd0" + "36d2b81fd1810f57ec9c32c3b25f3572" ], [ "Imp.reg", @@ -360,7 +360,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "60531565cfeb29f1011ed5790afcb121" + "edce8fc6eab0c067613fc96996f21445" ], [ "Imp.__proj__Add__item___0", @@ -373,7 +373,7 @@ "refinement_interpretation_Imp_Tm_refine_e6ce28c4b80443ebde698de45d7d9ff5" ], 0, - "b9b92e6cad6015bffe593c307a9e07e4" + "97c5ec4dd41a15f82823dc9caca80702" ], [ "Imp.__proj__Add__item___1", @@ -386,7 +386,7 @@ "refinement_interpretation_Imp_Tm_refine_e6ce28c4b80443ebde698de45d7d9ff5" ], 0, - "d53de09aade6d9cc94555531bf75eb1c" + "6d736d5430b3414b1c33c6bab10fbafb" ], [ "Imp.__proj__Add__item___2", @@ -399,7 +399,7 @@ "refinement_interpretation_Imp_Tm_refine_e6ce28c4b80443ebde698de45d7d9ff5" ], 0, - "512a36e7b051d894dc0ac6152a2e4406" + "164c410a4e024b9c7ea2cf1eae4ee4b7" ], [ "Imp.__proj__Sub__item___0", @@ -412,7 +412,7 @@ "refinement_interpretation_Imp_Tm_refine_6a21b5ee6f026c7c16d0946bc061a6f1" ], 0, - "a22b617d5a08b555e006befd91726bcc" + "ea3851331285194a490faf4305d2f87e" ], [ "Imp.__proj__Sub__item___1", @@ -425,7 +425,7 @@ "refinement_interpretation_Imp_Tm_refine_6a21b5ee6f026c7c16d0946bc061a6f1" ], 0, - "28a5d21dbe1b241a8041b8fb93c36b65" + "a5818e7ba8574aef5adcf180cb73ee92" ], [ "Imp.__proj__Sub__item___2", @@ -438,7 +438,7 @@ "refinement_interpretation_Imp_Tm_refine_6a21b5ee6f026c7c16d0946bc061a6f1" ], 0, - "9b49906e359d37b894330793db8cdcb7" + "3b15b501810d74a1661be5ade3f530fc" ], [ "Imp.__proj__Mul__item___0", @@ -451,7 +451,7 @@ "refinement_interpretation_Imp_Tm_refine_eba13340a4747cc74a458556f1746952" ], 0, - "7a586d9ca5954894dd23e9d9b865ac00" + "52ead2d25e66414d971329b8fedee6a0" ], [ "Imp.__proj__Mul__item___1", @@ -464,7 +464,7 @@ "refinement_interpretation_Imp_Tm_refine_eba13340a4747cc74a458556f1746952" ], 0, - "28ea9cadc71323cb008749ecec1b9200" + "8563250a2d660ec49928d65ebe19fbef" ], [ "Imp.__proj__Mul__item___2", @@ -477,7 +477,7 @@ "refinement_interpretation_Imp_Tm_refine_eba13340a4747cc74a458556f1746952" ], 0, - "e9f44d40a17c4081d4c20167b48966ea" + "050280622749777faec3dca6018b54ae" ], [ "Imp.__proj__Const__item___0", @@ -490,7 +490,7 @@ "refinement_interpretation_Imp_Tm_refine_01ac0c7f58b13b9a9cb14230122b0e7a" ], 0, - "a8dfd7c13368f7e6150a0f4b3c69895e" + "605689aa445cc1be2cdb698cc3b217c8" ], [ "Imp.__proj__Const__item___1", @@ -503,7 +503,7 @@ "refinement_interpretation_Imp_Tm_refine_01ac0c7f58b13b9a9cb14230122b0e7a" ], 0, - "2f957deba6df58e8eb50884dfaf96a88" + "a8a561e7c12b68f7aaeade0345d95883" ], [ "Imp.size", @@ -518,7 +518,7 @@ "fuel_guarded_inversion_Imp.inst" ], 0, - "753ea5fbb7a9aa7701f0b1b316749201" + "5de1f1201700043dbc2febd9f1efd6ad" ], [ "Imp.size", @@ -536,7 +536,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "f26722e5f59c1e78a884c07b831a89ed" + "980386a6317bf7a4d740f8f5623f5258" ], [ "Imp.override", @@ -545,7 +545,7 @@ 1, [ "@query", "assumption_Imp.reg__uu___haseq" ], 0, - "768ad3090e20117064de3bfaac179e72" + "068d463ac9608a608fb0d98e967ca51d" ], [ "Imp.eval'", @@ -560,7 +560,7 @@ "fuel_guarded_inversion_Imp.inst" ], 0, - "2ec1b7ef5d2fd37a5a5cb71eb703c614" + "705f1865acbfdc3c2580a8ce40220826" ], [ "Imp.uu___68", @@ -569,7 +569,7 @@ 1, [ "@query" ], 0, - "1ec9e380ac8635e169a786ba75610604" + "d87459a0d2f07fb3235db99a52763925" ], [ "Imp.uu___69", @@ -578,7 +578,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "64220b2117e3b8adf7946fa03bf8bc97" + "dabb81103cd925a6bf22dc145de018b8" ], [ "Imp.uu___70", @@ -587,7 +587,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "00b96de4860dbd1d68c07c1343c2abd1" + "af16a9bdae78791068b536ea1ed7e6fa" ], [ "Imp.uu___71", @@ -596,7 +596,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "4b276429b9d303e0ae9c03bafd71ecdd" + "7194fd34bf1c7d26c6b765a77db0b053" ], [ "Imp.uu___72", @@ -605,7 +605,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "fc9ff0fecedb9d2edaf175be552b5dbf" + "94ec478e5510258a7c99fd3be032b41a" ], [ "Imp.uu___73", @@ -614,7 +614,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "9be9a7edcfdf2075c5de27661c11abb5" + "242a0924331177113ae31fd1f3a25f2b" ], [ "Imp.uu___74", @@ -623,7 +623,7 @@ 1, [ "@query" ], 0, - "647a16c63629c860fffd53cefa84c977" + "bfefbfbc0f48c08939a67ffeb76d9368" ], [ "Imp.uu___81", @@ -632,7 +632,7 @@ 1, [ "@query" ], 0, - "95f503da42a5d951b7fd64c3131244f5" + "1eb89d7b0317f5dea841571a71faafa6" ], [ "Imp.uu___82", @@ -641,7 +641,7 @@ 1, [ "@query" ], 0, - "d8424c57fc93231dd1b962fbb9bf7b8f" + "0eef31022be732a39fb92c7533be64b1" ], [ "Imp.uu___83", @@ -650,7 +650,7 @@ 1, [ "@query" ], 0, - "a2dd2f32a74418de98b15c311e70181a" + "d6b2551aaa914c6ccbbd8ff5b4589cfe" ], [ "Imp.uu___84", @@ -659,7 +659,7 @@ 1, [ "@query" ], 0, - "64451695747c2e096808cfac49a7ac3c" + "664bf641749d587c9cbde2fa27cacc5b" ], [ "Imp.uu___85", @@ -668,7 +668,7 @@ 1, [ "@query" ], 0, - "b75326c3470ece3fc4af6e48bb7f5fc4" + "f4ad55ee4d46f6cfd29a8ce88a3a391f" ], [ "Imp.uu___86", @@ -680,7 +680,7 @@ "primitive_Prims.op_Multiply", "projection_inverse_BoxInt_proj_0" ], 0, - "fa41ca082ec6d29f8166dc4fa4841379" + "764b0c7d1240afc95f1f4d986a08d00f" ], [ "Imp.uu___87", @@ -692,7 +692,7 @@ "primitive_Prims.op_Multiply", "projection_inverse_BoxInt_proj_0" ], 0, - "22e9f8d7293c2365011962a6d23ab493" + "95f79ae49c15f7b2b5b460c0d25b2269" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Inlining.fst.hints b/examples/tactics/Inlining.fst.hints index e583fd19719..7e47a12b404 100644 --- a/examples/tactics/Inlining.fst.hints +++ b/examples/tactics/Inlining.fst.hints @@ -69,7 +69,7 @@ "typing_FStar.Set.complement", "typing_FStar.Set.singleton" ], 0, - "5c11e337a76777dcb1f51ee8e64a8068" + "f381842e7274a4c22296af672f419b7d" ], [ "Inlining.create_add_1'", @@ -139,7 +139,7 @@ "typing_FStar.Set.complement", "typing_FStar.Set.singleton" ], 0, - "6f85f5ca1b484b84c25a6c034f5a2839" + "3e3b610a11c8d1ec7ea4b1760bcfa35c" ], [ "Inlining.create_add_1'", @@ -209,7 +209,7 @@ "typing_FStar.Set.complement", "typing_FStar.Set.singleton" ], 0, - "662e1c270608effd876d849ad56ee8a1" + "3a5e503b57af79fed3fe660a2927f68b" ], [ "Inlining.create_add_1'", @@ -279,7 +279,7 @@ "typing_FStar.Set.complement", "typing_FStar.Set.singleton" ], 0, - "06e8c2e10fd66d65958041fa12c2b666" + "a2dea9ba932d49ab29b9678c5af4723e" ], [ "Inlining.create_and_set", @@ -326,7 +326,7 @@ "typing_FStar.Monotonic.HyperStack.poppable" ], 0, - "4e306e049383e2c52945cb932a803932" + "f5587abeb6891a3bc1e0e8ece0d3eb76" ], [ "Inlining.create_and_set'", @@ -373,7 +373,7 @@ "typing_FStar.Monotonic.HyperStack.poppable" ], 0, - "7034a9bc9beb8347aeb3a8878a5de122" + "27be17ef251578256260727b014dcfb3" ], [ "Inlining.create_and_set'", @@ -409,7 +409,7 @@ "refinement_interpretation_Inlining_Tm_refine_eaaf1fb3627697929673d8661ada1c2c" ], 0, - "7bbb1c18187b60fc1e2178edbd675de9" + "1f3f4f75b00ba64610531e97e09787d1" ], [ "Inlining.create_and_set'", @@ -445,7 +445,7 @@ "refinement_interpretation_Inlining_Tm_refine_eaaf1fb3627697929673d8661ada1c2c" ], 0, - "7466875f730e7a20c153d893a390876b" + "c28b0007421cb3c88d8db37b3a6c4d0d" ], [ "Inlining.set_to_1", @@ -476,7 +476,7 @@ "typing_FStar.UInt32.v" ], 0, - "dbae5bf88a463c205dc149f587c52134" + "570ff4a8a618f933ff327da6f3e6eb25" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Join.fst.hints b/examples/tactics/Join.fst.hints index fcbff631b3e..1bdb9f720fc 100644 --- a/examples/tactics/Join.fst.hints +++ b/examples/tactics/Join.fst.hints @@ -23,7 +23,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "d0cf3d81693268d8c716398d97a8835a" + "7fe59ff61c022359ff26978015f65887" ], [ "Join.test1", @@ -47,7 +47,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "a67a85c195553c960257587c35135440" + "e83941800ae4a84c8b20b0f7df44f5e8" ], [ "Join.test1", @@ -71,7 +71,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "93e1bd354958774abf0be884ec7c834d" + "214af957f94c75c856b8273d8c4c5296" ], [ "Join.test1", @@ -95,7 +95,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "ddc04efff742452e6260c9883deb45e3" + "52b6f366da7b7c16b86c14a4d3a0b747" ], [ "Join.test1", @@ -119,7 +119,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "e0035548b07fdadaa9d92b86f7dda8e7" + "a107ce04601db510b4d763ee0344208a" ], [ "Join.test1", @@ -143,7 +143,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "5ce15410999a7072357d6a410870cf94" + "10547b209aa473fa5a11883a24ac8e7c" ], [ "Join.test1", @@ -167,7 +167,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "9fc294e56ebce1c3fed35ea1d95c0f16" + "e2857dc9da3235e50cf953a4da2b153a" ], [ "Join.test1", @@ -191,7 +191,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "a76febda8e925ea12132a4b7aae13e74" + "34b0cf5edfcb8d546db8a0f3ef59705b" ], [ "Join.test1", @@ -215,7 +215,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "aac61d7e86c8a2ae79d80da3dd118d84" + "e33e67f2a61545c4e5bb0d901ac00bf1" ], [ "Join.test1", @@ -239,7 +239,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "c8ad22cc09dad22fc421c2ef0a116013" + "ef5834664c0cbc17f492efe447d5e8f7" ], [ "Join.test1", @@ -263,7 +263,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "69ab298cfce754473981c8eea7fb468f" + "e9579eca76706e8cbbb4af6070958880" ], [ "Join.test1", @@ -287,7 +287,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "334f64b9e0758ea8a105beb0f446d9c5" + "3e182746e86a3b7648e41cf1597bb3bc" ], [ "Join.test1", @@ -311,7 +311,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "7029aef8eabc981cd76e2b9682365da5" + "a58b26e242228a0d1d93ab82aec7c262" ], [ "Join.test1", @@ -335,7 +335,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "65dde31650c134ea022b67d5822907f2" + "2972e9892a1ecd04f7874ee6851d45b2" ], [ "Join.test1", @@ -359,7 +359,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "8dfe87bd04ec71d8705c2f453ed16c23" + "ab4d09f10d34a6d3f9c20cbbc722c601" ], [ "Join.test1", @@ -383,7 +383,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "aa761ad5e3bf6ea41a5b2315c7f93f6d" + "f7074ea41c0e5642d3625944b7e97928" ], [ "Join.test1", @@ -407,7 +407,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "c202c771c56556edfac388eefde76998" + "894a4cbe6049a611f1b5acc6cba8e021" ], [ "Join.test1", @@ -431,7 +431,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "bece1889f3e70ab685b16b39b6999a83" + "853b5f3f113c72fbc7cdd9eacf6bf3f4" ], [ "Join.test1", @@ -455,7 +455,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "98e79077958356ff5c00dc047e0692d8" + "63d64d82eedff9062c56e64c0ab58e73" ], [ "Join.test1", @@ -479,7 +479,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "9fcdc37b5972f0c40707f04ced5619f8" + "3db93234c2a0afece795c980161208ba" ], [ "Join.test1", @@ -503,7 +503,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "a390adb8e69f71d9c108b83bc3aab6da" + "234e6ccb2e79d4d78e8637aabc98de42" ], [ "Join.test1", @@ -527,7 +527,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "a193997e296a914dd4cce20f782c3e6a" + "5143441bc05650585765f076798eb6c1" ], [ "Join.test1", @@ -551,7 +551,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "ce88206e3be295d77e1299d43c1dff03" + "f5ee2cb3d6926c35f3a658636373fc0f" ], [ "Join.test1", @@ -575,7 +575,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "c62f28e9fb74683e9bffd169d9cdcc55" + "432fa2705319dd1bddd370aa739846a4" ], [ "Join.test1", @@ -599,7 +599,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "7c447c2f80429998f87e55b1fb19d441" + "8bd379022b3b15daf3cec0b2aa746d0a" ], [ "Join.test1", @@ -623,7 +623,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "a9fa4857be8a3069b94e1af3fbbb160c" + "3991527368905c23396e6a9b2648f1f2" ], [ "Join.test1", @@ -647,7 +647,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "01def77ce3870bbc006599d99d564d76" + "368478ca642450b4db16b15596ac3c5f" ], [ "Join.test1", @@ -671,7 +671,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "3fb165207acdca23272284b7a1ab935f" + "3e8046a540edc2b901455962e340399a" ], [ "Join.test1", @@ -695,7 +695,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "357917fdcd68d30b390c2709d5c727e6" + "96676d6688ae2c76b4e4bea4e355e528" ], [ "Join.test1", @@ -719,7 +719,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "30304ba2bf7ee55f1523610361f0012d" + "aed14030b1a62d410cb95d1d7dd807a1" ], [ "Join.test1", @@ -731,7 +731,7 @@ "refinement_interpretation_Join_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "fd8836d1c961900a5e9f32524b4cb677" + "abf2f3d3d3d3553c1ba42fc591d7c091" ], [ "Join.test1", @@ -755,7 +755,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "437b56e5739a4bc0b4f0397e04cf8958" + "f32abcefee2db5c91894090e1f9f5eb1" ], [ "Join.test1", @@ -779,7 +779,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "4ba9204e0cee20af5a5d0da281f69146" + "a371ccf26dc1b7d41fbd885a8aad18aa" ], [ "Join.test1", @@ -803,7 +803,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "7c684af3b25eb5a9f0cf9a52b510d1c1" + "def8c6f851a31d0135d034dee318364e" ], [ "Join.test1", @@ -827,7 +827,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "0545f2772a86a90836dce5593779471e" + "53754952b0d3b678374b3d7d9af69509" ], [ "Join.test1", @@ -851,7 +851,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "56e3205d1f4e1774a662849ce01c41d6" + "714f50b1713dcacb8c407ccb2fff8770" ], [ "Join.test1", @@ -875,7 +875,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "085511bf562ab07d27e728b0df0d0b93" + "c4b6f819350e0a6abba6177dc198954d" ], [ "Join.test1", @@ -899,7 +899,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "97284679bf363e78ce9762b1853b3664" + "43c08b458350c6ea2dfa47938e4e27ef" ], [ "Join.test1", @@ -923,7 +923,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "973c3868353645bebec1e2e3bc407d9e" + "11e880a9af0efc8c4bc576615ab866f1" ], [ "Join.test1", @@ -947,7 +947,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "d3e2feb8c409ed4b36b9165c5aa11714" + "95b9a31424a80c7e7d3d5e63935f227f" ], [ "Join.test1", @@ -971,7 +971,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "f367328b12fa87e89fae9d8e99862cd7" + "0fed06679288b99f372fa9f3186caa2e" ], [ "Join.test1", @@ -995,7 +995,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "e88fdffc0bf85746d3f8d3b1eac458ae" + "9ccec2fb6bb0352cb2fcf812e61a6a8c" ], [ "Join.test1", @@ -1019,7 +1019,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "2d8beaec178a5456e5e896bc787964e2" + "82fa929d0d9e2bae075a6f5469e270e8" ], [ "Join.test1", @@ -1043,7 +1043,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "5cc22c57c83c87b10265fad54ddce515" + "7f6a410798effafdc2405a59c80ccf7b" ], [ "Join.test1", @@ -1067,7 +1067,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "76759e449bafbee55e6488dd01a1df19" + "606f8b4e71c6ba57085f3f76543ca1b4" ], [ "Join.test1", @@ -1091,7 +1091,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "04840ea579cadacfba3294fa61b6eac0" + "69f3b2626520f63827920caca6f8f03d" ], [ "Join.test1", @@ -1115,7 +1115,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "0ca7e88f77fdde3ba25c9457b0a13281" + "b865a5304aaba0cff4d94060338a1de7" ], [ "Join.test1", @@ -1139,7 +1139,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "8011cb41c72f0428e39ad4fb0e455665" + "1317b845c752cb2431ac52219b90e112" ], [ "Join.test1", @@ -1163,7 +1163,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "cdeb285c864c545bbad5ff55b55c7944" + "679b6aac9796f52d2d5afa2b15fefbc6" ], [ "Join.test1", @@ -1187,7 +1187,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "fc351b21bd70f90c3bb0d2fc84894552" + "afa153f07bef953fc37627b25d9f7b8c" ], [ "Join.test1", @@ -1211,7 +1211,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "eecce3a7fb58e2c322cb87ac91d1b3ea" + "b424de754e3c7e6a89ff1a1b2c2caf3d" ], [ "Join.test1", @@ -1235,7 +1235,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "2b5ad2a63b3086dece4a4b5d87ef8715" + "684f28c70b9d652bf1b2283da138ebf9" ], [ "Join.test1", @@ -1259,7 +1259,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "27912866376aead1a882533b5dfcf466" + "4697163deadbeaed5d478f98910fff32" ], [ "Join.test1", @@ -1283,7 +1283,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "252319d61d6150466bd2d4296355fc6a" + "7bd6d4f9653ecbc5bd7f76e5537c7111" ], [ "Join.test2", @@ -1307,7 +1307,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "594c67fabe9af8305e3c0a49969ce9d1" + "d4122f58fb5e48e547d1910fda4b584b" ], [ "Join.uu___63", @@ -1331,7 +1331,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "18012934dee446c27c29b447d796696b" + "76f449aa444abb4ac138d3be7b2e7ebf" ], [ "Join.implies_intro'", @@ -1348,7 +1348,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "82a065c0d47bfd3884f66c193d3df448" + "c6071878e96ad08367bd1ef3cb6a281e" ], [ "Join.tau", @@ -1367,7 +1367,7 @@ "typing_FStar.Tactics.Result.uu___is_Success", "unit_typing" ], 0, - "ed47eb759eaff2674e9427ecff01096f" + "bd40e611358d6384f50e198c60faba8b" ], [ "Join.test1", @@ -1391,7 +1391,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "1e4d1109c41b1ae80bbd5a2367413e04" + "50b5e3c58c28ed55b9ded4e8de220c93" ], [ "Join.test1", @@ -1415,7 +1415,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "f64c2b73e7d5112db04dcda8294ec814" + "72aa3e54b92687e712577323cbad02ea" ], [ "Join.test1", @@ -1439,7 +1439,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "71fe7458300be8a46bdd210e7efb9c8d" + "9cd91ddd3254467dc8097c5f5b8fa721" ], [ "Join.test1", @@ -1463,7 +1463,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "db5910fd66f7247aac306b3f62ee2fee" + "6923cff4964cc87e1ee819bcd5ad8e7c" ], [ "Join.test1", @@ -1487,7 +1487,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "87fb7779351b51c45ea3369110b078ab" + "dfa325a3b854e513f75c3a96b10af091" ], [ "Join.test1", @@ -1511,7 +1511,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "2d874f0f282cef53d490ad3300eded73" + "587c6a7540b5fa8cd36cb82a561dc339" ], [ "Join.test1", @@ -1535,7 +1535,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "072180b8272a7e619a2ae9b95bbd667b" + "54db9388ebd3dcf001c85cce72d7ac01" ], [ "Join.test1", @@ -1559,7 +1559,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "167c22e1e96736617d947d71fbb238e1" + "9761b616047d2a40d0e79eab9840ec8f" ], [ "Join.test1", @@ -1583,7 +1583,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "87593e6b6d17b12f48eebaf6857451b9" + "94c7efe8d8232dd41150c27abac03220" ], [ "Join.test1", @@ -1607,7 +1607,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "3ddc048c9773cb9aa6b46a6db2819a5c" + "c19cd19e729bc0bc7716284ae899771b" ], [ "Join.test1", @@ -1631,7 +1631,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "51fcea266a5354cbe71e02c0ccebf251" + "6188aa497b92d900050c116bda49d67f" ], [ "Join.test1", @@ -1655,7 +1655,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "8d965fbd8cbc3ae9a89554998a9b6414" + "d28831f780346623ab3687d7e7e0e5f1" ], [ "Join.test1", @@ -1679,7 +1679,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "21a1f81fecfd630447b4a97809c5cfb9" + "1e99a7d3d9222560e383727c677321a3" ], [ "Join.test1", @@ -1703,7 +1703,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "6371c03cb460a07a05f615b3c092f8db" + "101ddce9213f5e3c2769c6ccfa4c3963" ], [ "Join.test1", @@ -1727,7 +1727,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "8ed48754ef1fbfed4824f73488c9be8b" + "06d0ab2039bc55ad6f913a5fcc5e101c" ], [ "Join.test1", @@ -1751,7 +1751,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "a18bb1939d4346097693314bcb58fd70" + "cf05953b2413bda4984ef30ef0dab598" ], [ "Join.test1", @@ -1775,7 +1775,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "c790b2fe0facdb2b8b4ec4832d2ada09" + "ef12db7b133bf175f4c0806037f58172" ], [ "Join.test1", @@ -1799,7 +1799,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "7482609c0441e79099d59f1fd04681ae" + "a49a1f18660e195674a29448b07376b1" ], [ "Join.test1", @@ -1823,7 +1823,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "d96fb909ffaba5e76a7157e5f643db83" + "b626923ba15fcbe18932d8ade3c224f9" ], [ "Join.test1", @@ -1847,7 +1847,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "e85a6dbefece3364e593622a9d554d7a" + "0ffe7866212d726a28f7f20454bfaed3" ], [ "Join.test1", @@ -1871,7 +1871,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "4777b686e5d2064fd9f949b1f413e9f0" + "75d7741f91162b6fd1d95a6fe8b1a3a5" ], [ "Join.test1", @@ -1895,7 +1895,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "fe9ab7df77b4040f9ee243d690612570" + "2b12e3e686bfd3dd7bb479fd3cae796c" ], [ "Join.test1", @@ -1919,7 +1919,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "0e5b7d252f12e210fb13b091122f1a8d" + "1b47864138a89976dfef8425e1cd224f" ], [ "Join.test1", @@ -1943,7 +1943,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "eaf93899936958960bcacf62fa21d7e5" + "030fe30e33271665715cbee932919142" ], [ "Join.test1", @@ -1967,7 +1967,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "6aa501874d44f0ae878361b9460e1484" + "d4fef5a0bea275ca12ecb31c66d74067" ], [ "Join.test1", @@ -1991,7 +1991,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "c9643b98dbe87358e2725d3b4fa8b5a8" + "8f45cc333fa8039d69c822e0a45c1bd8" ], [ "Join.test1", @@ -2015,7 +2015,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "fbb7616d7a7e8d36691289b5b65ad79d" + "91e262baf2a7b738e2fc4c2f291c0a90" ], [ "Join.test1", @@ -2039,7 +2039,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "c7812a753589fd6c4d128de0095835d5" + "da9ca256eea2636d38d65ccb486d6432" ], [ "Join.test1", @@ -2063,7 +2063,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "6055a653c4393be77c452a05334d673f" + "49cbabe22f0c9cedaec21dc723215706" ], [ "Join.test1", @@ -2075,7 +2075,7 @@ "refinement_interpretation_Join_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "b2fca16108427c2830f567f602fd21be" + "0ad1d98d050405bd774a7231f14a615f" ], [ "Join.test1", @@ -2099,7 +2099,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "621b71822072eae540e5b7e723c3f230" + "9cdd82cd919af6e242ca4969ac9160e9" ], [ "Join.test1", @@ -2123,7 +2123,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "017b85195745b792be1f75760c07fdfc" + "2be7e5a23c4e7c3f40eb4c98e6978684" ], [ "Join.test1", @@ -2147,7 +2147,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "704e5518996585fb8beb95ab57b80ddf" + "546c352b63bc763baa294911ce4c5487" ], [ "Join.test1", @@ -2171,7 +2171,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "fb1ae4436705567f140cf6e9628205ff" + "64102957090c8d876a97895ea9e6291b" ], [ "Join.test1", @@ -2195,7 +2195,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "37855740b0b3419bc85c0563f7ec77d4" + "a0d2c3acb59e8c5bf58de1defe206fe9" ], [ "Join.test1", @@ -2219,7 +2219,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "2df57fdc98cfc17db2ae468771df39a1" + "ff71a354ab7f47b4590642e2f2350349" ], [ "Join.test1", @@ -2243,7 +2243,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "acf339fa6ff0f1f34963b4be6f0150df" + "4a3ec7496fd690a2d69ea65ec64b570c" ], [ "Join.test1", @@ -2267,7 +2267,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "6f0ca97c5edb391de2a85a3f3fe34441" + "97069e1bf188c13ff7914a41a2b21483" ], [ "Join.test1", @@ -2291,7 +2291,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "26c7dbb766ef88044ec29e6f4a46d3ca" + "b49fbfbadd682acb9cb6d9e3550abddf" ], [ "Join.test1", @@ -2315,7 +2315,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "ac3f2e574ea9aa2260b14c28effe7a3c" + "9930e097441373cdff6f840753e4f5c7" ], [ "Join.test1", @@ -2339,7 +2339,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "55894f33b14fed93aff99894498d64bb" + "25625afb5998262a2cc484efd8f87626" ], [ "Join.test1", @@ -2363,7 +2363,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "d73c31e6e13be34ac094e579b7271830" + "5472014bd8e46ee7c7d724a8749ebe5c" ], [ "Join.test1", @@ -2387,7 +2387,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "189f96a83d6bd1e11123d5b58f0a903e" + "cdd90de391379b6767e9ebd65ef35839" ], [ "Join.test1", @@ -2411,7 +2411,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "f10de8f7b30529ff0f79f05017910366" + "aee30fd8f745b93a700de3b9f48e19d0" ], [ "Join.test1", @@ -2435,7 +2435,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "cc88c20025c2674fd80d77a60ae1ee82" + "f8482de1ea966a52380f3edd9340d971" ], [ "Join.test1", @@ -2459,7 +2459,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "2a2db81a6c79ad4775e928ac57d0707d" + "07491eef0004baedc7a1332bcc664b20" ], [ "Join.test1", @@ -2483,7 +2483,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "4064186c7efbc0a31445a341625843cb" + "f98c0e826f45b3166f9ee872b0097766" ], [ "Join.test1", @@ -2507,7 +2507,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "4988c8e65cedc5f43dd418ba76e338ef" + "af853994f849fbbdee520992770fa50b" ], [ "Join.test1", @@ -2531,7 +2531,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "eb72610a40e959c1eda564838254733a" + "f6fad214572f4d2ac9b299403a8f70d8" ], [ "Join.test1", @@ -2555,7 +2555,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "907594f4f82dfab003abd849576d91a7" + "5b47858bd0fb1f51e3dd007ac30dd72c" ], [ "Join.test1", @@ -2579,7 +2579,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "c82f76d21823e462810a71e751fe9d83" + "185ef2b488354d529f6a2f273ba91c08" ], [ "Join.test1", @@ -2603,7 +2603,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "522484ffb3422c453d517ee48d6a1240" + "caf4120dd1f5a79e50e25308005cdb70" ], [ "Join.test1", @@ -2627,7 +2627,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "6fb5798798222b34e15c5b2c37b034ab" + "ab75638bb9bcd587f39f83f7f79e50c5" ], [ "Join.test2", @@ -2651,7 +2651,7 @@ "token_correspondence_Prims.pow2.fuel_instrumented" ], 0, - "e8078b38c57f166879fa4d1b8e3f38ef" + "fee9801deaad0eec860639c7fcc8e6c1" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Labels.fst.hints b/examples/tactics/Labels.fst.hints index 694eecb69e7..8a69df3e33a 100644 --- a/examples/tactics/Labels.fst.hints +++ b/examples/tactics/Labels.fst.hints @@ -14,7 +14,7 @@ "fuel_guarded_inversion_Prims.list" ], 0, - "19ac4a4c4cb058dc80da5c7f21822875" + "1f8205bf3ad50edc08b14e9a56801312" ], [ "Labels.uu___63", @@ -29,7 +29,7 @@ "fuel_guarded_inversion_Prims.list", "true_interp" ], 0, - "54a8bba362615e9d0d6563ae1a9bd147" + "3a26ba398f9586c64d6c7dcf5571ab8e" ], [ "Labels.uu___63", @@ -44,7 +44,7 @@ "fuel_guarded_inversion_Prims.list" ], 0, - "ddd69de50801e309bc1ac3fec8ac48f5" + "b6dddd7adc6d0e9ea21240b65cc0e090" ], [ "Labels.uu___63", @@ -59,7 +59,7 @@ "fuel_guarded_inversion_Prims.list", "true_interp" ], 0, - "6b463a7c0a98722058452a7a0634a09c" + "dc0181b559e679334a37d3eaf0a9c0c3" ] ] ] \ No newline at end of file diff --git a/examples/tactics/LemmaArgs.fst.hints b/examples/tactics/LemmaArgs.fst.hints index 7eb4d090928..5b91c5c6048 100644 --- a/examples/tactics/LemmaArgs.fst.hints +++ b/examples/tactics/LemmaArgs.fst.hints @@ -11,7 +11,7 @@ "refinement_interpretation_LemmaArgs_Tm_refine_f0496eb03f3fb51b5e4ca0d53ea58c01" ], 0, - "af4d65a9a972e304c2aaecfc33aa849f" + "f345bd5ebc4004164e6c000dd406f083" ], [ "LemmaArgs.lemma_example1", @@ -23,7 +23,7 @@ "refinement_interpretation_LemmaArgs_Tm_refine_f0496eb03f3fb51b5e4ca0d53ea58c01" ], 0, - "31df01c109cec83cac6acb39d8d6648b" + "981a335f4ef096dfe7667bba0cb0ea24" ], [ "LemmaArgs.example0", @@ -32,7 +32,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int", "true_interp" ], 0, - "89a1c7b00bd4d52b03c11c985588b842" + "82fabe767c88d61a455d4cb68cd2a2b2" ], [ "LemmaArgs.example0", @@ -47,7 +47,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "e63744dc0c5153fb30fb596f9412159b" + "a552858a3c0a709d92a078ad90e00da6" ], [ "LemmaArgs.example1", @@ -56,7 +56,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int", "true_interp" ], 0, - "8bccc061f3d2d9dbcc20db7fe97e6f77" + "133ddbf998f23c4355531b4d8fe4eb5a" ], [ "LemmaArgs.lemma_example1", @@ -65,7 +65,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "7013e7279307ff166aaa71bd5a97f41d" + "6b6829cdd8a1450a28ac05b0a0dbad56" ], [ "LemmaArgs.example0", @@ -74,7 +74,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "49c8cc943fd425a2dc0075daee1facf5" + "41ace88702319d563698318f3f18f576" ] ] ] \ No newline at end of file diff --git a/examples/tactics/MetaArgs.fst.hints b/examples/tactics/MetaArgs.fst.hints index 38e533c5828..f2e87ad1308 100644 --- a/examples/tactics/MetaArgs.fst.hints +++ b/examples/tactics/MetaArgs.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "equation_MetaArgs.test1" ], 0, - "c024e6dc4e55527d458a4142764b8983" + "9ac02aa777dba6197e5297dcc845843b" ], [ "MetaArgs.uu___64", @@ -17,7 +17,7 @@ 1, [ "@query", "equation_MetaArgs.diag" ], 0, - "921d9546de6d2a4bf66095126884d80f" + "5ae0d03c02c2cf8d03ce23c310a66349" ], [ "MetaArgs.uu___65", @@ -26,7 +26,7 @@ 1, [ "@query", "equation_MetaArgs.diag" ], 0, - "eb0b917b6c0e159dbf1c6e69aea22068" + "d90bd8101ec348ebedca688bbc9b9c9f" ], [ "MetaArgs.uu___63", @@ -35,7 +35,7 @@ 1, [ "@query", "equation_MetaArgs.test1" ], 0, - "7ae3dd3910465233cbf26bf9c1cff6b9" + "d52c3c74f0bb0f593b256403b6686fe8" ], [ "MetaArgs.same_as", @@ -52,7 +52,7 @@ "typing_FStar.Tactics.Result.uu___is_Failed" ], 0, - "4827c95893aaecc4d67d616615dcff5e" + "9499beb7277318f5a3c7cc5c6fd79558" ], [ "MetaArgs.uu___64", @@ -61,7 +61,7 @@ 1, [ "@query", "equation_MetaArgs.diag" ], 0, - "1566689958c9ddd2124ccf01284ade24" + "9d3278c00d4ea560167aa64c071ebd63" ], [ "MetaArgs.uu___65", @@ -70,7 +70,7 @@ 1, [ "@query", "equation_MetaArgs.diag" ], 0, - "5e84221ffc88db073019a165541393d9" + "e942022919a3a52575eb1d1cc43aefce" ] ] ] \ No newline at end of file diff --git a/examples/tactics/MkList.fst.hints b/examples/tactics/MkList.fst.hints index f7f8e3654ac..ec8dfe5cbb4 100644 --- a/examples/tactics/MkList.fst.hints +++ b/examples/tactics/MkList.fst.hints @@ -18,7 +18,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "09a8cf1d90918f03ff5df19d8bb126e4" + "7263325f5107a243d87cfd6d6c9ea0ae" ], [ "MkList.l2", @@ -40,7 +40,7 @@ "refinement_interpretation_FStar.List.Tot.Properties_Tm_refine_fbb3412f12fd58a91571022d7c9fa36d" ], 0, - "6c1d966ec0da10dd20f47364424f7ed2" + "217d8eb5f65eeda6c2eb8e4da1567c30" ], [ "MkList.l1", @@ -59,7 +59,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "ef2bfbfd208071627d97f1be09932ba6" + "ae02af833ded9c2d2393c1ba760ccd7e" ], [ "MkList.l2", @@ -81,7 +81,7 @@ "refinement_interpretation_FStar.List.Tot.Properties_Tm_refine_fbb3412f12fd58a91571022d7c9fa36d" ], 0, - "8c2f60946f8e29d551d5987b4076b16f" + "a5cdbba623f462795c8ac12a02bb6192" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Neg.fst.hints b/examples/tactics/Neg.fst.hints index 22e2d575883..5f555b75153 100644 --- a/examples/tactics/Neg.fst.hints +++ b/examples/tactics/Neg.fst.hints @@ -13,7 +13,7 @@ "true_interp" ], 0, - "71d4a3f0f8870a3bbcb6b3e656020e14" + "ec96439640353ed6e81c292b4cf22cfe" ], [ "Neg.c3", @@ -26,7 +26,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "f1a51a4ad2f2237b69840f19936b71d3" + "f09d48d1706aaa7b8c6b287f094d5931" ] ] ] \ No newline at end of file diff --git a/examples/tactics/NormBinderType.fst.hints b/examples/tactics/NormBinderType.fst.hints index 397b3d83af7..517953c8ed5 100644 --- a/examples/tactics/NormBinderType.fst.hints +++ b/examples/tactics/NormBinderType.fst.hints @@ -11,7 +11,7 @@ "refinement_interpretation_NormBinderType_Tm_refine_bb26061a0b65cfdbbd4fbb3aba2011c7" ], 0, - "83674fd8496da266311d04c391a997cd" + "ff617f954c7241f0fa507a2313545d7b" ], [ "NormBinderType.g", @@ -24,7 +24,7 @@ "refinement_interpretation_NormBinderType_Tm_refine_9c82b93e266cb0aa7d252a122683f7de" ], 0, - "c51e51d0742683900c50bdc09a266b6f" + "cc2f55eb57f2a469eeb16d538b87988e" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Normalization.fst.hints b/examples/tactics/Normalization.fst.hints index bef8d6767d8..2dfbbd37157 100644 --- a/examples/tactics/Normalization.fst.hints +++ b/examples/tactics/Normalization.fst.hints @@ -23,7 +23,7 @@ "typing_FStar.Reflection.Basic.lookup_typ" ], 0, - "7b1521483afe279a3e90634e1abfe199" + "3766a1494045b139da56d86ea42421a1" ], [ "Normalization.uu___63", @@ -36,7 +36,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "065cf6100542a8e1e24b22b8d5cd3310" + "54420adf0345d44e7ff5fa7f4c198259" ], [ "Normalization.uu___63", @@ -49,7 +49,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "51febb172dbd264a1feea8c372e32287" + "120a8d76252ab4ee64c59c75e7f62ff1" ], [ "Normalization.uu___64", @@ -62,7 +62,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "057b6042f3d426fcc139be5bdd99e621" + "6ea8712d03eeb9cecc789bcf52894621" ], [ "Normalization.uu___64", @@ -75,7 +75,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "2079f186ec5514f0a5d90e1bbe5073e6" + "49e49aca0bdc7acce4f57d442b580ad5" ], [ "Normalization.uu___65", @@ -90,7 +90,7 @@ "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0" ], 0, - "8713001fc9786bedca80ba8116e61c55" + "425f5f2a96dc59549c3cdb16f3ad7728" ], [ "Normalization.uu___66", @@ -103,7 +103,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "bf538ad9861b7ea7e824943fb9ba322f" + "dff47e45bbbb4615b074f6ed3428c729" ], [ "Normalization.uu___66", @@ -116,7 +116,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "e34eb2ac0d10dc1f6fde8d0390522754" + "f064a8b09b513581204cdd45137462e1" ], [ "Normalization.def_of", @@ -140,7 +140,7 @@ "typing_FStar.Reflection.Basic.lookup_typ" ], 0, - "4e92b518b2729a7dd966ca54177133eb" + "42ac540fd80a2b29a56455816a5b4aa8" ], [ "Normalization.uu___63", @@ -153,7 +153,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "fe6e40506b79caa22f81c053d88fe3f2" + "cc54bac513dfcc557e60a567c1c0a1de" ], [ "Normalization.uu___63", @@ -166,7 +166,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "9a3b47380c0ec279167eb9a83e6c53b1" + "5e75cb93143b8770a150f2316ca7d495" ], [ "Normalization.uu___64", @@ -179,7 +179,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "3da662011afe2278986306fb9656d92f" + "8fe22aae1180467566d4a79661efa528" ], [ "Normalization.uu___64", @@ -192,7 +192,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "e72659d3b24f87e65c53797cf64cc03c" + "dd4afafbff6850e8af84f9dccab5a029" ], [ "Normalization.uu___65", @@ -207,7 +207,7 @@ "primitive_Prims.op_Addition", "projection_inverse_BoxInt_proj_0" ], 0, - "2e52acd5f06a922dd4e053491b024fb8" + "91b2d639766715d2285dcff069c23abb" ], [ "Normalization.uu___66", @@ -220,7 +220,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result" ], 0, - "f5fe2d0bf262167a9908cf22ab349c78" + "678c1c785cd6b7a8cff9cfb849422390" ], [ "Normalization.uu___66", @@ -233,7 +233,7 @@ "fuel_guarded_inversion_FStar.Tactics.Result.__result", "true_interp" ], 0, - "46e64ffd406902c8d795eab940b6423a" + "a3ec7ae9b929ad6baf1fb8c9cc03c7fc" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Poly.fst.hints b/examples/tactics/Poly.fst.hints index 7b3425a5d7c..c0dd181f7f2 100644 --- a/examples/tactics/Poly.fst.hints +++ b/examples/tactics/Poly.fst.hints @@ -12,7 +12,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "383edfc3500fcfeee6dcabb3758e1650" + "3c703747fbdd382a083a2a4cdc7e4216" ], [ "Poly.lemma_div_mod", @@ -24,7 +24,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "78e37797072fdbd8228d70127e658be4" + "05548b9ad6a0e9fbad87a3f574af8011" ], [ "Poly.lemma_poly_multiply_canon", @@ -37,7 +37,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "95039eed115bb1038c3ede1cd7c0347c" + "e73d76fb186b974ab9943afba98aec94" ], [ "Poly.modulo_addition_lemma", @@ -50,7 +50,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "4beeb14782f062e521340939c5f4f588" + "6d03b863602049f1759e4cfef23c8249" ], [ "Poly.lemma_div_mod", @@ -62,7 +62,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "26b9ed2b9ed4b12650b971cea4b12dc2" + "71077b28fe38295dd1722e4a8d6aed20" ], [ "Poly.lemma_poly_multiply_canon", @@ -75,7 +75,7 @@ "projection_inverse_BoxInt_proj_0" ], 0, - "ce19bfc383b8fbd153f64ebd75b3a3bc" + "2fa66423a7b88a6a313b28473ce68f62" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Pose.fst.hints b/examples/tactics/Pose.fst.hints index 1857ad69054..85e616fa8d1 100644 --- a/examples/tactics/Pose.fst.hints +++ b/examples/tactics/Pose.fst.hints @@ -12,7 +12,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "ae1de3f0dd505326cb25bf4390d752f8" + "8bc588eddcc6d2d5df9ba237c7c507ea" ], [ "Pose.uu___63", @@ -25,7 +25,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "aa20d4e05197b0b5ab0fd731e0d99be7" + "54d7b03f1bfa49b71cb0ce152e575e32" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Postprocess.fst.hints b/examples/tactics/Postprocess.fst.hints index 48b739a89ce..f8b64137b84 100644 --- a/examples/tactics/Postprocess.fst.hints +++ b/examples/tactics/Postprocess.fst.hints @@ -8,7 +8,7 @@ 1, [ "@query", "equation_Postprocess.x" ], 0, - "cd1330b5b077c150d06674e20f90cdc6" + "3ffe51b20eb83518d717767b0c1b98f1" ], [ "Postprocess.uu___68", @@ -17,7 +17,7 @@ 1, [ "@query", "equation_Postprocess.y" ], 0, - "b20518c7359fe72b08140991b78e6eec" + "143243bed9082bfc0016e92ae8f1eef2" ], [ "Postprocess.__proj__B1__item___0", @@ -30,7 +30,7 @@ "refinement_interpretation_Postprocess_Tm_refine_17e22ae7e75398217bad910401b33530" ], 0, - "5da42b2e68cde0ac159995ce67f8ebfd" + "2eb3557ddd68cf66c61dc3696b8fe026" ], [ "Postprocess.__proj__C1__item___0", @@ -43,7 +43,7 @@ "refinement_interpretation_Postprocess_Tm_refine_60aa030648fef8e7bd28516f822e9a0c" ], 0, - "3b52e8e4ef36db2921a9fa7bb2c3fa68" + "8c17c358475ec874a1b6ee40867331cd" ], [ "Postprocess.__proj__B2__item___0", @@ -56,7 +56,7 @@ "refinement_interpretation_Postprocess_Tm_refine_a571d0930fe419c0a3557e389115132f" ], 0, - "3d4f458b6f56e10eab80fae2d6f96925" + "be1a6100b8aa52472221ea683196714c" ], [ "Postprocess.__proj__C2__item___0", @@ -69,7 +69,7 @@ "refinement_interpretation_Postprocess_Tm_refine_d350a2c0136fefb41ae2d218a2b66a7b" ], 0, - "d15454bc9c0f6d1c23b715d7ea9db7dc" + "07d279a70718290d94839becd2827e42" ], [ "Postprocess.lift", @@ -86,7 +86,7 @@ "subterm_ordering_Postprocess.C1", "typing_tok_Postprocess.A1@tok" ], 0, - "6b50979172f55c8847de4be75845969e" + "b9e5060261f46bae0c5dcdab1784fe2a" ], [ "Postprocess.lemA", @@ -101,7 +101,7 @@ "equation_with_fuel_Postprocess.lift.fuel_instrumented" ], 0, - "931de2643a1dbe2fe5f12f8166d3168f" + "0bf122e0e1775c7b1d44c9dc3ef5975f" ], [ "Postprocess.lemB", @@ -116,7 +116,7 @@ "projection_inverse_Postprocess.B1__0" ], 0, - "f591710b73201e71275e25c74fe98131" + "e261f719344fb7d901aa7023321fa3be" ], [ "Postprocess.lemC", @@ -125,7 +125,7 @@ 1, [ "@query" ], 0, - "bd5e0279eeacc732f97169f948ee59da" + "eb38f72ceb9e26639a24896e73f21971" ], [ "Postprocess.congB", @@ -138,7 +138,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "6e66c138cc729b0bb99ace313b4e1410" + "76b826c10482fd50236a582048815f8b" ], [ "Postprocess.congC", @@ -151,7 +151,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "21522b600952621445e40466cc2f9074" + "e871d2d45094c32f8822c2db660d34b6" ], [ "Postprocess.apply_feq_lem", @@ -164,7 +164,7 @@ "equation_FStar.FunctionalExtensionality.feq" ], 0, - "092d8a775efe835da648a903e883783e" + "61a1732e850d86d18ec8b70170908d0a" ], [ "Postprocess._onL", @@ -177,7 +177,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "9c08290883560a630c6106e47b3dffb1" + "e7b5593f2afe79ffe4db5585259ce846" ], [ "Postprocess.push_lifts'", @@ -196,14 +196,14 @@ "equation_FStar.Reflection.Types.typ", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v" ], 0, - "c62625d451acbd20326af2a50d67b23f" + "c0205d1908b5b27bb3450fb41670de86" ], [ "Postprocess.push_lifts'", @@ -228,7 +228,7 @@ "typing_FStar.Tactics.Result.uu___is_Success", "unit_typing" ], 0, - "5288a65dce7765805f1567c7adc8fca2" + "f6364151a941088066e9dcf905d365d1" ], [ "Postprocess.uu___67", @@ -237,7 +237,7 @@ 1, [ "@query", "equation_Postprocess.x" ], 0, - "8ba64dbaa04592b690c75e84f6bdbefb" + "c04f5f7871cfe1607d370304806b1a17" ], [ "Postprocess.uu___68", @@ -246,7 +246,7 @@ 1, [ "@query", "equation_Postprocess.y" ], 0, - "634ca61aa1e0163fbb848a1e66de261a" + "5e3bbdd1a805c38d2e4c58bcbc17022a" ], [ "Postprocess.__proj__B1__item___0", @@ -259,7 +259,7 @@ "refinement_interpretation_Postprocess_Tm_refine_17e22ae7e75398217bad910401b33530" ], 0, - "ee84d37a78a6455c2aa21c89ddc33158" + "507fcd91ee60b691f42b3fa3a31238af" ], [ "Postprocess.__proj__C1__item___0", @@ -272,7 +272,7 @@ "refinement_interpretation_Postprocess_Tm_refine_60aa030648fef8e7bd28516f822e9a0c" ], 0, - "fc5f38db5ec1de791eaf3ce3e05887bb" + "313314479aaef5e2815f4e478380b151" ], [ "Postprocess.__proj__B2__item___0", @@ -285,7 +285,7 @@ "refinement_interpretation_Postprocess_Tm_refine_a571d0930fe419c0a3557e389115132f" ], 0, - "e4267f8769a8650e564e55e8250cf29e" + "aaa015ea125b33e8ad837e9abcbaeea5" ], [ "Postprocess.__proj__C2__item___0", @@ -298,7 +298,7 @@ "refinement_interpretation_Postprocess_Tm_refine_d350a2c0136fefb41ae2d218a2b66a7b" ], 0, - "62959035456d333f9a9073c45b0bf76f" + "4cc5ee0abdfbecf774eba30996d49c85" ], [ "Postprocess.lift", @@ -315,7 +315,7 @@ "subterm_ordering_Postprocess.C1", "typing_tok_Postprocess.A1@tok" ], 0, - "ba46b89d00558aebff33482ba1171cf7" + "9ae4f28c521093dd500d2995de981e29" ], [ "Postprocess.fext", @@ -336,7 +336,7 @@ "typing_FStar.Tactics.Result.uu___is_Success", "unit_typing" ], 0, - "f8b6f0feeb5b5fbea05dbb319f9e5856" + "9be5bd818a6d7c57b02f40171d00f6f9" ], [ "Postprocess.push_lifts'", @@ -355,14 +355,14 @@ "equation_FStar.Reflection.Types.typ", "fuel_guarded_inversion_FStar.Tactics.Result.__result", "projection_inverse_FStar.Tactics.Result.Failed_a", - "projection_inverse_FStar.Tactics.Result.Failed_msg", + "projection_inverse_FStar.Tactics.Result.Failed_exn", "projection_inverse_FStar.Tactics.Result.Failed_ps", "projection_inverse_FStar.Tactics.Result.Success_a", "projection_inverse_FStar.Tactics.Result.Success_ps", "projection_inverse_FStar.Tactics.Result.Success_v" ], 0, - "719ea0b09032ee52650d152739709f5f" + "4ad19cc780c93c2d7594d1becc7dc58a" ], [ "Postprocess.push_lifts'", @@ -387,7 +387,7 @@ "typing_FStar.Tactics.Result.uu___is_Success", "unit_typing" ], 0, - "73081d7ae8b3c9a380cf8fc92d184b82" + "3a59072bbe8f49557b469350ea065748" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Printers.fst.hints b/examples/tactics/Printers.fst.hints index b9682a67866..0defe05588d 100644 --- a/examples/tactics/Printers.fst.hints +++ b/examples/tactics/Printers.fst.hints @@ -13,7 +13,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "b3c37ccd7efeff6125402d5adff9c141" + "ed4719fa34f8f21bac6a4bca5451ab5d" ], [ "Printers.__proj__A__item___0", @@ -26,7 +26,7 @@ "refinement_interpretation_Printers_Tm_refine_1a7b69b43f7b02549720ebdb7731aa7f" ], 0, - "e8c87a2ddaf0c4db5d9e110c2f1938c1" + "daa8bc96a1a8ae49dee8c6942e0873fb" ], [ "Printers.__proj__A__item___1", @@ -39,7 +39,7 @@ "refinement_interpretation_Printers_Tm_refine_1a7b69b43f7b02549720ebdb7731aa7f" ], 0, - "5f98f7301865431cdcdf01ccf18b5947" + "d2424ace1282352f3b82ef50a07b0076" ], [ "Printers.__proj__B__item___0", @@ -52,7 +52,7 @@ "refinement_interpretation_Printers_Tm_refine_c8b4b75e38b41b48b268ea0a3f90e3cd" ], 0, - "233561ae0a17a594918b7f33cd51d31c" + "38e08f31a89d36787e3a8c9eaf712716" ], [ "Printers.__proj__B__item___1", @@ -65,7 +65,7 @@ "refinement_interpretation_Printers_Tm_refine_c8b4b75e38b41b48b268ea0a3f90e3cd" ], 0, - "c543bbf0f972b3d33f04d15580465c03" + "04bd41c947ee82fac90fc023dc0465fc" ], [ "Printers.__proj__D__item___0", @@ -78,7 +78,7 @@ "refinement_interpretation_Printers_Tm_refine_3c3099d8265cd24e0a96805751c994d1" ], 0, - "13379c0d16b0f5d818c5bc65437d194c" + "9c250a24a7aadc2b15263588957e94b0" ], [ "Printers.__proj__E__item___0", @@ -91,7 +91,7 @@ "refinement_interpretation_Printers_Tm_refine_410bdfe840bb48a5ed0357e092bfc39f" ], 0, - "f6d40650a9a3d22ab61d94bfc433b9f9" + "6acf3c23059f0609b7ba6cdca1f25a43" ], [ "Printers.__proj__F__item___0", @@ -104,7 +104,7 @@ "refinement_interpretation_Printers_Tm_refine_9c3e9566abf10c7d01bd5254baeab0f0" ], 0, - "3efed01f2833b1c570f6586280559c18" + "824ce02dc5d4938c947480784cb40a45" ], [ "Printers.t1_print", @@ -119,7 +119,7 @@ "subterm_ordering_Printers.B", "subterm_ordering_Printers.E" ], 0, - "b265e0293edcfc0ce129ad38097520b1" + "4d798e164f3d16b97c2f8bf52caa786a" ], [ "Printers.uu___63", @@ -128,7 +128,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "2ea83b71dbe08420e4dd76ceed4f3b85" + "d42080a94ae7289ec12773825837c32a" ], [ "Printers.uu___64", @@ -137,7 +137,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "a651958e203d86b7315fe3c08ef4b282" + "855263855a37f3bcfbc393eb3acdc527" ], [ "Printers.uu___65", @@ -146,7 +146,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "d04d1e54c9d91911818bb52829a2a793" + "21d40896a294489262180a1cdcc70b1f" ], [ "Printers.uu___66", @@ -155,7 +155,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "d9c31e1d9ccf4c92ac676852e2fb51ae" + "69954813627c9ae5387509fd88cf6277" ], [ "Printers.uu___67", @@ -164,7 +164,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "bc38e0685db56ca669bb3d19092dc921" + "15702d2ac264d87d9fb8db0af084e0e0" ], [ "Printers.uu___68", @@ -173,7 +173,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "3c8102a31f83f9ebd8fc8696c508d3fc" + "b495121887671852ba5febd57361102e" ], [ "Printers.maplast", @@ -187,7 +187,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "00e3e31145bca3a9a4b983ad512214f2" + "f344655b9e204fcbd36fdd60966f28bc" ], [ "Printers.__proj__A__item___0", @@ -200,7 +200,7 @@ "refinement_interpretation_Printers_Tm_refine_1a7b69b43f7b02549720ebdb7731aa7f" ], 0, - "b92351d89cff55f833fb9d925714c826" + "4ab722ea9f7a49a81e296c207632613d" ], [ "Printers.__proj__A__item___1", @@ -213,7 +213,7 @@ "refinement_interpretation_Printers_Tm_refine_1a7b69b43f7b02549720ebdb7731aa7f" ], 0, - "213ccbcaf5c718d78e1a6734d78d8b24" + "1fd39d090dfcf749b4ba49c538051791" ], [ "Printers.__proj__B__item___0", @@ -226,7 +226,7 @@ "refinement_interpretation_Printers_Tm_refine_c8b4b75e38b41b48b268ea0a3f90e3cd" ], 0, - "a8107df6dcc5f2a35e8f4b5da4e57314" + "6ddbd36d0f18afab23751e4c702ee810" ], [ "Printers.__proj__B__item___1", @@ -239,7 +239,7 @@ "refinement_interpretation_Printers_Tm_refine_c8b4b75e38b41b48b268ea0a3f90e3cd" ], 0, - "e258121a63b4533ea98baecc89d7bba2" + "b8492c777a3bb17e1e976f1213065eb2" ], [ "Printers.__proj__D__item___0", @@ -252,7 +252,7 @@ "refinement_interpretation_Printers_Tm_refine_3c3099d8265cd24e0a96805751c994d1" ], 0, - "0b3df075cbfc85a4731d2b81b4047e9b" + "349f8240407810e08a76dceb1ee524b0" ], [ "Printers.__proj__E__item___0", @@ -265,7 +265,7 @@ "refinement_interpretation_Printers_Tm_refine_410bdfe840bb48a5ed0357e092bfc39f" ], 0, - "52b8b4cdc8cadc0fec69d64aca7a24d3" + "5d02632d6847a0b494fab31747e668b7" ], [ "Printers.__proj__F__item___0", @@ -278,7 +278,7 @@ "refinement_interpretation_Printers_Tm_refine_9c3e9566abf10c7d01bd5254baeab0f0" ], 0, - "3d0d69cb557bfd0231537d50108948da" + "a08e074462f43b9c9d082e9bfc643034" ], [ "Printers.t1_print", @@ -293,7 +293,7 @@ "subterm_ordering_Printers.B", "subterm_ordering_Printers.E" ], 0, - "82c41815f83019c256d42d1a6bf31b09" + "f5606eb18d19e1aa8c9f97116d213379" ], [ "Printers.uu___63", @@ -302,7 +302,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "6ec15bfecef5731b55453b49f259182b" + "44a57dbd926a072853f0d40c7aef9163" ], [ "Printers.uu___64", @@ -311,7 +311,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "4352e239fdee2af64cbc22e160fd3233" + "b59d966a7a9c920277eb6ad37ab3e503" ], [ "Printers.uu___65", @@ -320,7 +320,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "2fcae23a04fc05dc881f9a46ffc5b8a4" + "506eec8561f801f5f46b49e657048804" ], [ "Printers.uu___66", @@ -329,7 +329,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "288ad28556e478a263c8d6fce92c902b" + "fba6b999a52e12ef82c9ba945586e0ec" ], [ "Printers.uu___67", @@ -338,7 +338,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "6c9b5d44ebb2691f20eddf7e19c0ffb3" + "67e5fad1927d5a7c3a9ec84079062f26" ], [ "Printers.uu___68", @@ -347,7 +347,7 @@ 1, [ "@query", "assumption_Prims.HasEq_string" ], 0, - "2378afc8a39a398b29b5deec8863d7f4" + "54f79efbc31be371587d1e0359796c8d" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Pruning.fst.hints b/examples/tactics/Pruning.fst.hints index 0773ab338eb..6c0b6704cb6 100644 --- a/examples/tactics/Pruning.fst.hints +++ b/examples/tactics/Pruning.fst.hints @@ -23,7 +23,7 @@ "projection_inverse_FStar.Pervasives.Native.Mktuple2__2" ], 0, - "c27bfc2e34d837f6c57fa04233c1cb16" + "9aec4d672111e0f7838fcbae2d2a7659" ], [ "Pruning.uu___70", @@ -41,7 +41,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "e54ebc5791a0232b3ec9766535eadbd2" + "79c65128d15bc9c903bc30c7a4054816" ], [ "Pruning.uu___71", @@ -59,7 +59,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "dcccc7e4244e6d3673039ef8b86455c0" + "5c2d26644d02ca3745d1770857e555b7" ], [ "Pruning.f", @@ -68,7 +68,7 @@ 1, [ "@query", "primitive_Prims.op_Addition" ], 0, - "a57fc95e243eda13f872544676d64b2e" + "84d97baf8a5b6238015d34c0b3516b57" ], [ "Pruning.uu___70", @@ -86,7 +86,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "b587869e75174ff8a61434cd6692b0e3" + "c3c869059ba209b92945fa356f767a66" ], [ "Pruning.uu___71", @@ -104,7 +104,7 @@ "projection_inverse_Prims.Cons_tl", "projection_inverse_Prims.Nil_a" ], 0, - "9b8a16fa3eb1490307a227f799a1d283" + "6d5deb6f81061f0dfc01aa7bf5370e47" ] ] ] \ No newline at end of file diff --git a/examples/tactics/Raise.fst.hints b/examples/tactics/Raise.fst.hints new file mode 100644 index 00000000000..b30260edfdb --- /dev/null +++ b/examples/tactics/Raise.fst.hints @@ -0,0 +1,115 @@ +[ + "\u0000rls", [] ] \ No newline at end of file +[ + "&)\tr\u0015[njMH5q", + [ + [ + "FStar.Tactics.Types.__proj__TacticFailure__item__uu___", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "disc_equation_FStar.Tactics.Types.TacticFailure", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_FStar.Tactics.Types_Tm_refine_f49633c0c264cfe426b78eef812b39f3" + ], + 0, + "cd3b192ae39c0816e9c658419e34be83" + ] + ] +] \ No newline at end of file diff --git a/ulib/FStar.Tactics.Util.fst.hints b/ulib/FStar.Tactics.Util.fst.hints index 3c692abc984..fec1187f0b7 100644 --- a/ulib/FStar.Tactics.Util.fst.hints +++ b/ulib/FStar.Tactics.Util.fst.hints @@ -11,7 +11,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "2b72909d942762be713a1b619c1e9d5a" + "77ff2d02e72ad6f78a8d59abea25b7f4" ], [ "FStar.Tactics.Util.fold_left", @@ -23,7 +23,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "e01c243c718f1746521073c65956d210" + "d8c468baa7a1cbfe33c10842a9ffb531" ], [ "FStar.Tactics.Util.fold_right", @@ -35,7 +35,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "0f4191d6858d1568b00e603ca1eb6f09" + "518bb96723ee6b43f0e28da4e4b1311b" ], [ "FStar.Tactics.Util.filter_map_acc", @@ -53,7 +53,7 @@ "lemma_FStar.Pervasives.invertOption" ], 0, - "5c5428679b6d66c5eec7eba31453404e" + "23bdfcec6ab38fbdc2a050dbf07e60cb" ], [ "FStar.Tactics.Util.map", @@ -65,7 +65,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "b7c259d00a4b5d4d5d63fd4ecacb182a" + "10f38b8f595d681a3843ad62c792b6d2" ], [ "FStar.Tactics.Util.fold_left", @@ -77,7 +77,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "3028a15f0203380b635cd26d68be7c17" + "f78ce0f579dd1fb3e83709135ff470db" ], [ "FStar.Tactics.Util.fold_right", @@ -89,7 +89,7 @@ "disc_equation_Prims.Nil", "fuel_guarded_inversion_Prims.list" ], 0, - "10f2459089b621c62832a1b2d88a26b8" + "6993927dbe1c6da93a4a0e6ea11f57f5" ], [ "FStar.Tactics.Util.filter_map_acc", @@ -107,7 +107,7 @@ "lemma_FStar.Pervasives.invertOption" ], 0, - "42055da099f0f6a67b2474349785ca10" + "9f56f95630328343c6cf17dbb432d164" ] ] ] \ No newline at end of file diff --git a/ulib/FStar.TaggedUnion.fst.hints b/ulib/FStar.TaggedUnion.fst.hints index 5ed651aed05..eab913e65ef 100644 --- a/ulib/FStar.TaggedUnion.fst.hints +++ b/ulib/FStar.TaggedUnion.fst.hints @@ -176,7 +176,7 @@ "typing_FStar.List.Tot.Base.noRepeats" ], 0, - "c5003de13b312c63899aed7ccba7419a" + "04b388b7dc6b90965476daff1adb62eb" ], [ "FStar.TaggedUnion.field_of_tag", @@ -315,7 +315,7 @@ "typing_FStar.List.Tot.Base.noRepeats" ], 0, - "be810b2390b62625471dfe1f7c4cb81c" + "b8e015847faf7c10c47da6a24b7255b6" ], [ "FStar.TaggedUnion.tag_of_field", diff --git a/ulib/FStar.TaggedUnion.fsti.hints b/ulib/FStar.TaggedUnion.fsti.hints index 575bd2db6b5..dcd130a48bb 100644 --- a/ulib/FStar.TaggedUnion.fsti.hints +++ b/ulib/FStar.TaggedUnion.fsti.hints @@ -78,7 +78,7 @@ "typing_FStar.List.Tot.Base.noRepeats" ], 0, - "2f718061b1319eeac972d5b16ea91f27" + "4efaac49ea20b786a8161b706d83b039" ], [ "FStar.TaggedUnion.field_of_tag", @@ -159,7 +159,7 @@ "typing_FStar.List.Tot.Base.noRepeats" ], 0, - "288bf0c41249615b2f81475e59fc6bc9" + "787436daca58845dcac48a09cf1d23cf" ], [ "FStar.TaggedUnion.tag_of_field", diff --git a/ulib/FStar.Tcp.fsti.hints b/ulib/FStar.Tcp.fsti.hints index 62d3aedd412..e6834135fe8 100644 --- a/ulib/FStar.Tcp.fsti.hints +++ b/ulib/FStar.Tcp.fsti.hints @@ -13,7 +13,7 @@ "refinement_interpretation_Prims_Tm_refine_414d0a9f578ab0048252f8c8f552b99f" ], 0, - "87f723981f9c837c9dbf2d587f50daad" + "98aaacb91281ff852aca28a2b7c7a3cf" ], [ "FStar.Tcp.__proj__RecvError__item___0", @@ -27,7 +27,7 @@ "refinement_interpretation_FStar.Tcp_Tm_refine_0b16c523f4a6aeeba204a171d1e8f098" ], 0, - "cddab5aab3ce39b6b00034e7040a9984" + "7d9ee6d9c9a7aa8ada08a8712d087dfc" ], [ "FStar.Tcp.__proj__Received__item___0", @@ -40,7 +40,7 @@ "refinement_interpretation_FStar.Tcp_Tm_refine_e0e9f2a62a06f869cff002e4825e3dc6" ], 0, - "c7ffe77663d3802d73427c4bb4e9a89a" + "8aa4fa7040854303acde731255f2735d" ] ] ] \ No newline at end of file diff --git a/ulib/FStar.UInt.fst.hints b/ulib/FStar.UInt.fst.hints index b0f0091dbfe..22addf820d7 100644 --- a/ulib/FStar.UInt.fst.hints +++ b/ulib/FStar.UInt.fst.hints @@ -800,7 +800,7 @@ "well-founded-ordering-on-nat" ], 0, - "9c9c5a4c20ccf124debbab77ea76b6e5" + "6241754565298fedd638d37496c87a13" ], [ "FStar.UInt.from_vec", @@ -836,7 +836,7 @@ "well-founded-ordering-on-nat" ], 0, - "61b2d082d65d0bfb03354c2efddd110e" + "9daa56a148af0ba6140ac7ae8e8b836a" ], [ "FStar.UInt.to_vec_lemma_1", @@ -932,7 +932,7 @@ "well-founded-ordering-on-nat" ], 0, - "86fcd8934c5ac39fa8e0140731e0ab10" + "5ba63e8044d8370a869c1de7a502af2e" ], [ "FStar.UInt.inverse_aux", @@ -1373,7 +1373,7 @@ "well-founded-ordering-on-nat" ], 0, - "838565b8b4c5f1437b9e3f82e0de2b91" + "28031fe85cf5838c7517cb41ac454bd5" ], [ "FStar.UInt.append_lemma", @@ -3163,7 +3163,7 @@ "typing_FStar.UInt.from_vec", "well-founded-ordering-on-nat" ], 0, - "7d07d33abc8093ffdd25aeb21ee5364e" + "c8bf0bc72f0421c3ecc1edf207031089" ], [ "FStar.UInt.logand_le", @@ -4044,7 +4044,7 @@ "well-founded-ordering-on-nat" ], 0, - "721b0343b103ce6e63051b7499f261b9" + "789166721e343a49801a0aa4624b7f71" ], [ "FStar.UInt.logor_ge", @@ -6977,7 +6977,7 @@ "well-founded-ordering-on-nat" ], 0, - "5b3bf95c8b4e1e9f09aea346f81bc6f2" + "f9500a4711f7bd9a234d9480f2068e24" ], [ "FStar.UInt.from_vec", @@ -7011,7 +7011,7 @@ "typing_FStar.Seq.Base.length", "well-founded-ordering-on-nat" ], 0, - "5b4261b5392a0bdaead1043da731409c" + "b26860bc6362944527dc03913cfb21dc" ], [ "FStar.UInt.to_vec_lemma_1", diff --git a/ulib/FStar.WellFounded.fst.hints b/ulib/FStar.WellFounded.fst.hints index e2be35d7029..3cd74c11546 100644 --- a/ulib/FStar.WellFounded.fst.hints +++ b/ulib/FStar.WellFounded.fst.hints @@ -36,7 +36,7 @@ "subterm_ordering_FStar.WellFounded.AccIntro" ], 0, - "16190dd0353a4aca54d5327ba9223dbc" + "dd9b1d9841d0277fd0fd2397006fe77d" ], [ "FStar.WellFounded.acc_inv", @@ -73,7 +73,7 @@ "subterm_ordering_FStar.WellFounded.AccIntro" ], 0, - "11a18fd0a81622f3c0a90cb19fc1d457" + "a3888f76d787f305ffa130e4b9ca1147" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.Buffer.fst.hints b/ulib/LowStar.Buffer.fst.hints index 19c44051a2c..356508ce8ea 100644 --- a/ulib/LowStar.Buffer.fst.hints +++ b/ulib/LowStar.Buffer.fst.hints @@ -13,7 +13,7 @@ "true_interp" ], 0, - "658c92fd42b4d808f37632177d49b517" + "83a62f0d5721fb62ace85a0a3ce16429" ], [ "LowStar.Buffer.assign_list_t", @@ -28,7 +28,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "cca4064e64021c16d403772eb94011fe" + "899f6ed4840bf415f3c05230805e37ea" ], [ "LowStar.Buffer.assign_list", @@ -132,7 +132,7 @@ "unit_typing" ], 0, - "7bca5a8d081a3685a753f8386e301fe2" + "92a06d04c41dc2b12fd549f917e2ad62" ], [ "LowStar.Buffer.trivial_preorder", @@ -146,7 +146,7 @@ "true_interp" ], 0, - "ea216c065aa78fcd585da4a865993e12" + "7a86f73d9e82e74fdb6fccbb55460d3d" ], [ "LowStar.Buffer.gsub", @@ -161,7 +161,7 @@ "true_interp" ], 0, - "ccabf366292cb90c98259e7d2662e997" + "688c6edb07efa5c4403adb96e2f00f4d" ], [ "LowStar.Buffer.gsub", @@ -186,7 +186,7 @@ "typing_FStar.UInt32.v" ], 0, - "3d22a8ade1497ecf88da05f96592a071" + "ac084c2e8418fdbc71ebdaf17659359f" ], [ "LowStar.Buffer.gsub_inj", @@ -202,7 +202,7 @@ "true_interp" ], 0, - "ef2763a4d867961efad214b9809a460d" + "beb53670886c8a37c9b3bf3b3241f04a" ], [ "LowStar.Buffer.gsub_inj", @@ -231,7 +231,7 @@ "true_interp", "typing_FStar.UInt32.v" ], 0, - "5ae3327a7086f6f7aa69e1d4d82ac88a" + "523f3d7bda1cc0de60fed0a679cfe96f" ], [ "LowStar.Buffer.sub", @@ -250,7 +250,7 @@ "true_interp" ], 0, - "8499cf0c275f6c703263f19eb4b30304" + "8201731f42c47806fe3f9d0877c91747" ], [ "LowStar.Buffer.sub", @@ -285,7 +285,7 @@ "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.UInt32.v" ], 0, - "5be1a767a8ce2000839f1a69fce9fde7" + "2df994bb114d0a9835408cdcc84ac650" ], [ "LowStar.Buffer.offset", @@ -316,7 +316,7 @@ "true_interp", "typing_FStar.UInt32.v" ], 0, - "7bb5de59c607a10d9217c968f4c38cd6" + "f7a75b05932839cf315da29152ab6dab" ], [ "LowStar.Buffer.offset", @@ -356,7 +356,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "146a6f3d84f23749f6926168a91004a8" + "860060c64927da1afc3b74181ff6dad5" ], [ "LowStar.Buffer.gcmalloc", @@ -373,7 +373,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_c91c357d8b481b71bcfe70f0ece722d9" ], 0, - "e56319e1b5dd2942cbabc11243bd4526" + "061c39334fedc8e18b312d36ddd01482" ], [ "LowStar.Buffer.gcmalloc", @@ -390,7 +390,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "730059989f2057f6c14d53fd1ec0a5ac" + "ca16b9de652dfaa41a4805cb55068a4c" ], [ "LowStar.Buffer.malloc", @@ -407,7 +407,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_353217ed671579f785639196f4ac2ab0" ], 0, - "2522d1224eae7d458711e2e7ab8b4fac" + "8140bc0ef66c8779bd6f756584d91493" ], [ "LowStar.Buffer.malloc", @@ -421,7 +421,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "cfed9e94a5c0df417d13c377955efcc3" + "96c2f57a3581f6fcdf6335ec5fe98d73" ], [ "LowStar.Buffer.alloca", @@ -442,7 +442,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "04e940a95bbfb3b2a95941c8d9dfc7db" + "0cb8788e2b99aea7078c957b093a8261" ], [ "LowStar.Buffer.alloca", @@ -553,7 +553,7 @@ "typing_FStar.UInt32.v", "typing_LowStar.Buffer.lseq_of_vec" ], 0, - "7e3271fbe2f366c1fe295f70c3510950" + "57da2ef1cea852f66b8e78f3dd64d377" ], [ "LowStar.Buffer.alloca_of_list", @@ -566,7 +566,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_fdd6ab907516d1d3b973a4a3f9b40794" ], 0, - "c76e3657105da48c2bd1f39228b165fd" + "0e16d095eff505a48d84d134fcb42c45" ], [ "LowStar.Buffer.gcmalloc_of_list", @@ -579,7 +579,7 @@ "refinement_interpretation_LowStar.Buffer_Tm_refine_9dd87058574cd14a9111143cb7caaac7" ], 0, - "5939f17d30697deabed2d0052f40a3b8" + "b06872b5585ed6ce324d2e218d91239c" ], [ "LowStar.Buffer.assign_list_t", @@ -594,7 +594,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "040b5d371f45d7fd9f96bf189a68978a" + "6ded4d26a75db7e7729dfff0d01d4da6" ], [ "LowStar.Buffer.assign_list", @@ -698,7 +698,7 @@ "unit_typing" ], 0, - "0cc623c590fc6fbdc3d12342307e7847" + "c75ad91a56f5aa49f0d2b0201d8e7e27" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.BufferCompat.fst.hints b/ulib/LowStar.BufferCompat.fst.hints index 08bed5c46d9..d4a974547d4 100644 --- a/ulib/LowStar.BufferCompat.fst.hints +++ b/ulib/LowStar.BufferCompat.fst.hints @@ -14,7 +14,7 @@ "refinement_interpretation_LowStar.BufferCompat_Tm_refine_c91c357d8b481b71bcfe70f0ece722d9" ], 0, - "f40bacb6ce7e03af4ae8fbf18f98b67b" + "83d600877b9c5a183d9bc145d70bb8ec" ], [ "LowStar.BufferCompat.rcreate_mm", @@ -29,7 +29,7 @@ "refinement_interpretation_LowStar.BufferCompat_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "ea3d3634eaaa0d714430c894e7b664f7" + "eb86c9fd3b06d1cd4afa0124736d40cb" ], [ "LowStar.BufferCompat.create", @@ -44,7 +44,7 @@ "refinement_interpretation_LowStar.BufferCompat_Tm_refine_9b063033f9f8b075fbdcde91a96a63d9" ], 0, - "fa7c9814bf04fb97e9fe41408546c5fb" + "d75ef624d2d19eaa1d9ab20cb606f053" ], [ "LowStar.BufferCompat.createL", @@ -64,7 +64,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "55319219250e29efd882d0dd40b8e2f7" + "1f61ebe7eaa9ef5cd6c300298a010d77" ], [ "LowStar.BufferCompat.rcreate", @@ -77,7 +77,7 @@ "refinement_interpretation_LowStar.BufferCompat_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "ebbafe1e36e512f45508d3a50d691919" + "4225b683263489b3ceec2fcb1477bf1d" ], [ "LowStar.BufferCompat.rcreate_mm", @@ -90,7 +90,7 @@ "refinement_interpretation_LowStar.BufferCompat_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "4977bcdc61f1fbf4b75b4b5383acbbe8" + "a0f32a7efb6fa17197e0d1d085613cf3" ], [ "LowStar.BufferCompat.create", @@ -103,7 +103,7 @@ "refinement_interpretation_LowStar.BufferCompat_Tm_refine_9b063033f9f8b075fbdcde91a96a63d9" ], 0, - "9da80c26a8af74e26f6839aa9647da75" + "7394ce72896ee8cc8e6a84557a200b92" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.BufferOps.fst.hints b/ulib/LowStar.BufferOps.fst.hints index d899309acb4..49e2cc271f6 100644 --- a/ulib/LowStar.BufferOps.fst.hints +++ b/ulib/LowStar.BufferOps.fst.hints @@ -16,7 +16,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_3fe3d8508f54ae2dc29dd954960128e7" ], 0, - "bfc55499c90ce6deddc1a01e3c4ed728" + "808a61f73f850e0ac48709a1c4ad3c46" ], [ "LowStar.BufferOps.op_Star_Equals", @@ -46,7 +46,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "264ddeb3e25985784fd285794b85faac" + "5a3bdac5d6cbcc7897f0dafa11e072ef" ], [ "LowStar.BufferOps.op_Array_Access", @@ -64,7 +64,7 @@ "refinement_interpretation_LowStar.BufferOps_Tm_refine_5bc2d3af8b6b6b89753429fc786efe42" ], 0, - "1be0223fadf5f7624502154c2de41d28" + "5b377d897dd8fa95821d38277b77079f" ], [ "LowStar.BufferOps.op_Array_Assignment", @@ -82,7 +82,7 @@ "refinement_interpretation_LowStar.BufferOps_Tm_refine_f50e31f4b48141b4b7958abcf67da20e" ], 0, - "54278f69fdb83a74693758f36e62c7d7" + "84703e993681f948924cb9306baa538b" ], [ "LowStar.BufferOps.op_Bang_Star", @@ -96,7 +96,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_3fe3d8508f54ae2dc29dd954960128e7" ], 0, - "903e36301c2944e29ca92f4aa0c774f5" + "5aac5880520bc1654e87011e3c46211a" ], [ "LowStar.BufferOps.op_Star_Equals", @@ -111,7 +111,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_3fe3d8508f54ae2dc29dd954960128e7" ], 0, - "4968b488d6e6280f7d9493ce7b90db3e" + "a0bc5dc337f6378952f2c89d1df73052" ], [ "LowStar.BufferOps.blit", @@ -144,7 +144,7 @@ "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.frameOf" ], 0, - "459ef61b630112ff44ff67e7c0bd4b79" + "1f5134ff2cab720e106c09ad42352f47" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.BufferView.fst.hints b/ulib/LowStar.BufferView.fst.hints index 6566064f030..38f15a341f7 100644 --- a/ulib/LowStar.BufferView.fst.hints +++ b/ulib/LowStar.BufferView.fst.hints @@ -11,7 +11,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "cb59a75f15a287295f88591607998c47" + "0a08bb9f48b2d7fa87da0df7048d1d48" ], [ "LowStar.BufferView.__proj__View__item__get", @@ -20,7 +20,7 @@ 1, [ "@query" ], 0, - "9570ba289deb3b0c510104b57c999502" + "9000da320e20609393db85d4c4115f8d" ], [ "LowStar.BufferView.__proj__View__item__get", @@ -38,7 +38,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "f3a27f94f3c29ad6fea3cd49f475c4ee" + "3c91842f5d2f79a23187a0f379a12222" ], [ "LowStar.BufferView.__proj__View__item__put", @@ -47,7 +47,7 @@ 1, [ "@query" ], 0, - "80e32e408095b5dac5cf0fe4d31027a1" + "0c53e1c58f30ccc07bf404e01a7e6582" ], [ "LowStar.BufferView.__proj__View__item__put", @@ -70,7 +70,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "60751e32c5c509797603b00b6f7ad925" + "53543b79113e23aa076ca46962f2f3bc" ], [ "LowStar.BufferView.buffer_view", @@ -79,7 +79,7 @@ 1, [ "@query" ], 0, - "c2c880e5617ef36766a75fafebf5d7a6" + "627c3d83c5b45df8bbad29dcb5a0fa12" ], [ "LowStar.BufferView.__proj__BufferView__item__v", @@ -88,7 +88,7 @@ 1, [ "@query" ], 0, - "30fe6c520fcdc8c4a106691d55bceef2" + "e311f763ca1b11e6827922a96cd7f321" ], [ "LowStar.BufferView.__proj__BufferView__item__v", @@ -105,7 +105,7 @@ "refinement_interpretation_LowStar.BufferView_Tm_refine_7c199f5e2f4246a694d27d6ede4a8d11" ], 0, - "05367e1acbc4ec347d181dbf26040e1d" + "10d33d207b793447c31cdcb40abcf504" ], [ "LowStar.BufferView.mk_buffer_view", @@ -114,7 +114,7 @@ 1, [ "@query" ], 0, - "1b5d02dfc85d18f935389aada65122a2" + "05fc24f5e0e7641ec6cf121381afce3c" ], [ "LowStar.BufferView.mk_buffer_view", @@ -123,7 +123,7 @@ 1, [ "@query" ], 0, - "17cea6cbac27aa3eea17ceeddcc618b8" + "ff16ec156e98dc4ba86d60e73ce20712" ], [ "LowStar.BufferView.as_buffer_mk_buffer_view", @@ -132,7 +132,7 @@ 1, [ "@query" ], 0, - "578823c95204c7a6dc85e4b2a36498a8" + "9ea01bc35dda03bcce0f8ee4281f81fa" ], [ "LowStar.BufferView.as_buffer_mk_buffer_view", @@ -154,7 +154,7 @@ "refinement_interpretation_LowStar.BufferView_Tm_refine_7c199f5e2f4246a694d27d6ede4a8d11" ], 0, - "6687ec9e5ca86ad3ee058fa47438d2ea" + "29f9af29015548713e1f795c76ffe49c" ], [ "LowStar.BufferView.as_buffer_mk_buffer_view", @@ -176,7 +176,7 @@ "refinement_interpretation_LowStar.BufferView_Tm_refine_7c199f5e2f4246a694d27d6ede4a8d11" ], 0, - "22e7cc4976c0451385dc76bc816db569" + "070961a7f2dbf8746f4493d9301e69b5" ], [ "LowStar.BufferView.get_view_mk_buffer_view", @@ -185,7 +185,7 @@ 1, [ "@query" ], 0, - "35b06c29151c8fd91c460451cf1548f4" + "b0246652bb9944e9b1550340e0881dd2" ], [ "LowStar.BufferView.get_view_mk_buffer_view", @@ -207,7 +207,7 @@ "refinement_interpretation_LowStar.BufferView_Tm_refine_7c199f5e2f4246a694d27d6ede4a8d11" ], 0, - "c3243de1987f6e8589678452f8332210" + "641abfc991cf6eefd7927cb86ab91b7d" ], [ "LowStar.BufferView.get_view_mk_buffer_view", @@ -229,7 +229,7 @@ "refinement_interpretation_LowStar.BufferView_Tm_refine_7c199f5e2f4246a694d27d6ede4a8d11" ], 0, - "2a92a35cb5a8fcf6a81682a7ee3fcc5b" + "b67401d98249140892cb5e51ccdebad3" ], [ "LowStar.BufferView.length", @@ -269,7 +269,7 @@ "typing_Prims.__proj__Mkdtuple2__item___1" ], 0, - "dee3a351ab3f51f37d340e7bf32f9e3f" + "5c4ef77bd535d698bceab89d57ee8208" ], [ "LowStar.BufferView.length_eq", @@ -278,7 +278,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "2e21514b1c12b938312c812b49578229" + "bb5dc59265fe00331bb037b6631e0990" ], [ "LowStar.BufferView.length_eq", @@ -287,7 +287,7 @@ 1, [ "@query", "equation_LowStar.BufferView.length" ], 0, - "56f8b060947e175a8c6fa026040396e3" + "fb5ab4eb621e7183aa7dc23fb52b2bcd" ], [ "LowStar.BufferView.view_indexing", @@ -325,7 +325,7 @@ "typing_Prims.__proj__Mkdtuple2__item___1" ], 0, - "e35e9f4f26f71057a931c0417ae5ed0e" + "1ac338b6b0b8cf26fd3a1c36747813d2" ], [ "LowStar.BufferView.lt_leq_mul", @@ -341,7 +341,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "2502591adc819263421a484a9fbdab25" + "773ec3141a1ea095366b265469e75881" ], [ "LowStar.BufferView.split_at_i", @@ -414,7 +414,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "44299546be2975be3218ca6af552c3f9" + "7448f4317584fadf59a18f81f6d08917" ], [ "LowStar.BufferView.sel", @@ -433,7 +433,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "f15528309ca42275078c1e6f966dc7f0" + "946e00f3416c8ad90c0ca8fce6bfdbc0" ], [ "LowStar.BufferView.upd", @@ -479,7 +479,7 @@ "typing_LowStar.BufferView.get_view" ], 0, - "7dc02afac7ddd6288fc0a80c08201179" + "05c0a14bc6424dde5924d7f44f9c476b" ], [ "LowStar.BufferView.sel_upd1", @@ -487,8 +487,7 @@ 0, 1, [ - "@MaxFuel_assumption", "@MaxIFuel_assumption", - "@fuel_correspondence_Prims.pow2.fuel_instrumented", "@query", + "@MaxIFuel_assumption", "@query", "Prims_pretyping_ae567c2fb75be05905677af440075565", "bool_inversion", "data_elim_FStar.Pervasives.Native.Mktuple3", "data_elim_LowStar.BufferView.View", "data_elim_Prims.Mkdtuple2", @@ -498,7 +497,7 @@ "equation_FStar.Monotonic.HyperStack.mem", "equation_FStar.Pervasives.dfst", "equation_FStar.Pervasives.dsnd", "equation_FStar.Seq.Properties.lseq", - "equation_FStar.Seq.Properties.split", "equation_FStar.UInt.max_int", + "equation_FStar.Seq.Properties.split", "equation_FStar.UInt.min_int", "equation_FStar.UInt32.n", "equation_LowStar.Buffer.buffer", "equation_LowStar.Buffer.trivial_preorder", "equation_LowStar.BufferView.as_buffer", @@ -527,11 +526,10 @@ "lemma_FStar.Seq.Base.lemma_eq_refl", "lemma_FStar.Seq.Base.lemma_len_append", "lemma_FStar.Seq.Base.lemma_len_slice", - "lemma_FStar.UInt.pow2_values", "lemma_LowStar.Monotonic.Buffer.length_as_seq", - "primitive_Prims.op_Division", "primitive_Prims.op_LessThanOrEqual", - "primitive_Prims.op_Modulus", "primitive_Prims.op_Multiply", - "primitive_Prims.op_Subtraction", + "primitive_Prims.op_Addition", "primitive_Prims.op_Division", + "primitive_Prims.op_LessThanOrEqual", "primitive_Prims.op_Modulus", + "primitive_Prims.op_Multiply", "primitive_Prims.op_Subtraction", "proj_equation_LowStar.BufferView.View_get", "proj_equation_LowStar.BufferView.View_n", "proj_equation_LowStar.BufferView.View_put", @@ -565,7 +563,7 @@ "typing_LowStar.Monotonic.Buffer.as_seq" ], 0, - "3b78f62e925c3f50c2216211204c29d9" + "04ac5aefaabafb46f690011cff9ca0d3" ], [ "LowStar.BufferView.sel_upd2", @@ -659,7 +657,7 @@ "typing_LowStar.BufferView.split_at_i" ], 0, - "25508c6a2c286bdb74411533f7b13763" + "7a87aa2c814388ddaf1b4e9445141076" ], [ "LowStar.BufferView.sel_upd2", @@ -757,7 +755,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "84fd3f9f8d20c219af0eaf96a857a55f" + "fd8e0ff40f7e61dd85b30248fae26529" ], [ "LowStar.BufferView.sel_upd", @@ -775,7 +773,7 @@ "refinement_interpretation_LowStar.BufferView_Tm_refine_e00ebf011276c18c2a3282d5327992dd" ], 0, - "26d6842eec66fa5f5e4417d13288a840" + "6248bce1bbada59ffb40e6fc60192316" ], [ "LowStar.BufferView.sel_upd", @@ -812,7 +810,7 @@ "typing_LowStar.BufferView.get_view" ], 0, - "d7f509964a1d22d578c62ffc5419f4f3" + "162161c499f00b0efb7c61e1541dacc8" ], [ "LowStar.BufferView.upd_modifies", @@ -862,7 +860,7 @@ "typing_LowStar.BufferView.get_view" ], 0, - "3768f49d4f335c6963c39158b861b0b5" + "026edf26c39a3a0a28817c0c2f9b2be7" ], [ "LowStar.BufferView.as_seq'", @@ -917,7 +915,7 @@ "well-founded-ordering-on-nat" ], 0, - "10311dc0d54d2f814e44339afa40366d" + "747d75c21cb9c08aaf4791e5723f0f42" ], [ "LowStar.BufferView.as_seq", @@ -940,7 +938,7 @@ "typing_LowStar.BufferView.length" ], 0, - "66be1591596590413951604fc0816d53" + "d9745ed76483c599821ad3e4595bba85" ], [ "LowStar.BufferView.as_seq_sel", @@ -955,7 +953,7 @@ "typing_LowStar.BufferView.as_seq" ], 0, - "b346e6b7628d8d4a530dbf239fb5d17b" + "896ef80ab9737598219a72c1a33b2dc9" ], [ "LowStar.BufferView.as_seq_sel", @@ -1027,7 +1025,7 @@ "well-founded-ordering-on-nat" ], 0, - "9e0e1efc2b8a156b76e17c73df24bd12" + "eee18ea5e05820da107f9b9b115a6bfb" ], [ "LowStar.BufferView.get_sel", @@ -1102,7 +1100,7 @@ "typing_Prims.__proj__Mkdtuple2__item___1" ], 0, - "21204da869efe2f762953f74d24ecab2" + "516326d2fae6aaf2365996f402f31613" ], [ "LowStar.BufferView.get_sel", @@ -1182,7 +1180,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "b1d7c37c494e5aad1b1b39ea9d0eaa0b" + "13b52fb146357faf33d9be9e223a847f" ], [ "LowStar.BufferView.put_sel", @@ -1243,7 +1241,7 @@ "typing_Prims.__proj__Mkdtuple2__item___1" ], 0, - "16a606a409a67776bbd736fcdb8f09e1" + "79ac047e8e554237f275ed9b97f7315c" ], [ "LowStar.BufferView.put_sel", @@ -1328,7 +1326,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "5bd236360d130c9cd6542895bde21ad9" + "476a228bdd8b0937cdddca2db12f3f25" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.BufferView.fsti.hints b/ulib/LowStar.BufferView.fsti.hints index 112fc7730c6..23a6f93e6b5 100644 --- a/ulib/LowStar.BufferView.fsti.hints +++ b/ulib/LowStar.BufferView.fsti.hints @@ -11,7 +11,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "93e09cdccaa69fd550e860f46eb80273" + "c539e921aa23c38d8adaf1ede8b75ee5" ], [ "LowStar.BufferView.__proj__View__item__get", @@ -20,7 +20,7 @@ 1, [ "@query" ], 0, - "90e209ebf237b3b4a36e10619b9be631" + "cb07966fec3da0cf5d02ba0051c50b17" ], [ "LowStar.BufferView.__proj__View__item__get", @@ -38,7 +38,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "ebe5df0f9873b09d688932676dfac403" + "13fc29fd6b9bd454ab6eea58952e1bb7" ], [ "LowStar.BufferView.__proj__View__item__put", @@ -47,7 +47,7 @@ 1, [ "@query" ], 0, - "df55712baa9d3db28569a90df7c2b67e" + "9c801ff9668d8155a0be040a72b2f886" ], [ "LowStar.BufferView.__proj__View__item__put", @@ -70,7 +70,7 @@ "refinement_interpretation_Prims_Tm_refine_f048236b5f8051f83b495ea5eaa6127b" ], 0, - "192c082e4932f2d5857bd07f2597009f" + "0c93b62e5801365bef8bbd3dcaa1499d" ], [ "LowStar.BufferView.mk_buffer_view", @@ -79,7 +79,7 @@ 1, [ "@query" ], 0, - "6448a31c959cd41a627e9705edb38821" + "912cd374a0330d39ed173dc952bc6373" ], [ "LowStar.BufferView.as_buffer_mk_buffer_view", @@ -88,7 +88,7 @@ 1, [ "@query" ], 0, - "9f3862fde1e09950098b66f6f918f50d" + "df8bad14e5b354b2189741e15654567c" ], [ "LowStar.BufferView.get_view_mk_buffer_view", @@ -97,7 +97,7 @@ 1, [ "@query" ], 0, - "41f132e1f6ca82546975697610efa2d9" + "836c72a29bc6734922dea1d95bab3340" ], [ "LowStar.BufferView.length_eq", @@ -106,7 +106,7 @@ 1, [ "@query", "assumption_Prims.HasEq_int" ], 0, - "8184cd5309348d9b755e8fc60e20d0a9" + "532777d668202363906f98697b02ef3f" ], [ "LowStar.BufferView.sel_upd", @@ -124,7 +124,7 @@ "refinement_interpretation_LowStar.BufferView_Tm_refine_e00ebf011276c18c2a3282d5327992dd" ], 0, - "390437dc18c1dcae2780cefb829f5d68" + "d0e396af8a4473048ab84fd21607142f" ], [ "LowStar.BufferView.as_seq_sel", @@ -138,7 +138,7 @@ "typing_LowStar.BufferView.as_seq" ], 0, - "57b7988576ce43d21966f97525c46232" + "168cc571df4ae9a37e0fc35dfc54ab74" ], [ "LowStar.BufferView.get_sel", @@ -195,7 +195,7 @@ "typing_Prims.__proj__Mkdtuple2__item___1" ], 0, - "f24b78caadd1d56f8cc629096d31f4bd" + "6f89dfb5243e8ec07a3b1aaa5ac536a2" ], [ "LowStar.BufferView.put_sel", @@ -249,7 +249,7 @@ "typing_Prims.__proj__Mkdtuple2__item___1" ], 0, - "0c9e163a60f3ee1fe444316693e1b7a3" + "6cd97ff1b8b2e595f39ed7428642b51a" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.ImmutableBuffer.fst.hints b/ulib/LowStar.ImmutableBuffer.fst.hints index a83f0344854..cbb55184ecb 100644 --- a/ulib/LowStar.ImmutableBuffer.fst.hints +++ b/ulib/LowStar.ImmutableBuffer.fst.hints @@ -14,7 +14,7 @@ "lemma_FStar.Seq.Base.lemma_eq_refl" ], 0, - "0eda22076aa4025a7099b9525287b352" + "883963e7e7022667165f4acd73e4ee6d" ], [ "LowStar.ImmutableBuffer.igcmalloc", @@ -49,7 +49,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "97bd5babfb0185e5d51f892d5eb8ae15" + "dff2bce9e61a7cc77c895970ec90e5cd" ], [ "LowStar.ImmutableBuffer.igcmalloc_of_list", @@ -81,7 +81,7 @@ "typing_LowStar.Monotonic.Buffer.as_seq" ], 0, - "a331833ebbd703befde8733740c937ea" + "abc4661472550cf09b2c6650ba1f5ef3" ], [ "LowStar.ImmutableBuffer.witness_contents", @@ -106,7 +106,7 @@ "typing_LowStar.Monotonic.Buffer.as_seq" ], 0, - "c06727742d584eae8c4fc5af7264c2c5" + "3ca49efea860ca47f1bb1015c13f0b71" ], [ "LowStar.ImmutableBuffer.recall_contents", @@ -126,7 +126,7 @@ "typing_LowStar.Monotonic.Buffer.as_seq" ], 0, - "9e8ab334f362a7f6d3d9a79294f1e249" + "9640cee45456d6087acc93585666d0ed" ], [ "LowStar.ImmutableBuffer.immutable_preorder", @@ -141,7 +141,7 @@ "lemma_FStar.Seq.Base.lemma_eq_refl" ], 0, - "6ccf1203091eff9ec71958c87c40f74f" + "b495bf67871763752ad175ce50a5622f" ], [ "LowStar.ImmutableBuffer.igsub", @@ -150,7 +150,7 @@ 1, [ "@query" ], 0, - "08caa183c915ae92afea4e360705a787" + "867760e37eeb7f7942c2f2ec0ba02af9" ], [ "LowStar.ImmutableBuffer.igsub", @@ -181,7 +181,7 @@ "typing_FStar.Seq.Base.slice", "typing_FStar.UInt32.v" ], 0, - "9b15a8b3c8de36013565300274e9dff4" + "3a9f80cf087d9761b0ea2e360a1c66e4" ], [ "LowStar.ImmutableBuffer.igsub_inj", @@ -190,7 +190,7 @@ 1, [ "@query" ], 0, - "4d31a3f79dfa64322df226fde85a2519" + "af4d2b40aca0c8aa17f9aeea56e1d951" ], [ "LowStar.ImmutableBuffer.igsub_inj", @@ -223,7 +223,7 @@ "typing_FStar.UInt.fits", "typing_FStar.UInt32.v" ], 0, - "d5d7eba573a3374b75b24e0fa84ca5e7" + "b3fb661cf839cfe4973e0ca325cac7ce" ], [ "LowStar.ImmutableBuffer.isub", @@ -232,7 +232,7 @@ 1, [ "@query" ], 0, - "36d51a0277214fd5a55c17b642e9f5ca" + "83e337d1df607b81aec11787a0b7156e" ], [ "LowStar.ImmutableBuffer.isub", @@ -278,7 +278,7 @@ "typing_FStar.UInt32.v" ], 0, - "9ce86a75a287975905de432402d3af72" + "abd0d6e0c57b3757dd63e2cd1a6d96db" ], [ "LowStar.ImmutableBuffer.ioffset", @@ -287,7 +287,7 @@ 1, [ "@query" ], 0, - "9873d84a3bb59c52341bbe49b7bfd819" + "f91aa02446685aa3e15fc2177c830e95" ], [ "LowStar.ImmutableBuffer.ioffset", @@ -334,7 +334,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "46873b1f620ed2a0cd834f1f7bb58350" + "fb1a265a759803ff7908a66de6f2f7ca" ], [ "LowStar.ImmutableBuffer.igcmalloc", @@ -355,7 +355,7 @@ "typing_LowStar.Monotonic.Buffer.length" ], 0, - "ca7e141a9564c1291e212b562685e5ea" + "942e2628b97bcd5c32e27844d4a037d0" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.Monotonic.Buffer.fst.hints b/ulib/LowStar.Monotonic.Buffer.fst.hints index 5a43ffa5b63..0ab6504eae9 100755 --- a/ulib/LowStar.Monotonic.Buffer.fst.hints +++ b/ulib/LowStar.Monotonic.Buffer.fst.hints @@ -3108,7 +3108,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "6352db5f1b87fc20aa249bdc933f12ee" + "de200164e7a8eb75dca48d7fe1ea455e" ], [ "LowStar.Monotonic.Buffer.loc_pairwise_disjoint_aux", @@ -3123,7 +3123,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "7c558a6156418146c0bf044d76244316" + "4f55576d519ba650d81ff4071fa5b789" ], [ "LowStar.Monotonic.Buffer.loc_disjoint_sym", @@ -4594,6 +4594,67 @@ 0, "a07528224428180c0fa8df69252dfc44" ], + [ + "LowStar.Monotonic.Buffer.ralloc_post_fresh_loc", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", + "Prims_pretyping_f537159ed795b314b4e58c260361ae86", "bool_inversion", + "equation_FStar.HyperStack.ST.is_eternal_region", + "equation_FStar.HyperStack.ST.mreference", + "equation_FStar.HyperStack.ST.ralloc_post", + "equation_FStar.Monotonic.HyperHeap.hmap", + "equation_FStar.Monotonic.HyperStack.contains", + "equation_FStar.Monotonic.HyperStack.frameOf", + "equation_FStar.Monotonic.HyperStack.is_eternal_color", + "equation_FStar.Monotonic.HyperStack.is_eternal_region", + "equation_FStar.Monotonic.HyperStack.is_tip", + "equation_FStar.Monotonic.HyperStack.is_wf_with_ctr_and_tip", + "equation_FStar.Monotonic.HyperStack.live_region", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.Monotonic.HyperStack.mreference", + "equation_FStar.Monotonic.HyperStack.unused_in", + "equation_FStar.Monotonic.HyperStack.upd", "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.fresh_loc", + "equation_LowStar.Monotonic.Buffer.loc_addresses", + "equation_Prims.eqtype", + "fuel_guarded_inversion_FStar.Monotonic.HyperStack.mreference_", + "function_token_typing_FStar.Monotonic.Heap.heap", + "function_token_typing_FStar.Monotonic.HyperHeap.rid", + "function_token_typing_FStar.UInt32.n", "int_inversion", + "lemma_FStar.Map.lemma_ContainsDom", + "lemma_FStar.Map.lemma_InDomUpd1", "lemma_FStar.Map.lemma_SelUpd1", + "lemma_FStar.Monotonic.Heap.lemma_upd_contains", + "lemma_FStar.Monotonic.HyperStack.lemma_mk_mem__projectors", + "lemma_LowStar.Monotonic.Buffer.mreference_live_loc_not_unused_in", + "lemma_LowStar.Monotonic.Buffer.mreference_unused_in_loc_unused_in", + "primitive_Prims.op_AmpAmp", "primitive_Prims.op_BarBar", + "primitive_Prims.op_LessThanOrEqual", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_FStar.Pervasives.Native.Mktuple3__1", + "projection_inverse_FStar.Pervasives.Native.Mktuple3__2", + "projection_inverse_FStar.Pervasives.Native.Mktuple3__3", + "refinement_interpretation_FStar.HyperStack.ST_Tm_refine_003cbb363565c5358e7ed8a8d7dba6d4", + "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", + "refinement_interpretation_FStar.StrongExcludedMiddle_Tm_refine_94f72bfda5e23ac3960136c8bc3f958c", + "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_5162887c6054b4734f59cfb79dd5cf2f", + "typing_FStar.Map.contains", "typing_FStar.Map.sel", + "typing_FStar.Map.upd", "typing_FStar.Monotonic.Heap.contains", + "typing_FStar.Monotonic.Heap.unused_in", + "typing_FStar.Monotonic.Heap.upd", + "typing_FStar.Monotonic.HyperStack.as_ref", + "typing_FStar.Monotonic.HyperStack.frameOf", + "typing_FStar.Monotonic.HyperStack.get_hmap", + "typing_FStar.Monotonic.HyperStack.get_rid_ctr", + "typing_FStar.Monotonic.HyperStack.get_tip", + "typing_FStar.StrongExcludedMiddle.strong_excluded_middle" + ], + 0, + "aebb2a23abdb1dae83282d87b9b0c008" + ], [ "LowStar.Monotonic.Buffer.disjoint_neq", 1, @@ -4679,7 +4740,7 @@ "typing_LowStar.Monotonic.Buffer.ubuffer___3674" ], 0, - "5068c4e477d2408f214093aabba35b1d" + "6a7a5365b1782ce809bde15e79b0641a" ], [ "LowStar.Monotonic.Buffer.includes_live", @@ -4785,7 +4846,7 @@ "typing_LowStar.Monotonic.Buffer.ubuffer___3674" ], 0, - "fe3df58fa5dbb63e9067ffcac82d67d0" + "a012202c6095285ecf4f04e783a84dfb" ], [ "LowStar.Monotonic.Buffer.includes_frameOf_as_addr", @@ -4805,7 +4866,7 @@ "typing_LowStar.Monotonic.Buffer.g_is_null" ], 0, - "10fd80559abfcbe59906d4c69d38766b" + "ffb7c1bb6ebed293cab7b6f4b68ccd09" ], [ "LowStar.Monotonic.Buffer.deref", @@ -4819,7 +4880,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_3fe3d8508f54ae2dc29dd954960128e7" ], 0, - "2ebec9d9b8be5d0c31c8b002910e5954" + "aa0111d5e32fec0c0a6e183a2a2acb5f" ], [ "LowStar.Monotonic.Buffer.pointer_distinct_sel_disjoint", @@ -4833,7 +4894,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_3fe3d8508f54ae2dc29dd954960128e7" ], 0, - "1e46094d012b7b601f16ee80f9a9f3e5" + "454b45b036236d67905a41ab394fc702" ], [ "LowStar.Monotonic.Buffer.pointer_distinct_sel_disjoint", @@ -4953,7 +5014,7 @@ "typing_LowStar.Monotonic.Buffer.uu___is_Null", "unit_typing" ], 0, - "3242cb3b777babc97de93626e8ca42fa" + "6617aa247919e9d01607d7f5a2668f2a" ], [ "LowStar.Monotonic.Buffer.is_null", @@ -4979,7 +5040,7 @@ "typing_FStar.Monotonic.HyperStack.get_hmap" ], 0, - "1a18a0bedb2deaf0eee707757f987afe" + "2612cd3b34bc5ef7b0d066a2aeb19554" ], [ "LowStar.Monotonic.Buffer.msub", @@ -4992,7 +5053,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_fe6abc62014457623ceb986560f36c17" ], 0, - "9ffc8d3ed389379841fe8dbc3f67d9b3" + "f1a66d29ed83ffa0f0a6f80941516335" ], [ "LowStar.Monotonic.Buffer.msub", @@ -5071,7 +5132,7 @@ "typing_LowStar.Monotonic.Buffer.length", "unit_typing" ], 0, - "51f81b43a6993475d3236a6c53ee46a1" + "dd03b033969a7a9af64c1f61da8b57eb" ], [ "LowStar.Monotonic.Buffer.moffset", @@ -5097,7 +5158,7 @@ "typing_FStar.UInt32.v" ], 0, - "deb6b1b9991b4e34b50d3f9495c16507" + "893058c15cc94c6cf06286647c3a5e6f" ], [ "LowStar.Monotonic.Buffer.moffset", @@ -5173,7 +5234,7 @@ "typing_LowStar.Monotonic.Buffer.length", "unit_typing" ], 0, - "77b468ea45f9ae94fc46e47aaa2bbd42" + "1c41e4331de0c5f4b9997cf41cf559b4" ], [ "LowStar.Monotonic.Buffer.index", @@ -5191,7 +5252,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_5bc2d3af8b6b6b89753429fc786efe42" ], 0, - "ab0c351ea3e27260670592090c0b46d0" + "0e8e1df5d81503eb54aa3fd6ce058e37" ], [ "LowStar.Monotonic.Buffer.index", @@ -5254,7 +5315,7 @@ "typing_LowStar.Monotonic.Buffer.len", "unit_typing" ], 0, - "826cc10b3818c55b41ad454266a65627" + "166133d3866b10f49cc676ca4a55ffbd" ], [ "LowStar.Monotonic.Buffer.g_upd_seq", @@ -5322,7 +5383,7 @@ "typing_LowStar.Monotonic.Buffer.length", "unit_typing" ], 0, - "db1debaa83be33bf944f1a185ea7eb4d" + "ac53c6ac1c2433804d1a8bf57ac52689" ], [ "LowStar.Monotonic.Buffer.g_upd_seq_as_seq", @@ -5504,7 +5565,7 @@ "unit_typing" ], 0, - "f6da8186133744187f697309a68c2e91" + "651ba1b0671dd36bc6dd9b4f98039b68" ], [ "LowStar.Monotonic.Buffer.g_upd", @@ -5513,7 +5574,7 @@ 1, [ "@query", "lemma_LowStar.Monotonic.Buffer.length_as_seq" ], 0, - "f2ee2223d0138612fd6e495c923a569c" + "7d7e44d093f9178a90629513bd9f12e5" ], [ "LowStar.Monotonic.Buffer.g_upd", @@ -5533,7 +5594,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "02a276b941d01d83aa4520e5ed1879bf" + "5dcb0230be196a0cf43c61f17a190128" ], [ "LowStar.Monotonic.Buffer.upd'", @@ -5551,7 +5612,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_f50e31f4b48141b4b7958abcf67da20e" ], 0, - "6c4bad093314c491c6bb482d93235e3f" + "13d860f4a16be8c937db402116a728f2" ], [ "LowStar.Monotonic.Buffer.upd'", @@ -5633,7 +5694,7 @@ "typing_LowStar.Monotonic.Buffer.length", "unit_typing" ], 0, - "9c04b32d35804d52aa778c2ee8b2da3a" + "c7662b1eead1f728178d6803960a5320" ], [ "LowStar.Monotonic.Buffer.upd", @@ -5659,7 +5720,7 @@ "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.as_seq" ], 0, - "4deb75b610dc119de948fdcf93c6f23b" + "8f30bea01c13f3296368deec88251ee2" ], [ "LowStar.Monotonic.Buffer.recallable", @@ -5682,7 +5743,7 @@ "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87" ], 0, - "2d7950c45ecf2cce6f318bb60227a990" + "bb658050993855b4ae5671739505c5a7" ], [ "LowStar.Monotonic.Buffer.recallable_null", @@ -5698,7 +5759,7 @@ "typing_LowStar.Monotonic.Buffer.mnull" ], 0, - "e0cf337d98729b27c1ec1c9296a54e79" + "de9877c9ef7c1587282d3ed81cfa5a29" ], [ "LowStar.Monotonic.Buffer.recallable_includes", @@ -5783,7 +5844,7 @@ "typing_LowStar.Monotonic.Buffer.ubuffer___3674" ], 0, - "a1e1eb115e16fd5c6b594c64fb494dea" + "9206d7a10e051b837a945a277a328495" ], [ "LowStar.Monotonic.Buffer.recall", @@ -5838,7 +5899,7 @@ "typing_LowStar.Monotonic.Buffer.g_is_null" ], 0, - "dbb081ad8f15ea7d849d9d5d82be8787" + "bdbc5e3dbd8d7ff1b383ce1bf7650444" ], [ "LowStar.Monotonic.Buffer.lemma_stable_on_rel_is_stable_on_rrel", @@ -5903,7 +5964,7 @@ "typing_LowStar.Monotonic.Buffer.uu___is_Buffer", "unit_typing" ], 0, - "3a05774a0e6e48528df6a822b549c1ca" + "ce2f4f71b84d0d2d010e38f1ad9dee9e" ], [ "LowStar.Monotonic.Buffer.witness_p", @@ -5968,7 +6029,7 @@ "typing_LowStar.Monotonic.Buffer.g_is_null", "unit_typing" ], 0, - "d7ebba6a94a8f6a8214f5f4de51b3395" + "81be212fa6a683fa53d09fb4267c2d63" ], [ "LowStar.Monotonic.Buffer.recall_p", @@ -5997,7 +6058,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_7afb7dd10fac90332be2f11458c69dad" ], 0, - "4f7cdcc2ba4f4b6ad63125e250daee46" + "b306dd50997f454e2c64243f24280aa5" ], [ "LowStar.Monotonic.Buffer.freeable", @@ -6020,7 +6081,7 @@ "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87" ], 0, - "efc85f5d912cf2a7b29b463232c28776" + "ed8ab412c5ee22fd55a6e1632892c6f5" ], [ "LowStar.Monotonic.Buffer.free", @@ -6115,7 +6176,7 @@ "typing_LowStar.Monotonic.Buffer.loc_addresses" ], 0, - "8566fc4973b753579c8dc62c56c5942f" + "e2b44df8083060f71d80bfac207c9819" ], [ "LowStar.Monotonic.Buffer.freeable_length", @@ -6136,7 +6197,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "488651d504e70037e51c017e0f1628b1" + "efe1caedabac35ba42ba9c8fc1db8c7d" ], [ "LowStar.Monotonic.Buffer.freeable_disjoint", @@ -6148,7 +6209,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "5db588549111df3976b767efcfb5296e" + "55948cf7dec0adac3ff13554a3a82eb7" ], [ "LowStar.Monotonic.Buffer.freeable_disjoint", @@ -6234,7 +6295,7 @@ "typing_LowStar.Monotonic.Buffer.ubuffer___3674" ], 0, - "38b2eed02dae438de26433ea06be67fc" + "d3d04cc05ef870eb1ba10cfc0a0ceac6" ], [ "LowStar.Monotonic.Buffer.freeable_disjoint'", @@ -6260,7 +6321,7 @@ "typing_LowStar.Monotonic.Buffer.frameOf" ], 0, - "48ec37a33f2c3a802fe7e776e98f003a" + "cfd0976bb58ec6f2962fdce11387762d" ], [ "LowStar.Monotonic.Buffer.alloc_heap_common", @@ -6399,7 +6460,7 @@ "typing_LowStar.Monotonic.Buffer.srel_to_lsrel", "unit_typing" ], 0, - "3c8020e01cfabd9880f301a0ba1e8443" + "de0ed71c68497519fa3d91a1fa43cc92" ], [ "LowStar.Monotonic.Buffer.mgcmalloc", @@ -6416,7 +6477,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "69b68e6eb6ea0606310252710dfe224c" + "609bfbc0be2efe52498c0b5ec438bfad" ], [ "LowStar.Monotonic.Buffer.mgcmalloc", @@ -6441,7 +6502,7 @@ "typing_FStar.UInt32.v" ], 0, - "540c64f51fb60702c2e74447ae435abc" + "ea08be49f04c47c3fa91cbf453ad41ee" ], [ "LowStar.Monotonic.Buffer.mmalloc", @@ -6455,7 +6516,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "e2c077fed4ce350b6d51dc4bfe893ff8" + "3cc32ffa287ef8ec890389456f0ee312" ], [ "LowStar.Monotonic.Buffer.mmalloc", @@ -6504,7 +6565,7 @@ "unit_typing" ], 0, - "17ce1c9bd0a9d9d029555ce0b1d7f7a7" + "8152ae49800b341c931b691a612ce4c9" ], [ "LowStar.Monotonic.Buffer.malloca", @@ -6522,7 +6583,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "fe9bc4204ec9e104966a150b58160454" + "e5a5ab2f7d9049932b43fd894ed48ba3" ], [ "LowStar.Monotonic.Buffer.malloca", @@ -6632,7 +6693,7 @@ "typing_FStar.UInt.fits", "typing_FStar.UInt32.v" ], 0, - "ffc056b6f42ce837a1ed2af45c60b596" + "e8faaafd40a8136575cd89675d67aff3" ], [ "LowStar.Monotonic.Buffer.malloca_of_list", @@ -6756,7 +6817,7 @@ "typing_FStar.UInt.fits", "typing_FStar.UInt.max_int" ], 0, - "912a89acfe3f9a836d058a6c8bab897e" + "e2528339407acf24af6f7e5b4ccbcfea" ], [ "LowStar.Monotonic.Buffer.mgcmalloc_of_list", @@ -6870,7 +6931,7 @@ "typing_LowStar.Monotonic.Buffer.g_is_null" ], 0, - "e486bbd75858435c830985ab7bdd35e6" + "5f268d2fe77ead09bce8a0f6fe9fb162" ], [ "LowStar.Monotonic.Buffer.blit", @@ -6903,7 +6964,7 @@ "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.frameOf" ], 0, - "49eac72d8b6dbe5014024130b9f3f0f2" + "275da5a02ec9e1327e088e9aa986b717" ], [ "LowStar.Monotonic.Buffer.blit", @@ -7038,7 +7099,7 @@ "unit_typing" ], 0, - "d5297d352f82d899ea5e31c60dea88a9" + "94209567c21dc4e0caef53b6e34990af" ], [ "LowStar.Monotonic.Buffer.coerce", @@ -7050,7 +7111,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_de9aeb070296eed20d879692d0254af0" ], 0, - "0d624ef779b7dfd691051d0e39ac77ba" + "ca70189dbb6c991a1977db9d8591ba7e" ], [ "LowStar.Monotonic.Buffer.cloc_cls", @@ -7059,7 +7120,7 @@ 1, [ "@query" ], 0, - "3a2fb25ae6c84661d70fd3c3efe985b2" + "11df661b5bbe1438813975862088a187" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc", @@ -7077,7 +7138,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "ed735358e4ff6c17b64b24c2d2bf2478" + "f17446653c8b5a93b12a52ee0d8b1c29" ], [ "LowStar.Monotonic.Buffer.loc_of_cloc", @@ -7095,7 +7156,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "63d62ac3cf828e2e70e205380766b267" + "1a57e94a19f59c64b84c5a0a12e14097" ], [ "LowStar.Monotonic.Buffer.loc_of_cloc_of_loc", @@ -7115,7 +7176,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "61a4216a5e3082070b31820f5d597887" + "bb43d89d3f164dd2c5a0c06df039bffc" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_of_cloc", @@ -7135,7 +7196,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "d30177f7df1882829eb280affe09b034" + "f09f39043c2b111b6d3d8349bbb3952b" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_none", @@ -7155,7 +7216,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "688a79e5044d36072551caf648b70481" + "6510cefa52227e7a7df57ee4d9a55ed8" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_union", @@ -7176,7 +7237,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "0cf5f52edc554a064b576b5363e79f8b" + "713cc1c148a7a0c09889ccbc5140226e" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_addresses", @@ -7188,7 +7249,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "a7878efe310bd409ad04f9b0e08afafa" + "8c36b6c65318dc585ae2fda3edcbeb63" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_addresses", @@ -7200,7 +7261,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "580ec04e7dfe6635e82de84355496338" + "2e0ea6c726ec23d1b159b8862ea7d0bc" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_addresses", @@ -7220,7 +7281,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "e015a0f253b6fd33a102036b33a598c2" + "9be2a09cd18f7ae1d74598351216e8b0" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_regions", @@ -7240,7 +7301,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "623603c09d80e16acc2805bc20be8708" + "d2f1e44092d7832206492bba2cb09b69" ], [ "LowStar.Monotonic.Buffer.loc_includes_to_cloc", @@ -7260,7 +7321,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "76fe34136aacb734c1193bce3b7169e1" + "dc8abc954611a1c629195d6b38f57444" ], [ "LowStar.Monotonic.Buffer.loc_disjoint_to_cloc", @@ -7280,7 +7341,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "24319da70774b0a23eecc11b7b79753b" + "05e9f2982c56b17695612b94d78545f0" ], [ "LowStar.Monotonic.Buffer.modifies_to_cloc", @@ -7300,7 +7361,7 @@ "projection_inverse_FStar.ModifiesGen.Cls_aloc" ], 0, - "ad38badc01ba48e156bf3e7e87b8fd35" + "af6e47b5e25d0ad7eaa9b5908d8fdbfb" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.Monotonic.Buffer.fsti.hints b/ulib/LowStar.Monotonic.Buffer.fsti.hints index fa9f26bb4b6..a1b8a7576cf 100644 --- a/ulib/LowStar.Monotonic.Buffer.fsti.hints +++ b/ulib/LowStar.Monotonic.Buffer.fsti.hints @@ -1,5 +1,5 @@ [ - "\u0016Vs\u001fM\u0001˅\u0000_\u001e", + "\u0001B`:D::*", [ [ "LowStar.Monotonic.Buffer.live_is_null", @@ -641,7 +641,7 @@ "subterm_ordering_Prims.Cons" ], 0, - "e94382753eeeef8a61e847eaa4fa681d" + "b529e131f6526b2f236fbb7222a7e801" ], [ "LowStar.Monotonic.Buffer.loc_pairwise_disjoint_aux", @@ -655,7 +655,7 @@ "fuel_guarded_inversion_Prims.list", "subterm_ordering_Prims.Cons" ], 0, - "1e377a6a79d4a937891d2846b9a2341b" + "0f60245b64bc5724d1313cf1a6ff2acd" ], [ "LowStar.Monotonic.Buffer.loc_disjoint_sym'", @@ -963,6 +963,66 @@ 0, "2d8bccbcb57db2a01346ef76c29b1826" ], + [ + "LowStar.Monotonic.Buffer.ralloc_post_fresh_loc", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", + "Prims_pretyping_f537159ed795b314b4e58c260361ae86", "bool_inversion", + "equation_FStar.HyperStack.ST.is_eternal_region", + "equation_FStar.HyperStack.ST.mreference", + "equation_FStar.HyperStack.ST.ralloc_post", + "equation_FStar.Monotonic.HyperHeap.hmap", + "equation_FStar.Monotonic.HyperStack.contains", + "equation_FStar.Monotonic.HyperStack.frameOf", + "equation_FStar.Monotonic.HyperStack.is_eternal_color", + "equation_FStar.Monotonic.HyperStack.is_eternal_region", + "equation_FStar.Monotonic.HyperStack.is_tip", + "equation_FStar.Monotonic.HyperStack.is_wf_with_ctr_and_tip", + "equation_FStar.Monotonic.HyperStack.live_region", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.Monotonic.HyperStack.mreference", + "equation_FStar.Monotonic.HyperStack.unused_in", + "equation_FStar.Monotonic.HyperStack.upd", "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.fresh_loc", + "equation_Prims.eqtype", + "fuel_guarded_inversion_FStar.Monotonic.HyperStack.mreference_", + "function_token_typing_FStar.Monotonic.Heap.heap", + "function_token_typing_FStar.Monotonic.HyperHeap.rid", + "function_token_typing_FStar.UInt32.n", "int_inversion", + "lemma_FStar.Map.lemma_ContainsDom", + "lemma_FStar.Map.lemma_InDomUpd1", "lemma_FStar.Map.lemma_SelUpd1", + "lemma_FStar.Monotonic.Heap.lemma_upd_contains", + "lemma_FStar.Monotonic.HyperStack.lemma_mk_mem__projectors", + "lemma_LowStar.Monotonic.Buffer.mreference_live_loc_not_unused_in", + "lemma_LowStar.Monotonic.Buffer.mreference_unused_in_loc_unused_in", + "primitive_Prims.op_AmpAmp", "primitive_Prims.op_BarBar", + "primitive_Prims.op_LessThanOrEqual", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_FStar.Pervasives.Native.Mktuple3__1", + "projection_inverse_FStar.Pervasives.Native.Mktuple3__2", + "projection_inverse_FStar.Pervasives.Native.Mktuple3__3", + "refinement_interpretation_FStar.HyperStack.ST_Tm_refine_003cbb363565c5358e7ed8a8d7dba6d4", + "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", + "refinement_interpretation_FStar.StrongExcludedMiddle_Tm_refine_94f72bfda5e23ac3960136c8bc3f958c", + "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_5162887c6054b4734f59cfb79dd5cf2f", + "typing_FStar.Map.contains", "typing_FStar.Map.sel", + "typing_FStar.Map.upd", "typing_FStar.Monotonic.Heap.contains", + "typing_FStar.Monotonic.Heap.unused_in", + "typing_FStar.Monotonic.Heap.upd", + "typing_FStar.Monotonic.HyperStack.as_ref", + "typing_FStar.Monotonic.HyperStack.frameOf", + "typing_FStar.Monotonic.HyperStack.get_hmap", + "typing_FStar.Monotonic.HyperStack.get_rid_ctr", + "typing_FStar.Monotonic.HyperStack.get_tip", + "typing_FStar.StrongExcludedMiddle.strong_excluded_middle" + ], + 0, + "ec974d54d786f9a9016653968cb97354" + ], [ "LowStar.Monotonic.Buffer.deref", 1, @@ -975,7 +1035,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_3fe3d8508f54ae2dc29dd954960128e7" ], 0, - "b477f1d312a3051ea4fc3c7a99c7a165" + "0758735cd8c424fa7b4782f594a9d2b0" ], [ "LowStar.Monotonic.Buffer.pointer_distinct_sel_disjoint", @@ -989,7 +1049,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_3fe3d8508f54ae2dc29dd954960128e7" ], 0, - "45856d5ad762625102232f425058c782" + "f0ff98d0572cfd388c64d11c57ea141e" ], [ "LowStar.Monotonic.Buffer.msub", @@ -1002,7 +1062,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_fe6abc62014457623ceb986560f36c17" ], 0, - "fd1ef312c068e2b10808c1dda122cce0" + "8d30b876bedebcaf7d3626280b66d5c4" ], [ "LowStar.Monotonic.Buffer.moffset", @@ -1028,7 +1088,7 @@ "typing_FStar.UInt32.v" ], 0, - "29e68755f76856cfd1fd402f39767c38" + "68d6fbaa0c82354a5809017d26cc6543" ], [ "LowStar.Monotonic.Buffer.index", @@ -1046,7 +1106,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_5bc2d3af8b6b6b89753429fc786efe42" ], 0, - "2ff5f6686eab1416ac9cbba46fdc9801" + "b010c78864a8bb5eab3ac7594a3417c4" ], [ "LowStar.Monotonic.Buffer.g_upd", @@ -1055,7 +1115,7 @@ 1, [ "@query", "lemma_LowStar.Monotonic.Buffer.length_as_seq" ], 0, - "35cbdbb7b3c7036fb14139378b966170" + "9f1148ff8ab5dc17ac07681ab120feb6" ], [ "LowStar.Monotonic.Buffer.g_upd", @@ -1075,7 +1135,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "3181d0b8976e0c98fe77c3e9db46642f" + "ad8d9c5f46b70db6828f5771008bf21c" ], [ "LowStar.Monotonic.Buffer.upd'", @@ -1093,7 +1153,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_f50e31f4b48141b4b7958abcf67da20e" ], 0, - "ee76ae75181643928cdba0ecfd235aaa" + "3f3f10521a6f8dd794008e2a40c01ef0" ], [ "LowStar.Monotonic.Buffer.upd", @@ -1119,7 +1179,7 @@ "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.as_seq" ], 0, - "96fd15ac2bf05208d528875b7c0ac679" + "e9395226ce349d3928881fd4abacb92a" ], [ "LowStar.Monotonic.Buffer.freeable_disjoint", @@ -1131,7 +1191,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "16337036fa74ed82ea8d798a6ac09dcc" + "5e39d7b710cbac05f37db8977b799427" ], [ "LowStar.Monotonic.Buffer.freeable_disjoint'", @@ -1163,7 +1223,7 @@ "typing_LowStar.Monotonic.Buffer.len" ], 0, - "543ac8752c480d2be620e192bbea2daa" + "b5a5fc483d5253c339c5ac38bb42e0d5" ], [ "LowStar.Monotonic.Buffer.mgcmalloc", @@ -1180,7 +1240,7 @@ "refinement_interpretation_LowStar.Monotonic.Buffer_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" ], 0, - "03538e7fd442e22fa02264fb3dbff3fd" + "011e97bf2ce917896327cf152d838e5d" ], [ "LowStar.Monotonic.Buffer.mmalloc", @@ -1194,7 +1254,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "979d75d7bcf2094bb4fe1bf11255427a" + "a1ade3589ef7e6b32b51da10d248a26b" ], [ "LowStar.Monotonic.Buffer.malloca", @@ -1212,7 +1272,7 @@ "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "ce07e8aa8d9902e1a923640039c15cb9" + "62cb4c5abc669a3022395248e4d1c1bc" ], [ "LowStar.Monotonic.Buffer.blit", @@ -1245,7 +1305,7 @@ "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.frameOf" ], 0, - "6e8d20b5e3fa19d56c65463e247036ac" + "6893619bafa7c1c942d9d4b9ca9d7c46" ], [ "LowStar.Monotonic.Buffer.cloc_of_loc_addresses", @@ -1257,7 +1317,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "fd672530916a9ac123828ecec7afd8fa" + "74ad5834bb20b39364dcdaa82f1cc1d9" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.ToFStarBuffer.fst.hints b/ulib/LowStar.ToFStarBuffer.fst.hints index ade8c0ccdb0..24515a58648 100644 --- a/ulib/LowStar.ToFStarBuffer.fst.hints +++ b/ulib/LowStar.ToFStarBuffer.fst.hints @@ -21,7 +21,7 @@ "true_interp" ], 0, - "a809ec21d1acb60bf18441e691acc8b8" + "5e2376cadff3b4625b23d6639e46da5f" ], [ "LowStar.ToFStarBuffer.gsub_old_to_new", @@ -43,7 +43,7 @@ "true_interp" ], 0, - "3998b2b4b6c3ede9a5908abd2d226150" + "97a76dbee921395cb99d367b8e715c4b" ], [ "LowStar.ToFStarBuffer.old_and_new_cl", @@ -55,7 +55,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_aloc" ], 0, - "b195ad51845fab023c542cf166a52854" + "25a13e02387d15e898b39a7e42a2fc2c" ], [ "LowStar.ToFStarBuffer.new_to_union_loc", @@ -67,7 +67,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl" ], 0, - "4fa5076b28768893a17c6485df735d12" + "5b1c1853301be8f72225a1a1cfaef8a9" ], [ "LowStar.ToFStarBuffer.old_to_new_modifies", @@ -95,7 +95,7 @@ "typing_FStar.Monotonic.HyperStack.get_tip" ], 0, - "c256ff552ec44b6fc5538add156a6c57" + "8b56fe6d25ce4187f6c561586168b950" ], [ "LowStar.ToFStarBuffer.old_to_union_loc_none", @@ -110,7 +110,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "900b3197a073b0331c63f18c7e3eab4d" + "c7e57cdb6ee75e4cbefd736b552e3490" ], [ "LowStar.ToFStarBuffer.new_to_union_loc_none", @@ -124,7 +124,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl_union" ], 0, - "74f2189b819d779cbf0bd76ffc91462f" + "76a59abcbee6775cb4278209184b31ae" ], [ "LowStar.ToFStarBuffer.old_to_union_loc_union", @@ -140,7 +140,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "3a25bff6cf8454bee743204cc45a943f" + "a30619435ee6333819542980ef34e1a4" ], [ "LowStar.ToFStarBuffer.new_to_union_loc_union", @@ -155,7 +155,7 @@ "lemma_LowStar.Modifies.loc_union_comm" ], 0, - "3b3f27a05f9d65737361687a788870ec" + "c9f6e32e2ce01a592149407501bc9986" ], [ "LowStar.ToFStarBuffer.old_to_union_loc_addresses", @@ -175,7 +175,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "36c47fdbabf5934cd50141ada0fd1d9e" + "13217b83861030e265a1e19844bd205e" ], [ "LowStar.ToFStarBuffer.old_to_union_loc_addresses", @@ -190,7 +190,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "c3fd55293c91e51031739ddee0f634b3" + "0e125f7e2207452b7f6661e08285d756" ], [ "LowStar.ToFStarBuffer.new_to_union_loc_addresses", @@ -209,7 +209,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "865d4a8edede30a6a7fef26c02b00445" + "a8c2aedacd37f95da24b3e1a07048b9b" ], [ "LowStar.ToFStarBuffer.new_to_union_loc_addresses", @@ -223,7 +223,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl_union" ], 0, - "1a08d612f1049d4caf9d209fbdfb0c19" + "9f39a1f8eac28ef2840b3163ac331348" ], [ "LowStar.ToFStarBuffer.old_to_union_loc_regions", @@ -238,7 +238,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "b2400727f040546be90bfd9c3354ef1b" + "1aa74681073c878cca65cd7882b75c80" ], [ "LowStar.ToFStarBuffer.new_to_union_loc_regions", @@ -252,7 +252,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl_union" ], 0, - "18c4f6130f5748d28ea7978bc40b8217" + "83f0e1505fc38f14c5f68d92b98c91fb" ], [ "LowStar.ToFStarBuffer.union_loc_to_new", @@ -264,7 +264,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl" ], 0, - "b9bbce4537782e7b8fa35ab204a6aa61" + "6238b687bcc188156cdd38b7472c06f7" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_new_to_union_loc", @@ -278,7 +278,7 @@ "equation_LowStar.ToFStarBuffer.union_loc_to_new" ], 0, - "8c9a39a4983ae19c27a0d9e98f8252c7" + "41d5645fb0dcc8bc4fd41c806d857e4a" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_none", @@ -292,7 +292,7 @@ "equation_LowStar.ToFStarBuffer.union_loc_to_new" ], 0, - "2067fecd99b9ca97f020445de91bbf70" + "312c50fd7f3bb4ce143d9fa291656fef" ], [ "LowStar.ToFStarBuffer.coerce", @@ -304,7 +304,7 @@ "refinement_interpretation_LowStar.ToFStarBuffer_Tm_refine_de9aeb070296eed20d879692d0254af0" ], 0, - "525ce360149d00cffab79fdb3bfa3b2e" + "fe044af221536b7fb7ee20fccb31b300" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_union", @@ -325,7 +325,7 @@ "typing_FStar.ModifiesGen.lower_loc" ], 0, - "72743d64eac37570d94564a3b890086d" + "9b6f0182f54c2713f206252198d1452e" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_addresses", @@ -347,7 +347,7 @@ "typing_LowStar.Modifies.loc_addresses" ], 0, - "4a5e2e8021fe7badc572d2e113ab6c87" + "b70a077341348389a98a1cd2c7ca65c9" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_addresses", @@ -363,7 +363,7 @@ "typing_LowStar.Monotonic.Buffer.loc_addresses" ], 0, - "28f478822e6048fd503e15888b3ef91a" + "03e221262484b49e47ddc9755ccb1d12" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_regions", @@ -379,7 +379,7 @@ "typing_LowStar.Monotonic.Buffer.loc_regions" ], 0, - "d09efea6d4cc99609aa1e7310ad49b2e" + "76ebab7ca3ffcfebbf786d63fca00e14" ], [ "LowStar.ToFStarBuffer.old_to_new_modifies'", @@ -388,7 +388,7 @@ 1, [ "@query" ], 0, - "23696f54c81bee78abdd755d18f60754" + "edadbd4e9c16d61ad58ef6c84851d462" ], [ "LowStar.ToFStarBuffer.modifies_0_modifies", @@ -410,7 +410,7 @@ "refinement_interpretation_Prims_Tm_refine_8d65e998a07dd53ec478e27017d9dba5" ], 0, - "3ac93654a15040a54babc9b883be8d9a" + "2e4237777cd4347ed17a691d85a26db4" ], [ "LowStar.ToFStarBuffer.modifies_1_modifies", @@ -431,7 +431,7 @@ "typing_LowStar.ToFStarBuffer.new_to_old_ghost" ], 0, - "ce2ae7d2a1654f9c84d35d824e1b6bac" + "d3357197872ed56361184edb8063ead0" ], [ "LowStar.ToFStarBuffer.modifies_2_modifies", @@ -459,7 +459,7 @@ "typing_LowStar.ToFStarBuffer.union_loc_to_new" ], 0, - "07b8c80a8d1342ea3d7f16ab8c8a63dd" + "e68ea1599766880b9cfbbbc05185c0b7" ], [ "LowStar.ToFStarBuffer.ex1", @@ -508,7 +508,7 @@ "typing_LowStar.ToFStarBuffer.union_loc_to_new" ], 0, - "4597611b0e59a3af5688b8ed4e4efe31" + "fb27e64d8a5d1d71eca7f753a66f7af5" ], [ "LowStar.ToFStarBuffer.new_eqb", @@ -579,7 +579,7 @@ "typing_LowStar.ToFStarBuffer.old_to_new_ghost" ], 0, - "725cddf52388263958d35697352e10bc" + "a0c3d4e6acf6e1dcf8a122df373bd5c8" ], [ "LowStar.ToFStarBuffer.new_blit", @@ -629,7 +629,7 @@ "typing_LowStar.ToFStarBuffer.old_to_new_ghost" ], 0, - "070766c95513ee3ab6ef8ef2f61dac03" + "a6c2267b294262989739b5324369cdb9" ], [ "LowStar.ToFStarBuffer.new_fill", @@ -677,7 +677,7 @@ "typing_LowStar.Monotonic.Buffer.loc_buffer" ], 0, - "5bcfae0080eff04e600a4619e60097f3" + "bc6aadc03ea7f445aeaeb236e8ff3f68" ], [ "LowStar.ToFStarBuffer.ex1'", @@ -738,7 +738,7 @@ "typing_LowStar.ToFStarBuffer.old_to_new_ghost" ], 0, - "ed4554e0627be266c0e271c1e277686d" + "a7bb63266f8a08be86f446bfd53e01fb" ], [ "LowStar.ToFStarBuffer.ex1''", @@ -768,7 +768,7 @@ "typing_LowStar.ToFStarBuffer.old_to_new_ghost" ], 0, - "3756486c14487ff89496a42d15c8b534" + "bed8392a62af0baf54062df0da06f2fe" ], [ "LowStar.ToFStarBuffer.gsub_new_to_old", @@ -790,7 +790,7 @@ "true_interp" ], 0, - "68822d02ed54ebaa62fa7c38dcf0a174" + "48fc2713080d57f5acc876df258cf20f" ], [ "LowStar.ToFStarBuffer.gsub_old_to_new", @@ -812,7 +812,7 @@ "true_interp" ], 0, - "cf28bba273b54f08b18b9ddc58d5a789" + "77bb9255fcb1f793d8f30b4ad9438dc3" ], [ "LowStar.ToFStarBuffer.old_and_new_cl", @@ -824,7 +824,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_aloc" ], 0, - "7eed1e42c88828c6e7e99cc4af5d2ee7" + "faa9c1521f6153ca2f2013e143a53941" ], [ "LowStar.ToFStarBuffer.new_to_union_loc", @@ -836,7 +836,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl" ], 0, - "10772ce05338bf90de057a86e18df2ef" + "b7b39215fcf8a670d98f5b72eb69203e" ], [ "LowStar.ToFStarBuffer.old_to_union_loc_none", @@ -851,7 +851,7 @@ "projection_inverse_BoxBool_proj_0" ], 0, - "a572845ff54380de19ff27b618e882ac" + "a76e1065c8b79c886edcb761e24f8ca6" ], [ "LowStar.ToFStarBuffer.new_to_union_loc_none", @@ -865,7 +865,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl_union" ], 0, - "70ba595c6066e54f19617cb2350f9476" + "a3d7a77d4f6043cdfa31c3b66f87893c" ], [ "LowStar.ToFStarBuffer.old_to_union_loc_addresses", @@ -877,7 +877,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "43b7325906192da55d7b16d528a88b3c" + "2ef6c93ea714141026c95843287f7340" ], [ "LowStar.ToFStarBuffer.new_to_union_loc_addresses", @@ -889,7 +889,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "1e413a3e0d4267c0fe1162c3e5b26e5f" + "559d624ad6581d4a7a2e87be3f1fd1fd" ], [ "LowStar.ToFStarBuffer.union_loc_to_new", @@ -901,7 +901,7 @@ "equation_LowStar.ToFStarBuffer.old_and_new_cl" ], 0, - "12e1a5f37c03276b008e87b408323bbe" + "53e92136915f020cfd59d3d106d57fa9" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_none", @@ -915,7 +915,7 @@ "equation_LowStar.ToFStarBuffer.union_loc_to_new" ], 0, - "05f3a5b2eec33b425f5da3b8eed25e84" + "dabdeb3329db0efb8230cb4a7916868b" ], [ "LowStar.ToFStarBuffer.coerce", @@ -927,7 +927,7 @@ "refinement_interpretation_LowStar.ToFStarBuffer_Tm_refine_de9aeb070296eed20d879692d0254af0" ], 0, - "cd0c9a903a1db06e271b687d77abfb93" + "ebedd8576b94e862d2a726f2b6dffe8d" ], [ "LowStar.ToFStarBuffer.union_loc_to_new_addresses", @@ -939,7 +939,7 @@ "haseqPrims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d" ], 0, - "b384fa70c45673119afb421ac6c1b3ec" + "7c0444ee9d27c252820ca7245a1b3886" ], [ "LowStar.ToFStarBuffer.ex1", @@ -953,7 +953,7 @@ "refinement_interpretation_LowStar.ToFStarBuffer_Tm_refine_763bcef54285989e3ed60e8c18f79188" ], 0, - "01c535354f78bd1a127c1be52a4fde9e" + "e50824ee0f4ccc51a95cab6f9533acd4" ], [ "LowStar.ToFStarBuffer.new_eqb", @@ -976,7 +976,7 @@ "true_interp", "typing_FStar.UInt32.v" ], 0, - "43b65b298d725d15500dd3fb5a797ad8" + "2edc47439b49b6b374abaf309f3ab472" ], [ "LowStar.ToFStarBuffer.new_blit", @@ -1008,7 +1008,7 @@ "typing_LowStar.Monotonic.Buffer.frameOf" ], 0, - "71de44b507fb09e66d6bf5c8771cc633" + "c0bd0563250d3680a964152d550112a6" ], [ "LowStar.ToFStarBuffer.new_fill", @@ -1044,7 +1044,7 @@ "typing_LowStar.Buffer.trivial_preorder" ], 0, - "6fd32ba093890daf1234c6710ce530e8" + "0da3b02ec305c2b22ef94f1e70d8fba8" ], [ "LowStar.ToFStarBuffer.ex1'", @@ -1058,7 +1058,7 @@ "refinement_interpretation_LowStar.ToFStarBuffer_Tm_refine_e524f2a490314ad581b10efe414031e4" ], 0, - "45afb919c89a1ae8313c1a70c68b4d56" + "17ef4c739e934aea1beb755cbe66d367" ], [ "LowStar.ToFStarBuffer.ex1''", @@ -1072,7 +1072,7 @@ "refinement_interpretation_LowStar.ToFStarBuffer_Tm_refine_763bcef54285989e3ed60e8c18f79188" ], 0, - "4f0544705cfeac9643f22cb1b10a6b5b" + "16a7b55cdebeb06610b61b286aef234d" ] ] ] \ No newline at end of file diff --git a/ulib/LowStar.UninitializedBuffer.fst.hints b/ulib/LowStar.UninitializedBuffer.fst.hints new file mode 100644 index 00000000000..057fd929724 --- /dev/null +++ b/ulib/LowStar.UninitializedBuffer.fst.hints @@ -0,0 +1,679 @@ +[ + "\u0002%g\u0014fWɖ}\u0000@", + [ + [ + "LowStar.UninitializedBuffer.initialization_preorder", + 1, + 2, + 1, + [ + "@query", "eq2-interp", "equation_FStar.Preorder.preorder_rel", + "equation_Prims.l_Forall", "equation_Prims.logical", + "equation_Prims.nat", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "l_and-interp", "l_quant_interp__3538" + ], + 0, + "5a359a65dd85a1ba1d371f34f3b46056" + ], + [ + "LowStar.UninitializedBuffer.unull", + 1, + 2, + 1, + [ + "@query", "kinding_FStar.Pervasives.Native.option@tok", + "lemma_LowStar.Monotonic.Buffer.recallable_null", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "8a2dfd59252ceff2ec917a444e2e1996" + ], + [ + "LowStar.UninitializedBuffer.uindex", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", + "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.initialized_at", + "equation_LowStar.UninitializedBuffer.ipred", + "equation_LowStar.UninitializedBuffer.ubuffer", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_LowStar.UninitializedBuffer.ipred", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_1c5b46c0367b5f079b2235af621bbca9", + "kinding_FStar.Pervasives.Native.option@tok", "l_imp-interp", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "primitive_Prims.op_AmpAmp", "primitive_Prims.op_LessThan", + "primitive_Prims.op_LessThanOrEqual", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_85223ecfbcb31fdf746c856bc55b21d9", + "typing_FStar.UInt32.v", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "197da3ba2db018c61b2bfe3e9f34fff4" + ], + [ + "LowStar.UninitializedBuffer.uupd", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "constructor_distinct_FStar.Pervasives.Native.Some", + "data_typing_intro_FStar.Pervasives.Native.Some@tok", + "disc_equation_FStar.Pervasives.Native.None", + "disc_equation_FStar.Pervasives.Native.Some", "eq2-interp", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", + "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.initialization_preorder", + "equation_LowStar.UninitializedBuffer.initialized_at", + "equation_LowStar.UninitializedBuffer.ipred", + "equation_LowStar.UninitializedBuffer.ubuffer", + "equation_Prims.logical", "equation_Prims.nat", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_LowStar.UninitializedBuffer.initialization_preorder", + "function_token_typing_LowStar.UninitializedBuffer.ipred", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_1c5b46c0367b5f079b2235af621bbca9", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "kinding_FStar.Pervasives.Native.option@tok", "l_and-interp", + "l_imp-interp", "l_quant_interp__3544", + "lemma_FStar.Pervasives.invertOption", + "lemma_FStar.Seq.Base.lemma_index_upd1", + "lemma_FStar.Seq.Base.lemma_index_upd2", + "lemma_FStar.Seq.Base.lemma_len_upd", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "lemma_LowStar.Monotonic.Buffer.length_null_1", + "lemma_LowStar.Monotonic.Buffer.length_null_2", + "primitive_Prims.op_AmpAmp", "primitive_Prims.op_LessThan", + "primitive_Prims.op_LessThanOrEqual", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_FStar.Pervasives.Native.Some_a", + "projection_inverse_FStar.Pervasives.Native.Some_v", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_2ca062977a42c36634b89c1c4f193f79", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_36f208f2b1019ab7b5d9be73f4c89349", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_b5ad1dbfbd48faaf34d92bafda76205d", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_98ee5bca492854a87efa3fdf97082c41", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_efd10a39d41e4ae29ca8fcabfecff808", + "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", + "typing_FStar.Seq.Base.index", "typing_FStar.Seq.Base.upd", + "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.as_seq", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "ca92f1964f1ddb88ae780aaf2d607b3d" + ], + [ + "LowStar.UninitializedBuffer.ugcmalloc", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "equation_FStar.Monotonic.HyperStack.mem", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_68d4074054df2bfcbaf4824f0cb08ff4" + ], + 0, + "c56268b8ef8a8902eecbb228508b16a1" + ], + [ + "LowStar.UninitializedBuffer.ublit_post_j", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "bool_inversion", "equation_FStar.Monotonic.HyperHeap.hmap", + "equation_FStar.Monotonic.HyperStack.is_tip", + "equation_FStar.Monotonic.HyperStack.is_wf_with_ctr_and_tip", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", + "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.ubuffer", + "equation_Prims.eqtype", "equation_Prims.nat", + "function_token_typing_FStar.Monotonic.Heap.heap", + "function_token_typing_FStar.Monotonic.HyperHeap.rid", + "function_token_typing_FStar.UInt32.n", "int_inversion", + "kinding_FStar.Pervasives.Native.option@tok", + "lemma_FStar.Map.lemma_ContainsDom", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", + "primitive_Prims.op_LessThanOrEqual", + "primitive_Prims.op_Subtraction", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_BoxInt_proj_0", + "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6eed8fe1d6aaea2a400f085561998804", + "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", + "typing_FStar.Map.contains", + "typing_FStar.Monotonic.HyperStack.get_hmap", + "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.UInt32.v", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "aa97cdc6067d8e90af87566128b16cdc" + ], + [ + "LowStar.UninitializedBuffer.ublit", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "FStar.UInt32_pretyping_041e3a67a2d2b51fd702f1f88cfc3b44", + "Prims_pretyping_ae567c2fb75be05905677af440075565", + "assumption_FStar.UInt32.t__uu___haseq", "b2t_def", "bool_inversion", + "bool_typing", "data_typing_intro_FStar.Pervasives.Native.Some@tok", + "equation_FStar.HyperStack.ST.equal_domains", + "equation_FStar.Monotonic.Heap.equal_dom", + "equation_FStar.Monotonic.HyperHeap.hmap", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.lt", + "equation_FStar.UInt.max_int", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", + "equation_FStar.UInt32.lt", "equation_FStar.UInt32.n", + "equation_FStar.UInt32.n_minus_one", + "equation_LowStar.Monotonic.Buffer.disjoint", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.ubuffer", + "equation_Prims.eqtype", "equation_Prims.nat", + "function_token_typing_FStar.Monotonic.Heap.heap", + "function_token_typing_FStar.Monotonic.HyperHeap.rid", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_FStar.UInt32.n_minus_one", + "haseqLowStar.UninitializedBuffer_Tm_refine_63e00eb0a4b441bc1f4a5ff630033e0b", + "int_inversion", "int_typing", + "kinding_FStar.Pervasives.Native.option@tok", + "lemma_FStar.HyperStack.ST.lemma_equal_domains_trans", + "lemma_FStar.HyperStack.ST.lemma_same_refs_in_all_regions_intro", + "lemma_FStar.Seq.Base.lemma_index_upd1", + "lemma_FStar.Seq.Base.lemma_index_upd2", + "lemma_FStar.Seq.Properties.slice_upd", + "lemma_FStar.Set.lemma_equal_refl", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "lemma_LowStar.Monotonic.Buffer.loc_union_idem", + "lemma_LowStar.Monotonic.Buffer.modifies_inert_buffer_elim", + "lemma_LowStar.Monotonic.Buffer.modifies_inert_intro", + "lemma_LowStar.Monotonic.Buffer.modifies_refl", + "lemma_LowStar.Monotonic.Buffer.modifies_trans", + "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", + "primitive_Prims.op_Equality", "primitive_Prims.op_LessThan", + "primitive_Prims.op_LessThanOrEqual", + "primitive_Prims.op_Subtraction", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_BoxInt_proj_0", + "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_3321cbe2f573e3c988fd0895bf1f0cf9", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_36f208f2b1019ab7b5d9be73f4c89349", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_b5ad1dbfbd48faaf34d92bafda76205d", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6eed8fe1d6aaea2a400f085561998804", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_91971967136e03820d614d68c54f118a", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_a18ecb82040c978301074c06b1c779a5", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_a73cdd2bffa7eb510b9150d828f96cc6", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_b09996fec1b8e0f729e41438f7ead36a", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_cd02a8680910edb2a47270d917f8b5cf", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_cfb754147a155e7512f067844c74c8f3", + "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", + "typing_FStar.Map.domain", + "typing_FStar.Monotonic.HyperStack.get_hmap", + "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.as_seq", + "typing_LowStar.Monotonic.Buffer.len", + "typing_LowStar.Monotonic.Buffer.length", + "typing_LowStar.Monotonic.Buffer.loc_buffer", + "typing_LowStar.UninitializedBuffer.initialization_preorder", + "unit_inversion", "unit_typing" + ], + 0, + "0fae6212f486606e67a75e32aaa11b50" + ], + [ + "LowStar.UninitializedBuffer.witness_initialized", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "disc_equation_FStar.Pervasives.Native.Some", "eq2-interp", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.size", + "equation_FStar.UInt.uint_t", "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.initialization_preorder", + "equation_LowStar.UninitializedBuffer.initialized_at", + "equation_LowStar.UninitializedBuffer.ipred", + "equation_LowStar.UninitializedBuffer.ubuffer", + "equation_Prims.logical", "equation_Prims.nat", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_LowStar.UninitializedBuffer.initialization_preorder", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_1c5b46c0367b5f079b2235af621bbca9", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "kinding_FStar.Pervasives.Native.option@tok", "l_and-interp", + "l_imp-interp", "l_quant_interp__3544", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "primitive_Prims.op_AmpAmp", "primitive_Prims.op_LessThan", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_2ef4227f53606829f5d631eed9c15388", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", + "token_correspondence_LowStar.UninitializedBuffer.ipred", + "typing_FStar.UInt32.v", "typing_LowStar.Monotonic.Buffer.len", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "1ad53ac0b8c2c7aa9f6f197141c66fea" + ], + [ + "LowStar.UninitializedBuffer.recall_initialized", + 1, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", "b2t_def", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_LowStar.UninitializedBuffer.initialized_at", + "equation_LowStar.UninitializedBuffer.ipred", + "equation_LowStar.UninitializedBuffer.ubuffer", "equation_Prims.nat", + "function_token_typing_LowStar.UninitializedBuffer.ipred", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_1c5b46c0367b5f079b2235af621bbca9", + "kinding_FStar.Pervasives.Native.option@tok", "l_imp-interp", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "primitive_Prims.op_LessThan", "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_deec62e3eab3e2503db3f1d6877f45da", + "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "15a3499debfd06f2b10a6844ce3f4c9f" + ], + [ + "LowStar.UninitializedBuffer.initialization_preorder", + 2, + 2, + 1, + [ + "@query", "eq2-interp", "equation_FStar.Preorder.preorder_rel", + "equation_Prims.l_Forall", "equation_Prims.logical", + "equation_Prims.nat", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "l_and-interp", "l_quant_interp__3861" + ], + 0, + "b752cb35d448fbf2d1ac11f5795f3fdd" + ], + [ + "LowStar.UninitializedBuffer.unull", + 2, + 2, + 1, + [ + "@query", "kinding_FStar.Pervasives.Native.option@tok", + "lemma_LowStar.Monotonic.Buffer.recallable_null", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "5507333ae8f0a44ed20b711c8a93276f" + ], + [ + "LowStar.UninitializedBuffer.gsub", + 1, + 2, + 1, + [ "@query" ], + 0, + "2734a038905c76ae97ea63a22645ed0e" + ], + [ + "LowStar.UninitializedBuffer.gsub", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "eq2-interp", "equation_FStar.UInt.fits", + "equation_FStar.UInt.min_int", "equation_FStar.UInt.size", + "equation_FStar.UInt.uint_t", "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.initialization_preorder", + "equation_Prims.logical", "equation_Prims.nat", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_LowStar.UninitializedBuffer.initialization_preorder", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "kinding_FStar.Pervasives.Native.option@tok", "l_and-interp", + "lemma_FStar.Seq.Base.lemma_len_slice", + "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", + "primitive_Prims.op_LessThanOrEqual", + "primitive_Prims.op_Subtraction", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_BoxInt_proj_0", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_aebc5aa9049e78f605051015a3436e68", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_b612ee674c47165ef8c3a00ab676a2f0", + "typing_FStar.UInt32.v" + ], + 0, + "d61d6f4843bca733e2f32b980f200799" + ], + [ + "LowStar.UninitializedBuffer.gsub_inj", + 1, + 2, + 1, + [ "@query" ], + 0, + "b91331f0b95375e6476713a868cb5aac" + ], + [ + "LowStar.UninitializedBuffer.gsub_inj", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "eq2-interp", "equation_FStar.UInt.fits", + "equation_FStar.UInt.min_int", "equation_FStar.UInt.size", + "equation_FStar.UInt.uint_t", "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.initialization_preorder", + "equation_Prims.logical", "equation_Prims.nat", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_LowStar.UninitializedBuffer.initialization_preorder", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "kinding_FStar.Pervasives.Native.option@tok", "l_and-interp", + "lemma_FStar.Seq.Base.lemma_len_slice", + "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", + "primitive_Prims.op_LessThanOrEqual", + "primitive_Prims.op_Subtraction", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_BoxInt_proj_0", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_aebc5aa9049e78f605051015a3436e68", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_b612ee674c47165ef8c3a00ab676a2f0", + "typing_FStar.UInt32.v" + ], + 0, + "6df0e9fbdcbeb228d82fb2394685636b" + ], + [ + "LowStar.UninitializedBuffer.usub", + 1, + 2, + 1, + [ "@query" ], + 0, + "f4800c4ca26a9596a0c4c8cdf9f3813c" + ], + [ + "LowStar.UninitializedBuffer.usub", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "bool_inversion", "eq2-interp", + "equation_FStar.Monotonic.HyperHeap.hmap", + "equation_FStar.Monotonic.HyperStack.is_tip", + "equation_FStar.Monotonic.HyperStack.is_wf_with_ctr_and_tip", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", + "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.initialization_preorder", + "equation_Prims.eqtype", "equation_Prims.logical", + "equation_Prims.nat", + "function_token_typing_FStar.Monotonic.Heap.heap", + "function_token_typing_FStar.Monotonic.HyperHeap.rid", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_LowStar.UninitializedBuffer.initialization_preorder", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "kinding_FStar.Pervasives.Native.option@tok", "l_and-interp", + "lemma_FStar.Map.lemma_ContainsDom", + "lemma_FStar.Seq.Base.lemma_len_slice", + "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", + "primitive_Prims.op_LessThanOrEqual", + "primitive_Prims.op_Subtraction", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_BoxInt_proj_0", + "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_aebc5aa9049e78f605051015a3436e68", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_39d218f874370dbd95af12e77bdc6c26", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_b612ee674c47165ef8c3a00ab676a2f0", + "typing_FStar.Map.contains", + "typing_FStar.Monotonic.HyperStack.get_hmap", + "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.UInt32.v" + ], + 0, + "17aced7f8d47a3079bb14a9c0cd7afed" + ], + [ + "LowStar.UninitializedBuffer.uoffset", + 1, + 2, + 1, + [ "@query" ], + 0, + "04ad865c292ff64029157be6d6ca3eed" + ], + [ + "LowStar.UninitializedBuffer.uoffset", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "bool_inversion", "eq2-interp", + "equation_FStar.Monotonic.HyperHeap.hmap", + "equation_FStar.Monotonic.HyperStack.is_tip", + "equation_FStar.Monotonic.HyperStack.is_wf_with_ctr_and_tip", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.max_int", + "equation_FStar.UInt.min_int", "equation_FStar.UInt.size", + "equation_FStar.UInt.uint_t", "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.initialization_preorder", + "equation_Prims.eqtype", "equation_Prims.logical", + "equation_Prims.nat", + "function_token_typing_FStar.Monotonic.Heap.heap", + "function_token_typing_FStar.Monotonic.HyperHeap.rid", + "function_token_typing_FStar.UInt32.n", + "function_token_typing_LowStar.UninitializedBuffer.initialization_preorder", + "int_inversion", + "interpretation_LowStar.UninitializedBuffer_Tm_abs_45fb7196bd55c525a78a9c8bdaa6eef7", + "kinding_FStar.Pervasives.Native.option@tok", "l_and-interp", + "lemma_FStar.Map.lemma_ContainsDom", + "lemma_FStar.Seq.Base.lemma_len_slice", + "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", + "primitive_Prims.op_LessThanOrEqual", + "primitive_Prims.op_Subtraction", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_BoxInt_proj_0", + "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", + "refinement_interpretation_FStar.Seq.Base_Tm_refine_aebc5aa9049e78f605051015a3436e68", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_b612ee674c47165ef8c3a00ab676a2f0", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_fe618a37959e601c6d3afa286fa0a682", + "typing_FStar.Map.contains", + "typing_FStar.Monotonic.HyperStack.get_hmap", + "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.UInt32.v", + "typing_LowStar.Monotonic.Buffer.len", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "76a7114732136093bdba5c7d9ee092ac" + ], + [ + "LowStar.UninitializedBuffer.uindex", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", "b2t_def", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", + "equation_LowStar.UninitializedBuffer.ubuffer", + "kinding_FStar.Pervasives.Native.option@tok", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "primitive_Prims.op_AmpAmp", "primitive_Prims.op_LessThanOrEqual", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_85223ecfbcb31fdf746c856bc55b21d9", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "8f38ad545c36888f630868a37dda279e" + ], + [ + "LowStar.UninitializedBuffer.uupd", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", + "equation_FStar.UInt32.n", + "equation_LowStar.UninitializedBuffer.ubuffer", + "function_token_typing_FStar.UInt32.n", "int_inversion", + "kinding_FStar.Pervasives.Native.option@tok", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "primitive_Prims.op_AmpAmp", "primitive_Prims.op_LessThanOrEqual", + "projection_inverse_BoxBool_proj_0", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_efd10a39d41e4ae29ca8fcabfecff808", + "typing_FStar.UInt32.v", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "5c7015d3514d70514f9d4cf8e7a10bf7" + ], + [ + "LowStar.UninitializedBuffer.ugcmalloc", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "equation_FStar.Monotonic.HyperStack.mem", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_2f4c4317c33d464b36cc12cfcbde1c55" + ], + 0, + "2cdbdc8bbb2bb2566e742615433e4f92" + ], + [ + "LowStar.UninitializedBuffer.ublit_post_j", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "Prims_pretyping_ae567c2fb75be05905677af440075565", "b2t_def", + "bool_inversion", "equation_FStar.Monotonic.HyperHeap.hmap", + "equation_FStar.Monotonic.HyperStack.is_tip", + "equation_FStar.Monotonic.HyperStack.is_wf_with_ctr_and_tip", + "equation_FStar.Monotonic.HyperStack.mem", + "equation_FStar.UInt.fits", "equation_FStar.UInt.min_int", + "equation_FStar.UInt.size", "equation_FStar.UInt.uint_t", + "equation_FStar.UInt32.n", + "equation_LowStar.Monotonic.Buffer.length", + "equation_LowStar.UninitializedBuffer.ubuffer", + "equation_Prims.eqtype", "equation_Prims.nat", + "function_token_typing_FStar.Monotonic.Heap.heap", + "function_token_typing_FStar.Monotonic.HyperHeap.rid", + "function_token_typing_FStar.UInt32.n", "int_inversion", + "kinding_FStar.Pervasives.Native.option@tok", + "lemma_FStar.Map.lemma_ContainsDom", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "primitive_Prims.op_Addition", "primitive_Prims.op_AmpAmp", + "primitive_Prims.op_LessThanOrEqual", + "primitive_Prims.op_Subtraction", + "projection_inverse_BoxBool_proj_0", + "projection_inverse_BoxInt_proj_0", + "refinement_interpretation_FStar.Monotonic.HyperStack_Tm_refine_9a74d818566e70513bc032cc3b65a144", + "refinement_interpretation_FStar.UInt_Tm_refine_a347709bfeba48709474ad26f4f6be87", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6eed8fe1d6aaea2a400f085561998804", + "refinement_interpretation_Prims_Tm_refine_ba523126f67e00e7cd55f0b92f16681d", + "typing_FStar.Map.contains", + "typing_FStar.Monotonic.HyperStack.get_hmap", + "typing_FStar.Monotonic.HyperStack.get_tip", "typing_FStar.UInt32.v", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "cde38eec91b818096734a4dd7b4cf5fd" + ], + [ + "LowStar.UninitializedBuffer.witness_initialized", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "equation_LowStar.UninitializedBuffer.ubuffer", + "kinding_FStar.Pervasives.Native.option@tok", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "ba159339525ef01bf985984b31b379d4" + ], + [ + "LowStar.UninitializedBuffer.recall_initialized", + 2, + 2, + 1, + [ + "@MaxIFuel_assumption", "@query", + "equation_LowStar.UninitializedBuffer.ubuffer", + "kinding_FStar.Pervasives.Native.option@tok", + "lemma_LowStar.Monotonic.Buffer.length_as_seq", + "refinement_interpretation_LowStar.UninitializedBuffer_Tm_refine_6a651958a62cf6fbed628aedc3b1e112", + "typing_LowStar.UninitializedBuffer.initialization_preorder" + ], + 0, + "fa974feee51451991e4940b28612140d" + ] + ] +] \ No newline at end of file diff --git a/ulib/prims.fst.hints b/ulib/prims.fst.hints index c714ac89d50..a902a621faf 100644 --- a/ulib/prims.fst.hints +++ b/ulib/prims.fst.hints @@ -121,7 +121,7 @@ "well-founded-ordering-on-nat" ], 0, - "80c243745238ace0a7e1dcad935be9ca" + "f8eb1d17688d136f8c7ee7c6fefea818" ], [ "Prims.Ghost", @@ -243,7 +243,7 @@ "well-founded-ordering-on-nat" ], 0, - "bee8dbcf7f5c117bd92472e99ba45d68" + "fb6d68b9900357e76cc59c2f42b47896" ] ] ] \ No newline at end of file