Quotient-Paper/Paper.thy
changeset 2264 2a95188263ec
parent 2263 d2ca79475103
parent 2262 5ced6472ac3c
child 2265 9c44db3eef95
equal deleted inserted replaced
2263:d2ca79475103 2264:2a95188263ec
   364   @{thm [mode=Rule, display, indent=10] pred_compI[of "R\<^isub>1" "x" "y" "R\<^isub>2" "z"]}
   364   @{thm [mode=Rule, display, indent=10] pred_compI[of "R\<^isub>1" "x" "y" "R\<^isub>2" "z"]}
   365   \end{definition}
   365   \end{definition}
   366 
   366 
   367   \noindent
   367   \noindent
   368   Unfortunately, restrictions in HOL's type-system prevent us from stating
   368   Unfortunately, restrictions in HOL's type-system prevent us from stating
   369   and proving a quotient type theorem, like \ref{funquot}, for compositions 
   369   and proving a quotient type theorem, like Proposition \ref{funquot}, for compositions 
   370   of relations. However, we can prove all instances where @{text R\<^isub>1} and 
   370   of relations. However, we can prove all instances where @{text R\<^isub>1} and 
   371   @{text "R\<^isub>2"} are built up by constituent equivalence relations.
   371   @{text "R\<^isub>2"} are built up by constituent equivalence relations.
   372 *}
   372 *}
   373 
   373 
   374 section {* Quotient Types and Quotient Definitions\label{sec:type} *}
   374 section {* Quotient Types and Quotient Definitions\label{sec:type} *}