src/HOL/IMP/Expr.thy
author wenzelm
Wed, 19 Dec 2001 00:26:04 +0100
changeset 12546 0c90e581379f
parent 12431 07ec657249e5
child 16417 9bc16273c2d4
permissions -rw-r--r--
tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
     1
(*  Title:      HOL/IMP/Expr.thy
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
     2
    ID:         $Id$
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
     3
    Author:     Heiko Loetzbeyer & Robert Sandner & Tobias Nipkow, TUM
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
     4
    Copyright   1994 TUM
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
     5
*)
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
     6
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
     7
header "Expressions"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
     8
12546
wenzelm
parents: 12431
diff changeset
     9
theory Expr = Main:
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    10
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    11
text {*
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    12
  Arithmetic expressions and Boolean expressions.
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    13
  Not used in the rest of the language, but included for completeness.
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    14
*}
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    15
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    16
subsection "Arithmetic expressions"
12546
wenzelm
parents: 12431
diff changeset
    17
typedecl loc
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    18
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    19
types
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    20
  state = "loc => nat"
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    21
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    22
datatype
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    23
  aexp = N nat
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    24
       | X loc
12546
wenzelm
parents: 12431
diff changeset
    25
       | Op1 "nat => nat" aexp
wenzelm
parents: 12431
diff changeset
    26
       | Op2 "nat => nat => nat" aexp aexp
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    27
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    28
subsection "Evaluation of arithmetic expressions"
1729
e4f8682eea2e Removal of special syntax for -a-> and -b->
paulson
parents: 1697
diff changeset
    29
consts  evala    :: "((aexp*state) * nat) set"
12546
wenzelm
parents: 12431
diff changeset
    30
syntax "_evala"  :: "[aexp*state,nat] => bool"         (infixl "-a->" 50)
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    31
translations
1729
e4f8682eea2e Removal of special syntax for -a-> and -b->
paulson
parents: 1697
diff changeset
    32
    "aesig -a-> n" == "(aesig,n) : evala"
1789
aade046ec6d5 Quotes now optional around inductive set
paulson
parents: 1729
diff changeset
    33
inductive evala
12546
wenzelm
parents: 12431
diff changeset
    34
  intros
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    35
  N:   "(N(n),s) -a-> n"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    36
  X:   "(X(x),s) -a-> s(x)"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    37
  Op1: "(e,s) -a-> n ==> (Op1 f e,s) -a-> f(n)"
12546
wenzelm
parents: 12431
diff changeset
    38
  Op2: "[| (e0,s) -a-> n0;  (e1,s)  -a-> n1 |]
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    39
        ==> (Op2 f e0 e1,s) -a-> f n0 n1"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    40
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    41
lemmas [intro] = N X Op1 Op2
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    42
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    43
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    44
subsection "Boolean expressions"
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    45
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    46
datatype
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    47
  bexp = true
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    48
       | false
12546
wenzelm
parents: 12431
diff changeset
    49
       | ROp  "nat => nat => bool" aexp aexp
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    50
       | noti bexp
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    51
       | andi bexp bexp         (infixl 60)
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    52
       | ori  bexp bexp         (infixl 60)
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    53
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    54
subsection "Evaluation of boolean expressions"
12546
wenzelm
parents: 12431
diff changeset
    55
consts evalb    :: "((bexp*state) * bool)set"
wenzelm
parents: 12431
diff changeset
    56
syntax "_evalb" :: "[bexp*state,bool] => bool"         (infixl "-b->" 50)
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    57
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    58
translations
1729
e4f8682eea2e Removal of special syntax for -a-> and -b->
paulson
parents: 1697
diff changeset
    59
    "besig -b-> b" == "(besig,b) : evalb"
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    60
1789
aade046ec6d5 Quotes now optional around inductive set
paulson
parents: 1729
diff changeset
    61
inductive evalb
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    62
  -- "avoid clash with ML constructors true, false"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    63
  intros
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    64
  tru:   "(true,s) -b-> True"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    65
  fls:   "(false,s) -b-> False"
12546
wenzelm
parents: 12431
diff changeset
    66
  ROp:   "[| (a0,s) -a-> n0; (a1,s) -a-> n1 |]
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    67
          ==> (ROp f a0 a1,s) -b-> f n0 n1"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    68
  noti:  "(b,s) -b-> w ==> (noti(b),s) -b-> (~w)"
12546
wenzelm
parents: 12431
diff changeset
    69
  andi:  "[| (b0,s) -b-> w0; (b1,s) -b-> w1 |]
1729
e4f8682eea2e Removal of special syntax for -a-> and -b->
paulson
parents: 1697
diff changeset
    70
          ==> (b0 andi b1,s) -b-> (w0 & w1)"
12546
wenzelm
parents: 12431
diff changeset
    71
  ori:   "[| (b0,s) -b-> w0; (b1,s) -b-> w1 |]
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    72
          ==> (b0 ori b1,s) -b-> (w0 | w1)"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    73
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    74
lemmas [intro] = tru fls ROp noti andi ori
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    75
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    76
subsection "Denotational semantics of arithmetic and boolean expressions"
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    77
consts
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    78
  A     :: "aexp => state => nat"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    79
  B     :: "bexp => state => bool"
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    80
5183
89f162de39cf Adapted to new datatype package.
berghofe
parents: 5102
diff changeset
    81
