File tree Expand file tree Collapse file tree 7 files changed +20
-16
lines changed
Construct/Quotient/Ring/Properties Expand file tree Collapse file tree 7 files changed +20
-16
lines changed Original file line number Diff line number Diff line change 11------------------------------------------------------------------------
2- -- The Chinese Remainder Theorem for arbitrary rings
3- --
42-- The Agda standard library
3+ --
4+ -- The Chinese Remainder Theorem for arbitrary rings
55------------------------------------------------------------------------
66
77{-# OPTIONS --safe --cubical-compatible #-}
Original file line number Diff line number Diff line change 11------------------------------------------------------------------------
2- -- Ideals of a ring
3- --
42-- The Agda standard library
3+ --
4+ -- Ideals of a ring
55------------------------------------------------------------------------
66
77{-# OPTIONS --safe --cubical-compatible #-}
Original file line number Diff line number Diff line change 11------------------------------------------------------------------------
2- -- Intersection of ideals
3- --
42-- The Agda standard library
3+ --
4+ -- Intersection of ideals
55------------------------------------------------------------------------
66
77{-# OPTIONS --safe --cubical-compatible #-}
Original file line number Diff line number Diff line change 1- {-# OPTIONS --safe --without-K #-}
1+ ------------------------------------------------------------------------
2+ -- The Agda standard library
3+ --
4+ -- The kernel of a ring homomorphism is an ideal
5+ ------------------------------------------------------------------------
6+
7+ {-# OPTIONS --safe --cubical-compatible #-}
28
39open import Algebra.Bundles
410open import Algebra.Morphism.Structures
Original file line number Diff line number Diff line change 11------------------------------------------------------------------------
2- -- Coprimality of ideals
3- --
42-- The Agda standard library
3+ --
4+ -- Coprimality of ideals
55------------------------------------------------------------------------
66
77{-# OPTIONS --safe --cubical-compatible #-}
Original file line number Diff line number Diff line change 11------------------------------------------------------------------------
2- -- Intersection of normal subgroups
3- --
42-- The Agda standard library
3+ --
4+ -- Intersection of normal subgroups
55------------------------------------------------------------------------
66
77{-# OPTIONS --safe --cubical-compatible #-}
@@ -84,5 +84,3 @@ N ∩ M = record
8484 where
8585 module N = NormalSubgroup N
8686 module M = NormalSubgroup M
87-
88-
Original file line number Diff line number Diff line change 11------------------------------------------------------------------------
2- -- The kernel of a group homomorphism is a normal subgroup
3- --
42-- The Agda standard library
3+ --
4+ -- The kernel of a group homomorphism is a normal subgroup
55------------------------------------------------------------------------
66
77{-# OPTIONS --safe --cubical-compatible #-}
@@ -52,7 +52,7 @@ x ∙ₖ y = record
5252 { element = G.ε
5353 ; inKernel = ρ.ε-homo
5454 }
55-
55+
5656_⁻¹ₖ : Kernel → Kernel
5757x ⁻¹ₖ = record
5858 { element = X.element G.⁻¹
You can’t perform that action at this time.
0 commit comments