Lots of rings (#82)

This commit is contained in:
Patrick Stevens
2019-11-22 19:52:57 +00:00
committed by GitHub
parent b33baa5fb7
commit 660d7aa27c
40 changed files with 1246 additions and 881 deletions

View File

@@ -19,4 +19,9 @@ module Rings.Isomorphisms.Definition {a b c d : _} {A : Set a} {S : Setoid {a} {
record RingIso (f : A B) : Set (a b c d) where
field
ringHom : RingHom R1 R2 f
bijective : Bijection f
bijective : SetoidBijection S T f
record RingsIsomorphic : Set (a b c d) where
field
f : A B
iso : RingIso f