aboutsummaryrefslogtreecommitdiff
path: root/HoTT.thy
blob: 724eebc8de98dde6961171a126e3c3664752eb23 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
(*  Title:  HoTT/HoTT.thy
    Author: Josh Chen

Load all the component modules for the HoTT logic.
*)

theory HoTT
imports

(* Basic theories *)
HoTT_Base
HoTT_Methods

(* Types *)
Prod
Sum
Equal
Coprod
Nat

(* Additional properties *)
EqualProps
Proj

begin
end