Theory CZH_SMC_Introduction
chapter‹Semicategories›
section‹Introduction›
theory CZH_SMC_Introduction
imports CZH_DG_Introduction
begin
subsection‹Background›
text‹
Many concepts that are normally associated with category theory can be
generalized to semicategories. It is the goal of
this chapter to expose these generalized concepts and provide a
foundation for the development of the notion of a category
in \<^cite>‹"milehins_category_2021"›.
›
subsection‹Preliminaries›
named_theorems smc_op_simps
named_theorems smc_op_intros
named_theorems smc_cs_simps
named_theorems smc_cs_intros
named_theorems smc_arrow_cs_intros
subsection‹CS setup for foundations›
lemmas (in 𝒵) [smc_cs_intros] = 𝒵_β
text‹\newpage›
end