src/Doc/Isar_Ref/Inner_Syntax.thy
changeset 60254 52110106c0ca
parent 59783 00b62aa9f430
child 60270 a147272b16f9
equal deleted inserted replaced
60253:478795f6e78a 60254:52110106c0ca
  1021   information still missing.  Explicit type constraints might be given by
  1021   information still missing.  Explicit type constraints might be given by
  1022   the user, or implicit position information by the system --- both
  1022   the user, or implicit position information by the system --- both
  1023   need to be passed-through carefully by syntax transformations.
  1023   need to be passed-through carefully by syntax transformations.
  1024 
  1024 
  1025   Pre-terms are further processed by the so-called \emph{check} and
  1025   Pre-terms are further processed by the so-called \emph{check} and
  1026   \emph{unckeck} phases that are intertwined with type-inference (see
  1026   \emph{uncheck} phases that are intertwined with type-inference (see
  1027   also @{cite "isabelle-implementation"}).  The latter allows to operate
  1027   also @{cite "isabelle-implementation"}).  The latter allows to operate
  1028   on higher-order abstract syntax with proper binding and type
  1028   on higher-order abstract syntax with proper binding and type
  1029   information already available.
  1029   information already available.
  1030 
  1030 
  1031   As a rule of thumb, anything that manipulates bindings of variables
  1031   As a rule of thumb, anything that manipulates bindings of variables