Rename some confusing fields (#51)

This commit is contained in:
Patrick Stevens
2019-10-13 09:31:54 +01:00
committed by GitHub
parent 96d15c6017
commit 959071214e
21 changed files with 441 additions and 441 deletions

View File

@@ -180,13 +180,13 @@ distLemma a b rewrite Semiring.commutative Semiring (a +N b *N a) b | Semirin
Ring : Ring (reflSetoid ) _+Z_ _*Z_
Ring.additiveGroup Ring = Group
Ring.multWellDefined Ring refl refl = refl
Ring.*WellDefined Ring refl refl = refl
Ring.1R Ring = nonneg 1
Ring.groupIsAbelian Ring {a} {b} = +ZCommutative a b
Ring.multAssoc Ring {a} {b} {c} = *ZAssociative a b c
Ring.multCommutative Ring {a} {b} = *ZCommutative a b
Ring.multDistributes Ring {a} {b} {c} = *ZDistributesOver+Z a b c
Ring.multIdentIsIdent Ring {a} = *ZleftIdent a
Ring.*Associative Ring {a} {b} {c} = *ZAssociative a b c
Ring.*Commutative Ring {a} {b} = *ZCommutative a b
Ring.*DistributesOver+ Ring {a} {b} {c} = *ZDistributesOver+Z a b c
Ring.identIsIdent Ring {a} = *ZleftIdent a
intDom : (a b : ) a *Z b nonneg 0 (a nonneg 0) || (b nonneg 0)
intDom (nonneg zero) (nonneg b) pr = inl refl