src/HOL/IMP/AExp.thy
author nipkow
Mon, 20 Aug 2018 20:54:26 +0200
changeset 68776 403dd13cf6e9
parent 67406 23307fd33906
child 69505 cc2d676d5395
permissions -rw-r--r--
avoid session qualification because no tex is generated when used; tuned sectioning
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
58889
5b7a9633cfa8 modernized header uniformly as section;
wenzelm
parents: 58310
diff changeset
     1
section "Arithmetic and Boolean Expressions"
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
     2
68776
403dd13cf6e9 avoid session qualification because no tex is generated when used;
nipkow
parents: 67406
diff changeset
     3
subsection "Arithmetic Expressions"
403dd13cf6e9 avoid session qualification because no tex is generated when used;
nipkow
parents: 67406
diff changeset
     4
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
     5
theory AExp imports Main begin
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
     6
45212
e87feee00a4c renamed name -> vname
nipkow
parents: 45015
diff changeset
     7
type_synonym vname = string
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
     8
type_synonym val = int
45212
e87feee00a4c renamed name -> vname
nipkow
parents: 45015
diff changeset
     9
type_synonym state = "vname \<Rightarrow> val"
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    10
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    11
text_raw\<open>\snip{AExpaexpdef}{2}{1}{%\<close>
58310
91ea607a34d8 updated news
blanchet
parents: 58249
diff changeset
    12
datatype aexp = N int | V vname | Plus aexp aexp
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    13
text_raw\<open>}%endsnip\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    14
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    15
text_raw\<open>\snip{AExpavaldef}{1}{2}{%\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    16
fun aval :: "aexp \<Rightarrow> state \<Rightarrow> val" where
45216
nipkow
parents: 45212
diff changeset
    17
"aval (N n) s = n" |
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    18
"aval (V x) s = s x" |
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    19
"aval (Plus a\<^sub>1 a\<^sub>2) s = aval a\<^sub>1 s + aval a\<^sub>2 s"
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    20
text_raw\<open>}%endsnip\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    21
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    22
44923
b80108b346a9 cleand up AbsInt fixpoint iteration; tuned syntax
nipkow
parents: 44036
diff changeset
    23
value "aval (Plus (V ''x'') (N 5)) (\<lambda>x. if x = ''x'' then 7 else 0)"
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    24
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    25
text \<open>The same state more concisely:\<close>
44923
b80108b346a9 cleand up AbsInt fixpoint iteration; tuned syntax
nipkow
parents: 44036
diff changeset
    26
value "aval (Plus (V ''x'') (N 5)) ((\<lambda>x. 0) (''x'':= 7))"
43158
686fa0a0696e imported rest of new IMP
kleing
parents: 43141
diff changeset
    27
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    28
text \<open>A little syntax magic to write larger states compactly:\<close>
43158
686fa0a0696e imported rest of new IMP
kleing
parents: 43141
diff changeset
    29
44923
b80108b346a9 cleand up AbsInt fixpoint iteration; tuned syntax
nipkow
parents: 44036
diff changeset
    30
definition null_state ("<>") where
b80108b346a9 cleand up AbsInt fixpoint iteration; tuned syntax
nipkow
parents: 44036
diff changeset
    31
  "null_state \<equiv> \<lambda>x. 0"
44036
d03f9f28d01d new state syntax with less conflicts
kleing
parents: 43250
diff changeset
    32
syntax 
d03f9f28d01d new state syntax with less conflicts
kleing
parents: 43250
diff changeset
    33
  "_State" :: "updbinds => 'a" ("<_>")
43158
686fa0a0696e imported rest of new IMP
kleing
parents: 43141
diff changeset
    34
translations
51040
faf7f0d4f9eb tuned state display
nipkow
parents: 49191
diff changeset
    35
  "_State ms" == "_Update <> ms"
54289
5a1be63f32cf Add output translation for <a := .., b := .., ..> state notation.
kleing
parents: 54252
diff changeset
    36
  "_State (_updbinds b bs)" <= "_Update (_State b) bs"
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    37
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    38
text \<open>\noindent
43158
686fa0a0696e imported rest of new IMP
kleing
parents: 43141
diff changeset
    39
  We can now write a series of updates to the function @{text "\<lambda>x. 0"} compactly:
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    40
\<close>
54252
a4a00347e59f use int example like in the rest of IMP (instead of nat)
kleing
parents: 53015
diff changeset
    41
lemma "<a := 1, b := 2> = (<> (a := 1)) (b := (2::int))"
43158
686fa0a0696e imported rest of new IMP
kleing
parents: 43141
diff changeset
    42
  by (rule refl)
686fa0a0696e imported rest of new IMP
kleing
parents: 43141
diff changeset
    43
44036
d03f9f28d01d new state syntax with less conflicts
kleing
parents: 43250
diff changeset
    44
