doc-src/IsarImplementation/Thy/unused.thy
changeset 20470 c839b38a1f32
parent 20460 351c63bb2704
child 20474 af069653f1d7
equal deleted inserted replaced
20469:bb75c1cdf913 20470:c839b38a1f32
     1 
     1 
     2 text {*
     2 text {*
       
     3 
       
     4   
       
     5 
       
     6   A \emph{fixed variable} acts like a local constant in the current
       
     7   context, representing some simple type @{text "\<alpha>"}, or some value
       
     8   @{text "x: \<tau>"} (for a fixed type expression @{text "\<tau>"}).  A
       
     9   \emph{schematic variable} acts like a placeholder for arbitrary
       
    10   elements, similar to outermost quantification.  The division between
       
    11   fixed and schematic variables tells which abstract entities are
       
    12   inside and outside the current context.
       
    13 
     3 
    14 
     4   @{index_ML Variable.trade: "Proof.context -> (thm list -> thm list) -> thm list -> thm list"} \\
    15   @{index_ML Variable.trade: "Proof.context -> (thm list -> thm list) -> thm list -> thm list"} \\
     5 
    16 
     6 
    17 
     7 
    18