fix(mpz_realloc): fix minor bugs in proof of mpz_realloc.

This commit is contained in:
xiaoh105
2025-06-21 22:23:37 +08:00
parent 1e627cdb84
commit f4db688a30
5 changed files with 97 additions and 141 deletions

View File

@ -15,8 +15,6 @@ Local Open Scope Z_scope.
Local Open Scope sets.
Local Open Scope string.
Local Open Scope list.
Require Import Coq.ZArith.ZArith.
Local Open Scope Z_scope.
Import naive_C_Rules.
Local Open Scope sac.
@ -243,4 +241,5 @@ Lemma proof_of_mpz_realloc_partial_solve_wit_9 : mpz_realloc_partial_solve_wit_9
Proof. Admitted.
Lemma proof_of_mpz_realloc_partial_solve_wit_10 : mpz_realloc_partial_solve_wit_10.
Proof. Admitted.
Proof. Admitted.