diff -r dd58f13a8eb4 -r eb85850d3eb7 src/HOL/Lambda/Type.thy --- a/src/HOL/Lambda/Type.thy Fri Nov 17 02:19:55 2006 +0100 +++ b/src/HOL/Lambda/Type.thy Fri Nov 17 02:20:03 2006 +0100 @@ -12,7 +12,7 @@ subsection {* Environments *} definition - shift :: "(nat \ 'a) \ nat \ 'a \ nat \ 'a" ("_<_:_>" [90, 0, 0] 91) + shift :: "(nat \ 'a) \ nat \ 'a \ nat \ 'a" ("_<_:_>" [90, 0, 0] 91) where "e = (\j. if j < i then e j else if j = i then a else e (j - 1))" notation (xsymbols) @@ -50,21 +50,23 @@ typings :: "(nat \ type) \ dB list \ type list \ bool" abbreviation - funs :: "type list \ type \ type" (infixr "=>>" 200) + funs :: "type list \ type \ type" (infixr "=>>" 200) where "Ts =>> T == foldr Fun Ts T" - typing_rel :: "(nat \ type) \ dB \ type \ bool" ("_ |- _ : _" [50, 50, 50] 50) +abbreviation + typing_rel :: "(nat \ type) \ dB \ type \ bool" ("_ |- _ : _" [50, 50, 50] 50) where "env |- t : T == (env, t, T) \ typing" +abbreviation typings_rel :: "(nat \ type) \ dB list \ type list \ bool" - ("_ ||- _ : _" [50, 50, 50] 50) + ("_ ||- _ : _" [50, 50, 50] 50) where "env ||- ts : Ts == typings env ts Ts" notation (xsymbols) typing_rel ("_ \ _ : _" [50, 50, 50] 50) notation (latex) - funs (infixr "\" 200) + funs (infixr "\" 200) and typings_rel ("_ \ _ : _" [50, 50, 50] 50) inductive typing