mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-12 07:08:40 +00:00
Lots of rings (#82)
This commit is contained in:
@@ -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
|
||||
|
Reference in New Issue
Block a user