primrec
1900
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    82
  "A(N(n)) = (%s. n)"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    83
  "A(X(x)) = (%s. s(x))"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    84
  "A(Op1 f a) = (%s. f(A a s))"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    85
  "A(Op2 f a0 a1) = (%s. f (A a0 s) (A a1 s))"
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    86
5183
89f162de39cf Adapted to new datatype package.
berghofe
parents: 5102
diff changeset
    87
primrec
1900
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    88
  "B(true) = (%s. True)"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    89
  "B(false) = (%s. False)"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    90
  "B(ROp f a0 a1) = (%s. f (A a0 s) (A a1 s))"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    91
  "B(noti(b)) = (%s. ~(B b s))"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    92
  "B(b0 andi b1) = (%s. (B b0 s) & (B b1 s))"
c7a869229091 Simplified primrec definitions.
berghofe
parents: 1789
diff changeset
    93
  "B(b0 ori b1) = (%s. (B b0 s) | (B b1 s))"
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
    94
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    95
lemma [simp]: "(N(n),s) -a-> n' = (n = n')"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    96
  by (rule,cases set: evala) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    97
12546
wenzelm
parents: 12431
diff changeset
    98
lemma [simp]: "(X(x),sigma) -a-> i = (i = sigma x)"
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
    99
  by (rule,cases set: evala) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   100
12546
wenzelm
parents: 12431
diff changeset
   101
lemma   [simp]:
wenzelm
parents: 12431
diff changeset
   102
  "(Op1 f e,sigma) -a-> i = (\<exists>n. i = f n \<and> (e,sigma) -a-> n)"
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   103
  by (rule,cases set: evala) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   104
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   105
lemma [simp]:
12546
wenzelm
parents: 12431
diff changeset
   106
  "(Op2 f a1 a2,sigma) -a-> i =
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   107
  (\<exists>n0 n1. i = f n0 n1 \<and> (a1, sigma) -a-> n0 \<and> (a2, sigma) -a-> n1)"
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   108
  by (rule,cases set: evala) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   109
12546
wenzelm
parents: 12431
diff changeset
   110
lemma [simp]: "((true,sigma) -b-> w) = (w=True)"
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   111
  by (rule,cases set: evalb) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   112
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   113
lemma [simp]:
12546
wenzelm
parents: 12431
diff changeset
   114
  "((false,sigma) -b-> w) = (w=False)"
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   115
  by (rule,cases set: evalb) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   116
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   117
lemma [simp]:
12546
wenzelm
parents: 12431
diff changeset
   118
  "((ROp f a0 a1,sigma) -b-> w) =
wenzelm
parents: 12431
diff changeset
   119
  (? m. (a0,sigma) -a-> m & (? n. (a1,sigma) -a-> n & w = f m n))"
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   120
  by (rule,cases set: evalb) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   121
12546
wenzelm
parents: 12431
diff changeset
   122
lemma [simp]:
wenzelm
parents: 12431
diff changeset
   123
  "((noti(b),sigma) -b-> w) = (? x. (b,sigma) -b-> x & w = (~x))"
wenzelm
parents: 12431
diff changeset
   124
  by (rule,cases set: evalb) auto
wenzelm
parents: 12431
diff changeset
   125
wenzelm
parents: 12431
diff changeset
   126
lemma [simp]:
wenzelm
parents: 12431
diff changeset
   127
  "((b0 andi b1,sigma) -b-> w) =
wenzelm
parents: 12431
diff changeset
   128
  (? x. (b0,sigma) -b-> x & (? y. (b1,sigma) -b-> y & w = (x&y)))"
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   129
  by (rule,cases set: evalb) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   130
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   131
lemma [simp]:
12546
wenzelm
parents: 12431
diff changeset
   132
  "((b0 ori b1,sigma) -b-> w) =
wenzelm
parents: 12431
diff changeset
   133
  (? x. (b0,sigma) -b-> x & (? y. (b1,sigma) -b-> y & w = (x|y)))"
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   134
  by (rule,cases set: evalb) auto
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   135
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   136
12546
wenzelm
parents: 12431
diff changeset
   137
lemma aexp_iff:
wenzelm
parents: 12431
diff changeset
   138
  "!!n. ((a,s) -a-> n) = (A a s = n)"
wenzelm
parents: 12431
diff changeset
   139
  by (induct a) auto
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   140
12546
wenzelm
parents: 12431
diff changeset
   141
lemma bexp_iff:
wenzelm
parents: 12431
diff changeset
   142
  "!!w. ((b,s) -b-> w) = (B b s = w)"
wenzelm
parents: 12431
diff changeset
   143
  by (induct b) (auto simp add: aexp_iff)
12431
07ec657249e5 converted to Isar
kleing
parents: 12338
diff changeset
   144
1697
687f0710c22d Arithemtic and boolean expressions are now in a separate theory.
nipkow
parents:
diff changeset
   145
end