value "aval (Plus (V ''x'') (N 5)) <''x'' := 7>"
43158
686fa0a0696e imported rest of new IMP
kleing
parents: 43141
diff changeset
    45
44923
b80108b346a9 cleand up AbsInt fixpoint iteration; tuned syntax
nipkow
parents: 44036
diff changeset
    46
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    47
text \<open>In  the @{term[source] "<a := b>"} syntax, variables that are not mentioned are 0 by default:
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    48
\<close>
44036
d03f9f28d01d new state syntax with less conflicts
kleing
parents: 43250
diff changeset
    49
value "aval (Plus (V ''x'') (N 5)) <''y'' := 7>"
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    50
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    51
text\<open>Note that this @{text"<\<dots>>"} syntax works for any function space
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    52
@{text"\<tau>\<^sub>1 \<Rightarrow> \<tau>\<^sub>2"} where @{text "\<tau>\<^sub>2"} has a @{text 0}.\<close>
44923
b80108b346a9 cleand up AbsInt fixpoint iteration; tuned syntax
nipkow
parents: 44036
diff changeset
    53
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    54
45255
nipkow
parents: 45246
diff changeset
    55
subsection "Constant Folding"
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    56
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    57
text\<open>Evaluate constant subsexpressions:\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    58
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    59
text_raw\<open>\snip{AExpasimpconstdef}{0}{2}{%\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    60
fun asimp_const :: "aexp \<Rightarrow> aexp" where
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    61
"asimp_const (N n) = N n" |
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    62
"asimp_const (V x) = V x" |
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    63
"asimp_const (Plus a\<^sub>1 a\<^sub>2) =
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    64
  (case (asimp_const a\<^sub>1, asimp_const a\<^sub>2) of
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    65
    (N n\<^sub>1, N n\<^sub>2) \<Rightarrow> N(n\<^sub>1+n\<^sub>2) |
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    66
    (b\<^sub>1,b\<^sub>2) \<Rightarrow> Plus b\<^sub>1 b\<^sub>2)"
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    67
text_raw\<open>}%endsnip\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    68
45238
nipkow
parents: 45216
diff changeset
    69
theorem aval_asimp_const:
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    70
  "aval (asimp_const a) s = aval a s"
45015
fdac1e9880eb Updated IMP to use new induction method
nipkow
parents: 44923
diff changeset
    71
apply(induction a)
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    72
apply (auto split: aexp.split)
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    73
done
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    74
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    75
text\<open>Now we also eliminate all occurrences 0 in additions. The standard
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    76
method: optimized versions of the constructors:\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    77
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    78
text_raw\<open>\snip{AExpplusdef}{0}{2}{%\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    79
fun plus :: "aexp \<Rightarrow> aexp \<Rightarrow> aexp" where
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    80
"plus (N i\<^sub>1) (N i\<^sub>2) = N(i\<^sub>1+i\<^sub>2)" |
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    81
"plus (N i) a = (if i=0 then a else Plus (N i) a)" |
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    82
"plus a (N i) = (if i=0 then a else Plus a (N i))" |
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    83
"plus a\<^sub>1 a\<^sub>2 = Plus a\<^sub>1 a\<^sub>2"
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    84
text_raw\<open>}%endsnip\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    85
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    86
lemma aval_plus[simp]:
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    87
  "aval (plus a1 a2) s = aval a1 s + aval a2 s"
45015
fdac1e9880eb Updated IMP to use new induction method
nipkow
parents: 44923
diff changeset
    88
apply(induction a1 a2 rule: plus.induct)
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    89
apply simp_all (* just for a change from auto *)
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    90
done
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    91
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    92
text_raw\<open>\snip{AExpasimpdef}{2}{0}{%\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    93
fun asimp :: "aexp \<Rightarrow> aexp" where
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    94
"asimp (N n) = N n" |
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    95
"asimp (V x) = V x" |
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52460
diff changeset
    96
"asimp (Plus a\<^sub>1 a\<^sub>2) = plus (asimp a\<^sub>1) (asimp a\<^sub>2)"
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    97
text_raw\<open>}%endsnip\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
    98
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
    99
text\<open>Note that in @{const asimp_const} the optimized constructor was
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   100
inlined. Making it a separate function @{const plus} improves modularity of
67406
23307fd33906 isabelle update_cartouches -c;
wenzelm
parents: 58889
diff changeset
   101
the code and the proofs.\<close>
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   102
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   103
value "asimp (Plus (Plus (N 0) (N 0)) (Plus (V ''x'') (N 0)))"
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   104
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   105
theorem aval_asimp[simp]:
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   106
  "aval (asimp a) s = aval a s"
45015
fdac1e9880eb Updated IMP to use new induction method
nipkow
parents: 44923
diff changeset
   107
apply(induction a)
43141
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   108
apply simp_all
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   109
done
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   110
11fce8564415 Replacing old IMP with new Semantics material
nipkow
parents:
diff changeset
   111
end