Unicode.agda 887 B

12345678910111213141516171819202122232425262728293031323334353637
  1. -- Agda supports full unicode everywhere. An Agda file should be written using
  2. -- the UTF-8 encoding.
  3. module Introduction.Unicode where
  4. module ユーニコード where
  5. data _∧_ (P Q : Prop) : Prop where
  6. ∧-intro : P -> Q -> P ∧ Q
  7. ∧-elim₁ : {P Q : Prop} -> P ∧ Q -> P
  8. ∧-elim₁ (∧-intro p _) = p
  9. ∧-elim₂ : {P Q : Prop} -> P ∧ Q -> Q
  10. ∧-elim₂ (∧-intro _ q) = q
  11. data _∨_ (P Q : Prop) : Prop where
  12. ∨-intro₁ : P -> P ∨ Q
  13. ∨-intro₂ : Q -> P ∨ Q
  14. ∨-elim : {P Q R : Prop} -> (P -> R) -> (Q -> R) -> P ∨ Q -> R
  15. ∨-elim f g (∨-intro₁ p) = f p
  16. ∨-elim f g (∨-intro₂ q) = g q
  17. data ⊥ : Prop where
  18. data ⊤ : Prop where
  19. ⊤-intro : ⊤
  20. data ¬_ (P : Prop) : Prop where
  21. ¬-intro : (P -> ⊥) -> ¬ P
  22. data ∏ {A : Set}(P : A -> Prop) : Prop where
  23. ∏-intro : ((x : A) -> P x) -> ∏ P