Skip to content

Commit

Permalink
Fix aatgroup for the experimental kernel
Browse files Browse the repository at this point in the history
  • Loading branch information
mn200 committed Aug 27, 2024
1 parent 2cb041d commit de7fb61
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions examples/algebra/aat/aatgroupScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -481,6 +481,7 @@ Theorem monoid_iso_isgroup:
Proof
xfer_back_tac[] >>
rw[monoidTheory.MonoidIso_def, monoidTheory.MonoidHomo_def] >>
rename [‘BIJ f g.carrier h.carrier’] >>
‘GroupHomo f g h’ by simp[groupTheory.GroupHomo_def] >>
‘GroupIso f g h’ by simp[groupTheory.GroupIso_def] >>
metis_tac[groupTheory.group_iso_group]
Expand Down

0 comments on commit de7fb61

Please sign in to comment.