Integer.agda 119 B

12345
  1. {-# OPTIONS --without-K #-}
  2. module Common.Integer where
  3. open import Agda.Builtin.Int public renaming (Int to Integer)