src/HOLCF/Fixrec.thy
author huffman
Mon, 07 Nov 2005 23:33:01 +0100
changeset 18112 dc1d6f588204
parent 18110 08ec4f1f116d
child 18293 4eaa654c92f2
permissions -rw-r--r--
reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     1
(*  Title:      HOLCF/Fixrec.thy
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     2
    ID:         $Id$
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     3
    Author:     Amber Telfer and Brian Huffman
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     4
*)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     5
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     6
header "Package for defining recursive functions in HOLCF"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     7
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
     8
theory Fixrec
16551
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
     9
imports Sprod Ssum Up One Tr Fix
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 16401
diff changeset
    10
uses ("fixrec_package.ML")
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    11
begin
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    12
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    13
subsection {* Maybe monad type *}
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    14
16776
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
    15
defaultsort cpo
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
    16
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    17
types 'a maybe = "one ++ 'a u"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    18
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    19
constdefs
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    20
  fail :: "'a maybe"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    21
  "fail \<equiv> sinl\<cdot>ONE"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    22
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    23
  return :: "'a \<rightarrow> 'a maybe"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    24
  "return \<equiv> sinr oo up"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    25
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    26
lemma maybeE:
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    27
  "\<lbrakk>p = \<bottom> \<Longrightarrow> Q; p = fail \<Longrightarrow> Q; \<And>x. p = return\<cdot>x \<Longrightarrow> Q\<rbrakk> \<Longrightarrow> Q"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    28
