ProgTutorial/Advanced.thy
changeset 481 32323727af96
parent 475 25371f74c768
child 484 490fe9483c0d
equal deleted inserted replaced
480:ae49c5e8868e 481:32323727af96
   185   \end{isabelle}
   185   \end{isabelle}
   186 
   186 
   187   The simplest morphism is the  @{ML_ind identity in Morphism}-morphism defined as
   187   The simplest morphism is the  @{ML_ind identity in Morphism}-morphism defined as
   188 *}
   188 *}
   189 
   189 
   190 ML{*val identity = Morphism.morphism {binding = I, typ = I, term = I, fact = I}*}
   190 ML{*val identity = Morphism.morphism {binding = [], typ = [], term = [], fact = []}*}
   191   
   191   
   192 text {*
   192 text {*
   193   Morphisms can be composed with the function @{ML_ind "$>" in Morphism}
   193   Morphisms can be composed with the function @{ML_ind "$>" in Morphism}
   194 *}
   194 *}
   195 
   195