feat(mpn_copyi): Proved correctness of mpn_copyi and other simple util functions.
This commit is contained in:
6
projects/lib/gmp_goal_check.v
Normal file
6
projects/lib/gmp_goal_check.v
Normal file
@ -0,0 +1,6 @@
|
||||
From Require Import gmp_goal gmp_proof_auto gmp_proof_manual.
|
||||
|
||||
Module VC_Correctness : VC_Correct.
|
||||
Include gmp_proof_auto.
|
||||
Include gmp_proof_manual.
|
||||
End VC_Correctness.
|
Reference in New Issue
Block a user