Lots of speedups (#116)

This commit is contained in:
Patrick Stevens
2020-04-16 13:41:51 +01:00
committed by GitHub
parent 1bcb3f8537
commit 9b80058157
63 changed files with 1082 additions and 564 deletions

View File

@@ -25,10 +25,10 @@ open Setoid S
open Equivalence eq
open import Rings.Lemmas R
open import Groups.Lemmas additiveGroup
open import Groups.Cyclic.Definition additiveGroup
fromN : A
fromN zero = 0R
fromN (succ n) = 1R + fromN n
fromN = positiveEltPower 1R
fromNPreserves+ : (a b : ) fromN (a +N b) (fromN a) + (fromN b)
fromNPreserves+ zero b = symmetric identLeft