aboutsummaryrefslogtreecommitdiff
path: root/hott/HoTT.thy
blob: 0b3040c83152a56d0811aab0822154c41bbfeca3 (plain)
1
2
3
4
5
6
7
8
9
10
theory HoTT
imports
  Identity
  Equivalence
  More_Types
  Nat

begin

end