view a02/agda/level1.agda @ 266:e5cf49902db3

...
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Wed, 17 Nov 2021 16:12:30 +0900
parents 7a0634a7c25a
children
line wrap: on
line source

module level1 where

open import Level

ex1 : { A B : Set} → Set
ex1 {A} {B} =  A → B

ex2 : { A B : Set} →  ( A → B ) → Set
ex2 {A} {B}  A→B  =  ex1 {A} {B}

ex7 : {A B : Set} → Set _
ex7 {A} {B} = lemma2 ( A → B ) _ -- → A → B


-- record FuncBad (A B : Set) : Set where
--   field
--      func : A → B → Set

record Func {n : Level} (A B : Set n ) : Set (suc n) where
  field
    func :  A → B  → Set n

record Func2 {n : Level} (A B : Set n ) : Set {!!} where
  field
    func : A → B  → Func A B