src/Doc/Implementation/Logic.thy
changeset 56579 4c94f631c595
parent 56420 b266e7a86485
child 58555 7975676c08c0
equal deleted inserted replaced
56578:e73723b39c82 56579:4c94f631c595
   295   variables.  Subsequently, we shall use the latter notation instead
   295   variables.  Subsequently, we shall use the latter notation instead
   296   of internal de-Bruijn representation.
   296   of internal de-Bruijn representation.
   297 
   297 
   298   The inductive relation @{text "t :: \<tau>"} assigns a (unique) type to a
   298   The inductive relation @{text "t :: \<tau>"} assigns a (unique) type to a
   299   term according to the structure of atomic terms, abstractions, and
   299   term according to the structure of atomic terms, abstractions, and
   300   applicatins:
   300   applications:
   301   \[
   301   \[
   302   \infer{@{text "a\<^sub>\<tau> :: \<tau>"}}{}
   302   \infer{@{text "a\<^sub>\<tau> :: \<tau>"}}{}
   303   \qquad
   303   \qquad
   304   \infer{@{text "(\<lambda>x\<^sub>\<tau>. t) :: \<tau> \<Rightarrow> \<sigma>"}}{@{text "t :: \<sigma>"}}
   304   \infer{@{text "(\<lambda>x\<^sub>\<tau>. t) :: \<tau> \<Rightarrow> \<sigma>"}}{@{text "t :: \<sigma>"}}
   305   \qquad
   305   \qquad