view and.agda @ 0:d9d5091eb899 draft default tip

Try 'and' definition on agda
author tatsuki
date Tue, 04 Mar 2014 15:04:53 +0900
parents
children
line wrap: on
line source

module and where

postulate U : Set
postulate V : Set
postulate T : Set

f : Set
f = U -> V

record _x_ (U V : Set) : Set where
  field
    pi1 : U
    pi2 : V

postulate <_,_> : U -> V -> (U x V)

open _x_
postulate u : U
postulate v : V

uv : U x V
uv = < u , v >
pair : Set
pair = U x V 


postulate t : T 

x : T 
x = t

data _==_ {A : Set} : A -> A -> Set where 
  refl : {x : A} -> x == x

lemma02 : U
lemma02 = pi1 (< u , v >)
lemma01 : (pi1 ( < u , v > )) == u
lemma01 = {!!}