Skip to content

Commit

Permalink
Fixes for 8.16
Browse files Browse the repository at this point in the history
  • Loading branch information
wjbs committed Jan 21, 2025
1 parent 8241173 commit 71163cc
Show file tree
Hide file tree
Showing 5 changed files with 8 additions and 6 deletions.
4 changes: 2 additions & 2 deletions src/CoreData/SemanticCore.v
Original file line number Diff line number Diff line change
Expand Up @@ -256,7 +256,7 @@ Proof.
rewrite kron_n_assoc; [| auto with wf_db].
unfold kron.
destruct (S j mod 2 ^S n) eqn:En.
+ destruct (Nat.Div0.mod_divides (S j) (2 ^ S n)).
+ destruct (Nat.mod_divides (S j) (2 ^ S n) (pow2_nonzero _)).

Check warning on line 259 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.17, default)

Notation Nat.mod_divides is deprecated since 8.17.

Check warning on line 259 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.17, default)

Notation Nat.mod_divides is deprecated since 8.17.

Check warning on line 259 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.18, default)

Notation Nat.mod_divides is deprecated since 8.17.

Check warning on line 259 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.18, default)

Notation Nat.mod_divides is deprecated since 8.17.
destruct (H En).
rewrite H1.
replace (2 ^ S n * x / 2 ^ S n)%nat with x.
Expand Down Expand Up @@ -324,7 +324,7 @@ Proof.
rewrite Nat.mod_1_r.
rewrite Nat.div_1_r.
destruct (S i mod 2 ^ S n) eqn:En.
+ destruct (Nat.Div0.mod_divides (S i) (2^S n)).
+ destruct (Nat.mod_divides (S i) (2^S n) (pow2_nonzero _)).

Check warning on line 327 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.17, default)

Notation Nat.mod_divides is deprecated since 8.17.

Check warning on line 327 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.17, default)

Notation Nat.mod_divides is deprecated since 8.17.

Check warning on line 327 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.18, default)

Notation Nat.mod_divides is deprecated since 8.17.

Check warning on line 327 in src/CoreData/SemanticCore.v

View workflow job for this annotation

GitHub Actions / build (8.18, default)

Notation Nat.mod_divides is deprecated since 8.17.
destruct H; [assumption |].
rewrite H.
rewrite Nat.mul_comm.
Expand Down
4 changes: 2 additions & 2 deletions src/CoreRules/ZXRules.v
Original file line number Diff line number Diff line change
Expand Up @@ -108,7 +108,7 @@ Proof.
replace (0)%R with (0 * PI)%R at 1 by lra.
replace (0)%R with (INR 0)%R by reflexivity.
zxrewrite X_state_copy.
rewrite INR_0, Rmult_0_l.
rewrite Rmult_0_l.
zxrefl.
Qed.

Expand All @@ -131,7 +131,7 @@ Proof.
replace (0)%R with (0 * PI)%R at 1 by lra.
replace (0)%R with (INR 0)%R by reflexivity.
zxrewrite Z_state_copy.
rewrite INR_0, Rmult_0_l.
rewrite Rmult_0_l.
zxrefl.
Qed.

Expand Down
2 changes: 1 addition & 1 deletion src/DiagramRules/Completeness.v
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ Proof.
rewrite X_2_1_0_semantics.
compute_matrix (Z_semantics 0 1 α ⊗ Z_semantics 0 1 (α + PI)).
compute_matrix (Z_semantics 0 2 (2 * α + PI)).
rewrite <- Cexp_add, <- Rplus_assoc, 3!Cexp_plus_PI, Rplus_diag.
rewrite <- Cexp_add, <- Rplus_assoc, 3!Cexp_plus_PI, <- double.

Check warning on line 17 in src/DiagramRules/Completeness.v

View workflow job for this annotation

GitHub Actions / build (8.18, default)

Notation double is deprecated since 8.19. Use Rplus_diag.

Check warning on line 17 in src/DiagramRules/Completeness.v

View workflow job for this annotation

GitHub Actions / build (8.18, default)

Notation double is deprecated since 8.19. Use Rplus_diag.

Check warning on line 17 in src/DiagramRules/Completeness.v

View workflow job for this annotation

GitHub Actions / build (8.18, default)

Notation double is deprecated since 8.19. Use Rplus_diag.
prep_matrix_equivalence.
by_cell; lca.
Qed.
Expand Down
2 changes: 1 addition & 1 deletion src/DiagramRules/Soundness.v
Original file line number Diff line number Diff line change
Expand Up @@ -52,7 +52,7 @@ Proof.
- C_field.
- rewrite Cmod_div by auto.
rewrite Hmod.
rewrite Rdiv_diag; [reflexivity|].
apply Rinv_r.
rewrite Cmod_eq_0_iff.
auto.
Qed.
Expand Down
2 changes: 2 additions & 0 deletions src/Permutations/ZXpermFacts.v
Original file line number Diff line number Diff line change
Expand Up @@ -896,6 +896,8 @@ Lemma zx_of_perm_zxperm n f :
ZXperm (zx_of_perm n f).
Proof.
unfold zx_of_perm.
rewrite zxperm_iff_cast'.
unfold zx_of_perm_uncast.
auto_zxperm.
Qed.

Expand Down

0 comments on commit 71163cc

Please sign in to comment.