apply (unfold fail_def return_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    29
apply (rule_tac p=p in ssumE, simp)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    30
apply (rule_tac p=x in oneE, simp, simp)
16754
1b979f8b7e8e renamed upE1 to upE
huffman
parents: 16551
diff changeset
    31
apply (rule_tac p=y in upE, simp, simp)
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    32
done
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    33
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    34
subsubsection {* Monadic bind operator *}
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    35
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    36
constdefs
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    37
  bind :: "'a maybe \<rightarrow> ('a \<rightarrow> 'b maybe) \<rightarrow> 'b maybe"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    38
  "bind \<equiv> \<Lambda> m f. sscase\<cdot>sinl\<cdot>(fup\<cdot>f)\<cdot>m"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    39
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    40
syntax ">>=" :: "['a maybe, 'a \<rightarrow> 'b maybe] \<Rightarrow> 'b maybe" (infixl ">>=" 50)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    41
translations "m >>= f" == "bind\<cdot>m\<cdot>f"
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    42
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    43
nonterminals
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    44
  maybebind maybebinds
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    45
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    46
syntax 
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    47
  "_MBIND"  :: "pttrn \<Rightarrow> 'a maybe \<Rightarrow> maybebind"         ("(2_ <-/ _)" 10)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    48
  ""        :: "maybebind \<Rightarrow> maybebinds"                ("_")
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    49
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    50
  "_MBINDS" :: "[maybebind, maybebinds] \<Rightarrow> maybebinds"  ("_;/ _")
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    51
  "_MDO"    :: "[maybebinds, 'a maybe] \<Rightarrow> 'a maybe"     ("(do _;/ (_))" 10)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    52
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    53
translations
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    54
  "_MDO (_MBINDS b bs) e" == "_MDO b (_MDO bs e)"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    55
  "do (x,y) <- m; e" == "m >>= (LAM <x,y>. e)" 
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    56
  "do x <- m; e"            == "m >>= (LAM x. e)"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    57
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    58
text {* monad laws *}
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    59
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    60
lemma bind_strict [simp]: "UU >>= f = UU"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    61
by (simp add: bind_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    62
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    63
lemma bind_fail [simp]: "fail >>= f = fail"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    64
by (simp add: bind_def fail_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    65
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    66
lemma left_unit [simp]: "(return\<cdot>a) >>= k = k\<cdot>a"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    67
by (simp add: bind_def return_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    68
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    69
lemma right_unit [simp]: "m >>= return = m"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    70
by (rule_tac p=m in maybeE, simp_all)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    71
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    72
lemma bind_assoc [simp]:
16779
ac1dc3d4746a changed orientation of bind_assoc rule
huffman
parents: 16776
diff changeset
    73
 "(do b <- (do a <- m; k\<cdot>a); h\<cdot>b) = (do a <- m; b <- k\<cdot>a; h\<cdot>b)"
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    74
by (rule_tac p=m in maybeE, simp_all)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    75
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    76
subsubsection {* Run operator *}
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    77
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    78
constdefs
16776
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
    79
  run:: "'a::pcpo maybe \<rightarrow> 'a"
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    80
  "run \<equiv> sscase\<cdot>\<bottom>\<cdot>(fup\<cdot>ID)"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    81
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    82
text {* rewrite rules for run *}
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    83
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    84
lemma run_strict [simp]: "run\<cdot>\<bottom> = \<bottom>"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    85
by (simp add: run_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    86
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    87
lemma run_fail [simp]: "run\<cdot>fail = \<bottom>"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    88
by (simp add: run_def fail_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    89
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    90
lemma run_return [simp]: "run\<cdot>(return\<cdot>x) = x"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    91
by (simp add: run_def return_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    92
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    93
subsubsection {* Monad plus operator *}
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
    94
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    95
constdefs
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    96
  mplus :: "'a maybe \<rightarrow> 'a maybe \<rightarrow> 'a maybe"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    97
  "mplus \<equiv> \<Lambda> m1 m2. sscase\<cdot>(\<Lambda> x. m2)\<cdot>(fup\<cdot>return)\<cdot>m1"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    98
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
    99
syntax "+++" :: "['a maybe, 'a maybe] \<Rightarrow> 'a maybe" (infixr "+++" 65)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   100
translations "m1 +++ m2" == "mplus\<cdot>m1\<cdot>m2"
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   101
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   102
text {* rewrite rules for mplus *}
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   103
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   104
lemma mplus_strict [simp]: "\<bottom> +++ m = \<bottom>"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   105
by (simp add: mplus_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   106
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   107
lemma mplus_fail [simp]: "fail +++ m = m"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   108
by (simp add: mplus_def fail_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   109
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   110
lemma mplus_return [simp]: "return\<cdot>x +++ m = return\<cdot>x"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   111
by (simp add: mplus_def return_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   112
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   113
lemma mplus_fail2 [simp]: "m +++ fail = m"
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   114
by (rule_tac p=m in maybeE, simp_all)
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   115
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   116
lemma mplus_assoc: "(x +++ y) +++ z = x +++ (y +++ z)"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   117
by (rule_tac p=x in maybeE, simp_all)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   118
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   119
subsubsection {* Fatbar combinator *}
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   120
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   121
constdefs
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   122
  fatbar :: "('a \<rightarrow> 'b maybe) \<rightarrow> ('a \<rightarrow> 'b maybe) \<rightarrow> ('a \<rightarrow> 'b maybe)"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   123
  "fatbar \<equiv> \<Lambda> a b x. a\<cdot>x +++ b\<cdot>x"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   124
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   125
syntax
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   126
  "\<parallel>" :: "['a \<rightarrow> 'b maybe, 'a \<rightarrow> 'b maybe] \<Rightarrow> 'a \<rightarrow> 'b maybe" (infixr "\<parallel>" 60)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   127
translations
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   128
  "m1 \<parallel> m2" == "fatbar\<cdot>m1\<cdot>m2"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   129
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   130
lemma fatbar1: "m\<cdot>x = \<bottom> \<Longrightarrow> (m \<parallel> ms)\<cdot>x = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   131
by (simp add: fatbar_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   132
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   133
lemma fatbar2: "m\<cdot>x = fail \<Longrightarrow> (m \<parallel> ms)\<cdot>x = ms\<cdot>x"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   134
by (simp add: fatbar_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   135
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   136
lemma fatbar3: "m\<cdot>x = return\<cdot>y \<Longrightarrow> (m \<parallel> ms)\<cdot>x = return\<cdot>y"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   137
by (simp add: fatbar_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   138
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   139
lemmas fatbar_simps = fatbar1 fatbar2 fatbar3
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   140
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   141
lemma run_fatbar1: "m\<cdot>x = \<bottom> \<Longrightarrow> run\<cdot>((m \<parallel> ms)\<cdot>x) = \<bottom>"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   142
by (simp add: fatbar_def)
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   143
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   144
lemma run_fatbar2: "m\<cdot>x = fail \<Longrightarrow> run\<cdot>((m \<parallel> ms)\<cdot>x) = run\<cdot>(ms\<cdot>x)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   145
by (simp add: fatbar_def)
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   146
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   147
lemma run_fatbar3: "m\<cdot>x = return\<cdot>y \<Longrightarrow> run\<cdot>((m \<parallel> ms)\<cdot>x) = y"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   148
by (simp add: fatbar_def)
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   149
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   150
lemmas run_fatbar_simps [simp] = run_fatbar1 run_fatbar2 run_fatbar3
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   151
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   152
subsection {* Pattern combinators *}
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   153
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   154
types ('a,'b,'c) pat = "'b \<rightarrow> 'a \<rightarrow> 'c maybe"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   155
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   156
constdefs
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   157
  wild_pat :: "('a, 'b, 'b) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   158
  "wild_pat \<equiv> \<Lambda> r a. return\<cdot>r"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   159
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   160
  var_pat :: "('a, 'a \<rightarrow> 'b, 'b) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   161
  "var_pat \<equiv> \<Lambda> r a. return\<cdot>(r\<cdot>a)"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   162
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   163
lemma wild_pat [simp]: "wild_pat\<cdot>r\<cdot>a = return\<cdot>r"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   164
by (simp add: wild_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   165
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   166
lemma var_pat [simp]: "var_pat\<cdot>r\<cdot>a = return\<cdot>(r\<cdot>a)"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   167
by (simp add: var_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   168
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   169
subsection {* Case syntax *}
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   170
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   171
nonterminals
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   172
  Case_syn  Cases_syn
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   173
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   174
syntax
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   175
  "_Case_syntax":: "['a, Cases_syn] => 'b"               ("(Case _ of/ _)" 10)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   176
  "_Case1"      :: "['a, 'b] => Case_syn"                ("(2_ =>/ _)" 10)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   177
  ""            :: "Case_syn => Cases_syn"               ("_")
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   178
  "_Case2"      :: "[Case_syn, Cases_syn] => Cases_syn"  ("_/ | _")
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   179
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   180
syntax (xsymbols)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   181
  "_Case1"      :: "['a, 'b] => Case_syn"                ("(2_ \<Rightarrow>/ _)" 10)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   182
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   183
text {* Intermediate tags for parsing/printing *}
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   184
syntax
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   185
  "_pat" :: "'a"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   186
  "_var" :: "'a"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   187
  "_match" :: "'a"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   188
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   189
text {* Parsing Case expressions *}
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   190
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   191
translations
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   192
  "_Case_syntax x cs" => "run\<cdot>(cs\<cdot>x)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   193
  "_Case2 c cs" => "fatbar\<cdot>c\<cdot>cs"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   194
  "_Case1 p r" => "_match (_var p) r"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   195
  "_var _" => "wild_pat"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   196
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   197
parse_translation {*
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   198
  let
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   199
    fun capp (t,u) = Syntax.const "Rep_CFun" $ t $ u;
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   200
    fun cabs (x,t) = (snd (mk_binder_tr ("_cabs", "Abs_CFun"))) [x,t];
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   201
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   202
    fun get_vars (Const ("_var",_) $ x) = [x]
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   203
    |   get_vars (t $ u) = get_vars t @ get_vars u
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   204
    |   get_vars t = [];
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   205
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   206
    fun rem_vars (Const ("_var",_) $ x) = Syntax.const "var_pat"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   207
    |   rem_vars (t $ u) = rem_vars t $ rem_vars u
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   208
    |   rem_vars t = t;
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   209
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   210
    fun match_tr [pat, rhs] =
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   211
          capp (rem_vars pat, foldr cabs rhs (get_vars pat))
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   212
    |   match_tr ts = raise TERM ("match_tr", ts);
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   213
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   214
  in [("_match", match_tr)] end;
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   215
*}
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   216
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   217
text {* Printing Case expressions *}
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   218
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   219
translations
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   220
  "_" <= "_pat wild_pat"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   221
  "x" <= "_pat (_var x)"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   222
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   223
print_translation {*
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   224
  let
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   225
    fun dest_cabs (Const ("Abs_CFun",_) $ t) =
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   226
          let val abs = case t of Abs abs => abs
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   227
                  | _ => ("x", dummyT, incr_boundvars 1 t $ Bound 0);
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   228
          in atomic_abs_tr' abs end
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   229
    |   dest_cabs _ = raise Match; (* too few vars: abort translation *)
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   230
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   231
    fun put_vars (Const ("var_pat",_), rhs) =
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   232
          let val (x, rhs') = dest_cabs rhs;
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   233
          in (Syntax.const "_var" $ x, rhs') end
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   234
    |   put_vars (t $ u, rhs) =
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   235
          let
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   236
            val (t', rhs') = put_vars (t,rhs);
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   237
            val (u', rhs'') = put_vars (u,rhs');
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   238
          in (t' $ u', rhs'') end
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   239
    |   put_vars (t, rhs) = (t, rhs);
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   240
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   241
    fun Case1_tr' (_ $ pat $ rhs) = let
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   242
          val (pat', rhs') = put_vars (pat, rhs);
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   243
        in Syntax.const "_Case1" $ (Syntax.const "_pat" $ pat') $ rhs' end;
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   244
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   245
    fun Case2_tr' (_ $ (_ $ Const ("fatbar",_) $ m) $ ms) =
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   246
          Syntax.const "_Case2" $ Case1_tr' m $ Case2_tr' ms
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   247
    |   Case2_tr' t = Case1_tr' t;
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   248
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   249
    fun Case_syntax_tr' [Const ("run",_), _ $ ms $ x] =
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   250
          Syntax.const "_Case_syntax" $ x $ Case2_tr' ms;
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   251
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   252
  in [("Rep_CFun", Case_syntax_tr')] end;
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   253
*}
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   254
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   255
subsection {* Pattern combinators for built-in types *}
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   256
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   257
constdefs
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   258
  cpair_pat :: "('a, _, _) pat \<Rightarrow> ('b, _, _) pat \<Rightarrow> ('a \<times> 'b, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   259
  "cpair_pat p1 p2 \<equiv> \<Lambda> r1 \<langle>x1,x2\<rangle>. bind\<cdot>(p1\<cdot>r1\<cdot>x1)\<cdot>(\<Lambda> r2. p2\<cdot>r2\<cdot>x2)"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   260
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   261
  spair_pat :: "(_, _, _) pat \<Rightarrow> (_, _, _) pat \<Rightarrow> (_, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   262
  "spair_pat p1 p2 \<equiv> \<Lambda> r (:x,y:). cpair_pat p1 p2\<cdot>r\<cdot>\<langle>x,y\<rangle>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   263
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   264
  sinl_pat :: "(_, _, _) pat \<Rightarrow> (_, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   265
  "sinl_pat p \<equiv> \<Lambda> r a. case a of sinl\<cdot>x \<Rightarrow> p\<cdot>r\<cdot>x | sinr\<cdot>y \<Rightarrow> fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   266
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   267
  sinr_pat :: "(_, _, _) pat \<Rightarrow> (_, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   268
  "sinr_pat p \<equiv> \<Lambda> r a. case a of sinl\<cdot>x \<Rightarrow> fail | sinr\<cdot>y \<Rightarrow> p\<cdot>r\<cdot>y"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   269
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   270
  up_pat :: "('a, _, _) pat \<Rightarrow> ('a u, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   271
  "up_pat p \<equiv> \<Lambda> r a. case a of up\<cdot>x \<Rightarrow> p\<cdot>r\<cdot>x"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   272
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   273
  Def_pat :: "'a::type \<Rightarrow> ('a lift, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   274
  "Def_pat x \<equiv> \<Lambda> r. FLIFT y. if x = y then return\<cdot>r else fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   275
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   276
  ONE_pat :: "(one, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   277
  "ONE_pat \<equiv> \<Lambda> r ONE. return\<cdot>r"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   278
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   279
  TT_pat :: "(tr, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   280
  "TT_pat \<equiv> \<Lambda> r b. If b then return\<cdot>r else fail fi"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   281
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   282
  FF_pat :: "(tr, _, _) pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   283
  "FF_pat \<equiv> \<Lambda> r b. If b then fail else return\<cdot>r fi"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   284
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   285
text {* Parse translations *}
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   286
translations
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   287
  "_var (cpair\<cdot>p1\<cdot>p2)" => "cpair_pat (_var p1) (_var p2)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   288
  "_var (spair\<cdot>p1\<cdot>p2)" => "spair_pat (_var p1) (_var p2)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   289
  "_var (sinl\<cdot>p1)"     => "sinl_pat (_var p1)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   290
  "_var (sinr\<cdot>p1)"     => "sinr_pat (_var p1)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   291
  "_var (up\<cdot>p1)"       => "up_pat (_var p1)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   292
  "_var (Def x)"       => "Def_pat x"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   293
  "_var ONE"           => "ONE_pat"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   294
  "_var TT"            => "TT_pat"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   295
  "_var FF"            => "FF_pat"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   296
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   297
text {* Print translations *}
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   298
translations
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   299
  "cpair\<cdot>(_pat p1)\<cdot>(_pat p2)" <= "_pat (cpair_pat p1 p2)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   300
  "spair\<cdot>(_pat p1)\<cdot>(_pat p2)" <= "_pat (spair_pat p1 p2)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   301
  "sinl\<cdot>(_pat p1)"            <= "_pat (sinl_pat p1)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   302
  "sinr\<cdot>(_pat p1)"            <= "_pat (sinr_pat p1)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   303
  "up\<cdot>(_pat p1)"              <= "_pat (up_pat p1)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   304
  "Def x"                     <= "_pat (Def_pat x)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   305
  "TT"                        <= "_pat (TT_pat)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   306
  "FF"                        <= "_pat (FF_pat)"
18097
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   307
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   308
lemma cpair_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   309
  "p1\<cdot>r\<cdot>x = \<bottom> \<Longrightarrow> cpair_pat p1 p2\<cdot>r\<cdot><x,y> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   310
  "p1\<cdot>r\<cdot>x = fail \<Longrightarrow> cpair_pat p1 p2\<cdot>r\<cdot><x,y> = fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   311
  "p1\<cdot>r\<cdot>x = return\<cdot>r' \<Longrightarrow> cpair_pat p1 p2\<cdot>r\<cdot><x,y> = p2\<cdot>r'\<cdot>y"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   312
by (simp_all add: cpair_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   313
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   314
lemma spair_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   315
  "spair_pat p1 p2\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   316
  "\<lbrakk>x \<noteq> \<bottom>; y \<noteq> \<bottom>\<rbrakk> \<Longrightarrow> spair_pat p1 p2\<cdot>r\<cdot>(:x, y:) = cpair_pat p1 p2\<cdot>r\<cdot>\<langle>x, y\<rangle>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   317
by (simp_all add: spair_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   318
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   319
lemma sinl_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   320
  "sinl_pat p\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   321
  "x \<noteq> \<bottom> \<Longrightarrow> sinl_pat p\<cdot>r\<cdot>(sinl\<cdot>x) = p\<cdot>r\<cdot>x"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   322
  "x \<noteq> \<bottom> \<Longrightarrow> sinl_pat p\<cdot>r\<cdot>(sinr\<cdot>x) = fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   323
by (simp_all add: sinl_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   324
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   325
lemma sinr_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   326
  "sinr_pat p\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   327
  "x \<noteq> \<bottom> \<Longrightarrow> sinr_pat p\<cdot>r\<cdot>(sinl\<cdot>x) = fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   328
  "x \<noteq> \<bottom> \<Longrightarrow> sinr_pat p\<cdot>r\<cdot>(sinr\<cdot>x) = p\<cdot>r\<cdot>x"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   329
by (simp_all add: sinr_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   330
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   331
lemma up_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   332
  "up_pat p\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   333
  "up_pat p\<cdot>r\<cdot>(up\<cdot>x) = p\<cdot>r\<cdot>x"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   334
by (simp_all add: up_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   335
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   336
lemma Def_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   337
  "Def_pat x\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   338
  "Def_pat x\<cdot>r\<cdot>(Def x) = return\<cdot>r"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   339
  "x \<noteq> y \<Longrightarrow> Def_pat x\<cdot>r\<cdot>(Def y) = fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   340
by (simp_all add: Def_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   341
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   342
lemma ONE_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   343
  "ONE_pat\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   344
  "ONE_pat\<cdot>r\<cdot>ONE = return\<cdot>r"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   345
by (simp_all add: ONE_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   346
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   347
lemma TT_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   348
  "TT_pat\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   349
  "TT_pat\<cdot>r\<cdot>TT = return\<cdot>r"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   350
  "TT_pat\<cdot>r\<cdot>FF = fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   351
by (simp_all add: TT_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   352
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   353
lemma FF_pat_simps [simp]:
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   354
  "FF_pat\<cdot>r\<cdot>\<bottom> = \<bottom>"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   355
  "FF_pat\<cdot>r\<cdot>TT = fail"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   356
  "FF_pat\<cdot>r\<cdot>FF = return\<cdot>r"
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   357
by (simp_all add: FF_pat_def)
d196d84c306f add case syntax stuff
huffman
parents: 18096
diff changeset
   358
18112
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   359
subsection {* As-patterns *}
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   360
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   361
syntax
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   362
  "_as_pattern" :: "['a, 'a] \<Rightarrow> 'a" (* infixr "as" 10 *)
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   363
  (* TODO: choose a non-ambiguous syntax for as-patterns *)
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   364
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   365
constdefs
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   366
  as_pat :: "('a,'b,'c) pat \<Rightarrow> ('a,'c,'d) pat \<Rightarrow> ('a,'b,'d) pat"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   367
  "as_pat p1 p2 \<equiv> \<Lambda> r a. cpair_pat p1 p2\<cdot>r\<cdot>\<langle>a, a\<rangle>"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   368
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   369
translations
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   370
  "_var (_as_pattern p1 p2)" => "as_pat (_var p1) (_var p2)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   371
  "_as_pattern (_pat p1) (_pat p2)" <= "_pat (as_pat p1 p2)"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   372
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   373
lemma as_pat [simp]: "as_pat p1 p2\<cdot>r\<cdot>a = cpair_pat p1 p2\<cdot>r\<cdot>\<langle>a, a\<rangle>"
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   374
by (simp add: as_pat_def)
dc1d6f588204 reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
huffman
parents: 18110
diff changeset
   375
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   376
subsection {* Match functions for built-in types *}
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   377
16776
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   378
defaultsort pcpo
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   379
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   380
constdefs
16776
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   381
  match_UU :: "'a \<rightarrow> unit maybe"
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   382
  "match_UU \<equiv> \<Lambda> x. fail"
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   383
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   384
  match_cpair :: "'a::cpo \<times> 'b::cpo \<rightarrow> ('a \<times> 'b) maybe"
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   385
  "match_cpair \<equiv> csplit\<cdot>(\<Lambda> x y. return\<cdot><x,y>)"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   386
16551
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   387
  match_spair :: "'a \<otimes> 'b \<rightarrow> ('a \<times> 'b) maybe"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   388
  "match_spair \<equiv> ssplit\<cdot>(\<Lambda> x y. return\<cdot><x,y>)"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   389
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   390
  match_sinl :: "'a \<oplus> 'b \<rightarrow> 'a maybe"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   391
  "match_sinl \<equiv> sscase\<cdot>return\<cdot>(\<Lambda> y. fail)"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   392
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   393
  match_sinr :: "'a \<oplus> 'b \<rightarrow> 'b maybe"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   394
  "match_sinr \<equiv> sscase\<cdot>(\<Lambda> x. fail)\<cdot>return"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   395
16776
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   396
  match_up :: "'a::cpo u \<rightarrow> 'a maybe"
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   397
  "match_up \<equiv> fup\<cdot>return"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   398
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   399
  match_ONE :: "one \<rightarrow> unit maybe"
18094
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   400
  "match_ONE \<equiv> \<Lambda> ONE. return\<cdot>()"
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   401
 
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   402
  match_TT :: "tr \<rightarrow> unit maybe"
18094
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   403
  "match_TT \<equiv> \<Lambda> b. If b then return\<cdot>() else fail fi"
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   404
 
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   405
  match_FF :: "tr \<rightarrow> unit maybe"
18094
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   406
  "match_FF \<equiv> \<Lambda> b. If b then fail else return\<cdot>() fi"
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   407
16776
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   408
lemma match_UU_simps [simp]:
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   409
  "match_UU\<cdot>x = fail"
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   410
by (simp add: match_UU_def)
a3899ac14a1c generalized types of monadic operators to class cpo; added match function for UU
huffman
parents: 16758
diff changeset
   411
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   412
lemma match_cpair_simps [simp]:
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   413
  "match_cpair\<cdot><x,y> = return\<cdot><x,y>"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   414
by (simp add: match_cpair_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   415
16551
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   416
lemma match_spair_simps [simp]:
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   417
  "\<lbrakk>x \<noteq> \<bottom>; y \<noteq> \<bottom>\<rbrakk> \<Longrightarrow> match_spair\<cdot>(:x,y:) = return\<cdot><x,y>"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   418
  "match_spair\<cdot>\<bottom> = \<bottom>"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   419
by (simp_all add: match_spair_def)
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   420
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   421
lemma match_sinl_simps [simp]:
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   422
  "x \<noteq> \<bottom> \<Longrightarrow> match_sinl\<cdot>(sinl\<cdot>x) = return\<cdot>x"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   423
  "x \<noteq> \<bottom> \<Longrightarrow> match_sinl\<cdot>(sinr\<cdot>x) = fail"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   424
  "match_sinl\<cdot>\<bottom> = \<bottom>"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   425
by (simp_all add: match_sinl_def)
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   426
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   427
lemma match_sinr_simps [simp]:
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   428
  "x \<noteq> \<bottom> \<Longrightarrow> match_sinr\<cdot>(sinr\<cdot>x) = return\<cdot>x"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   429
  "x \<noteq> \<bottom> \<Longrightarrow> match_sinr\<cdot>(sinl\<cdot>x) = fail"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   430
  "match_sinr\<cdot>\<bottom> = \<bottom>"
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   431
by (simp_all add: match_sinr_def)
7abf8a713613 added match functions for spair, sinl, sinr
huffman
parents: 16463
diff changeset
   432
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   433
lemma match_up_simps [simp]:
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   434
  "match_up\<cdot>(up\<cdot>x) = return\<cdot>x"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   435
  "match_up\<cdot>\<bottom> = \<bottom>"
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   436
by (simp_all add: match_up_def)
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   437
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   438
lemma match_ONE_simps [simp]:
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   439
  "match_ONE\<cdot>ONE = return\<cdot>()"
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   440
  "match_ONE\<cdot>\<bottom> = \<bottom>"
18094
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   441
by (simp_all add: match_ONE_def)
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   442
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   443
lemma match_TT_simps [simp]:
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   444
  "match_TT\<cdot>TT = return\<cdot>()"
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   445
  "match_TT\<cdot>FF = fail"
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   446
  "match_TT\<cdot>\<bottom> = \<bottom>"
18094
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   447
by (simp_all add: match_TT_def)
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   448
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   449
lemma match_FF_simps [simp]:
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   450
  "match_FF\<cdot>FF = return\<cdot>()"
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   451
  "match_FF\<cdot>TT = fail"
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   452
  "match_FF\<cdot>\<bottom> = \<bottom>"
18094
404f298220af simplify definitions
huffman
parents: 16779
diff changeset
   453
by (simp_all add: match_FF_def)
16460
72a08d509d62 added match functions for ONE, TT, and FF; added theorem mplus_fail2
huffman
parents: 16417
diff changeset
   454
16401
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   455
subsection {* Mutual recursion *}
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   456
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   457
text {*
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   458
  The following rules are used to prove unfolding theorems from
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   459
  fixed-point definitions of mutually recursive functions.
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   460
*}
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   461
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   462
lemma cpair_equalI: "\<lbrakk>x \<equiv> cfst\<cdot>p; y \<equiv> csnd\<cdot>p\<rbrakk> \<Longrightarrow> <x,y> \<equiv> p"
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   463
by (simp add: surjective_pairing_Cprod2)
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   464
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   465
lemma cpair_eqD1: "<x,y> = <x',y'> \<Longrightarrow> x = x'"
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   466
by simp
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   467
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   468
lemma cpair_eqD2: "<x,y> = <x',y'> \<Longrightarrow> y = y'"
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   469
by simp
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   470
16463
342d74ca8815 fixrec shows unsolved subgoals when proofs of rewrites fail
huffman
parents: 16460
diff changeset
   471
text {* lemma for proving rewrite rules *}
342d74ca8815 fixrec shows unsolved subgoals when proofs of rewrites fail
huffman
parents: 16460
diff changeset
   472
342d74ca8815 fixrec shows unsolved subgoals when proofs of rewrites fail
huffman
parents: 16460
diff changeset
   473
lemma ssubst_lhs: "\<lbrakk>t = s; P s = Q\<rbrakk> \<Longrightarrow> P t = Q"
342d74ca8815 fixrec shows unsolved subgoals when proofs of rewrites fail
huffman
parents: 16460
diff changeset
   474
by simp
342d74ca8815 fixrec shows unsolved subgoals when proofs of rewrites fail
huffman
parents: 16460
diff changeset
   475
16401
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   476
ML {*
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   477
val cpair_equalI = thm "cpair_equalI";
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   478
val cpair_eqD1 = thm "cpair_eqD1";
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   479
val cpair_eqD2 = thm "cpair_eqD2";
16463
342d74ca8815 fixrec shows unsolved subgoals when proofs of rewrites fail
huffman
parents: 16460
diff changeset
   480
val ssubst_lhs = thm "ssubst_lhs";
16401
57c35ede00b9 fixrec package now handles mutually-recursive definitions
huffman
parents: 16229
diff changeset
   481
*}
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   482
16758
c32334d98fcd fix typo
huffman
parents: 16754
diff changeset
   483
subsection {* Initializing the fixrec package *}
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   484
16229
77cae9c8e73e use fixrec_package.ML
huffman
parents: 16221
diff changeset
   485
use "fixrec_package.ML"
16221
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   486
879400e029bf New theory with lemmas for the fixrec package
huffman
parents:
diff changeset
   487
end