Mercurial > hg > Members > kono > Proof > category
diff src/list-nat0.agda @ 1124:f683d96fbc93 default tip
safe fix done
author | Shinji KONO <kono@ie.u-ryukyu.ac.jp> |
---|---|
date | Sun, 07 Jul 2024 22:28:50 +0900 |
parents | ac53803b3b2a |
children |
line wrap: on
line diff
--- a/src/list-nat0.agda Sun Jul 07 17:05:16 2024 +0900 +++ b/src/list-nat0.agda Sun Jul 07 22:28:50 2024 +0900 @@ -1,11 +1,12 @@ +{-# OPTIONS --cubical-compatible --safe #-} module list-nat0 where open import Level - -postulate a : Set -postulate b : Set -postulate c : Set +data i3 : Set where + a : i3 + b : i3 + c : i3 infixr 40 _::_ @@ -59,8 +60,8 @@ ( f : A → B ) → {x : A } → {y : A} → x ≡ y → f x ≡ f y cong1 f refl = refl -lemma11 : ∀{n} → ( Set n ) IsRelatedTo ( Set n ) -lemma11 = relTo refl +-- lemma11 : ∀{n} → ( Set n ) IsRelatedTo ( Set n ) +-- lemma11 = relTo refl lemma12 : {L : Set} ( x : List L ) → x ++ x ≡ x ++ x lemma12 x = begin x ++ x ∎