src/ZF/Coind/ECR.thy
author paulson
Wed, 02 Apr 1997 15:26:52 +0200
changeset 2871 ba585d52ea4e
parent 1478 2b8c2a7547ab
child 6117 f9aad8ccd590
permissions -rw-r--r--
Now checks for existence of theory Inductive (Fixedpt was too small)
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     1
(*  Title:      ZF/Coind/ECR.thy
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     2
    ID:         $Id$
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     3
    Author:     Jacob Frost, Cambridge University Computer Laboratory
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     4
    Copyright   1995  University of Cambridge
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     5
*)
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     6
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     7
ECR = Static + Dynamic +
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     8
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     9
(* The extended correspondence relation *)
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    10
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    11
consts
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 1155
diff changeset
    12
  HasTyRel :: i
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    13
coinductive
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    14
  domains "HasTyRel" <= "Val * Ty"
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    15
  intrs
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    16
    htr_constI
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    17
      "[| c:Const; t:Ty; isof(c,t) |] ==> <v_const(c),t>:HasTyRel"
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    18
    htr_closI
1155
928a16e02f9f removed \...\ inside strings
clasohm
parents: 930
diff changeset
    19
      "[| x:ExVar; e:Exp; t:Ty; ve:ValEnv; te:TyEnv; 
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
    20
          <te,e_fn(x,e),t>:ElabRel;  
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
    21
          ve_dom(ve) = te_dom(te);   
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
    22
          {<ve_app(ve,y),te_app(te,y)>.y:ve_dom(ve)}:Pow(HasTyRel)  
1155
928a16e02f9f removed \...\ inside strings
clasohm
parents: 930
diff changeset
    23
      |] ==>   
928a16e02f9f removed \...\ inside strings
clasohm
parents: 930
diff changeset
    24
      <v_clos(x,e,ve),t>:HasTyRel" 
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    25
  monos "[Pow_mono]"
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    26
  type_intrs "Val_ValEnv.intrs"
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    27
  
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    28
(* Pointwise extension to environments *)
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    29
 
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    30
consts
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 1155
diff changeset
    31
  hastyenv :: [i,i] => o
930
63f02d32509e Replaced rules by defs
lcp
parents: 915
diff changeset
    32
defs
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    33
  hastyenv_def 
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
    34
    " hastyenv(ve,te) ==                        
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
    35
     ve_dom(ve) = te_dom(te) &          
1155
928a16e02f9f removed \...\ inside strings
clasohm
parents: 930
diff changeset
    36
     (ALL x:ve_dom(ve). <ve_app(ve,x),te_app(te,x)>:HasTyRel)"
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    37
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    38
end