Skip to content

Commit

Permalink
Added Relations example (over types), with individual structures for …
Browse files Browse the repository at this point in the history
…product (through CompactClosed & DaggerSymmetricMonoidal) and sum (through SymmetricMonoidal & DaggerSymmetricMonoidal), as well as showing the latter cannot be a CompactClosedCategory.
  • Loading branch information
wjbs committed Mar 8, 2024
1 parent 2b2d006 commit b9b3c46
Show file tree
Hide file tree
Showing 3 changed files with 530 additions and 2 deletions.
4 changes: 2 additions & 2 deletions ViCaR/Classes/ExamplesAutomation.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,9 +2,9 @@ From VyZX Require Import PermutationAutomation.
Require Import String.

Ltac print_state :=
try (match goal with | H : ?p |- _ => idtac H ":" p; fail end);
try (match reverse goal with | H : ?p |- _ => idtac H ":" p; fail end);
idtac "---------------------------------------------------------";
match goal with |- ?P => idtac P; idtac ""
match reverse goal with |- ?P => idtac P; idtac ""
end.

Ltac is_C0 x := assert (x = C0) by (cbv; lca).
Expand Down
1 change: 1 addition & 0 deletions examples/NatRelationsExample.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
Require Import Setoid.
From ViCaR Require Export CategoryTypeclass.

Require Import Psatz.

Expand Down
Loading

0 comments on commit b9b3c46

Please sign in to comment.