src/ZF/Coind/Static.thy
author paulson
Tue, 19 Jan 1999 11:18:11 +0100
changeset 6141 a6922171b396
parent 1478 2b8c2a7547ab
child 11318 6536fb8c9fc6
permissions -rw-r--r--
removal of the (thm list) argument of mk_cases

(*  Title:      ZF/Coind/Static.thy
    ID:         $Id$
    Author:     Jacob Frost, Cambridge University Computer Laboratory
    Copyright   1995  University of Cambridge
*)

Static = BCR +

consts  ElabRel :: i

inductive
  domains "ElabRel" <= "TyEnv * Exp * Ty"
  intrs
    constI
      " [| te:TyEnv; c:Const; t:Ty; isof(c,t) |] ==>   
       <te,e_const(c),t>:ElabRel "
    varI
      " [| te:TyEnv; x:ExVar; x:te_dom(te) |] ==>   
       <te,e_var(x),te_app(te,x)>:ElabRel "
    fnI
      " [| te:TyEnv; x:ExVar; e:Exp; t1:Ty; t2:Ty;   
          <te_owr(te,x,t1),e,t2>:ElabRel |] ==>   
       <te,e_fn(x,e),t_fun(t1,t2)>:ElabRel "
    fixI
      " [| te:TyEnv; f:ExVar; x:ExVar; t1:Ty; t2:Ty;   
          <te_owr(te_owr(te,f,t_fun(t1,t2)),x,t1),e,t2>:ElabRel |] ==>   
       <te,e_fix(f,x,e),t_fun(t1,t2)>:ElabRel "
    appI
      " [| te:TyEnv; e1:Exp; e2:Exp; t1:Ty; t2:Ty;   
          <te,e1,t_fun(t1,t2)>:ElabRel;   
          <te,e2,t1>:ElabRel |] ==>   
       <te,e_app(e1,e2),t2>:ElabRel "
  type_intrs "te_appI::Exp.intrs@Ty.intrs"

end