More lecture notes (#126)

This commit is contained in:
Patrick Stevens
2020-04-19 20:15:02 +01:00
committed by GitHub
parent 485b27e009
commit cab004f6d8
11 changed files with 163 additions and 36 deletions

View File

@@ -35,3 +35,5 @@ record Ring {n m} {A : Set n} (S : Setoid {n} {m} A) (_+_ : A → A → A) (_*_
*DistributesOver+' = transitive *Commutative (transitive *DistributesOver+ (+WellDefined *Commutative *Commutative))
*Associative' : {a b c : A} ((a * b) * c) (a * (b * c))
*Associative' = symmetric *Associative
identIsIdent' : {a : A} a * 1R a
identIsIdent' = transitive *Commutative identIsIdent