src/HOL/Induct/Sexp.thy
author wenzelm
Fri, 17 Nov 2006 02:20:03 +0100
changeset 21404 eb85850d3eb7
parent 20820 58693343905f
child 23746 a455e69c31cc
permissions -rw-r--r--
more robust syntax for definition/abbreviation/notation;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
8840
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     1
(*  Title:      HOL/Induct/Sexp.thy
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     2
    ID:         $Id$
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     4
    Copyright   1992  University of Cambridge
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     5
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     6
S-expressions, general binary trees for defining recursive data
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     7
structures by hand.
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     8
*)
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
     9
20801
d3616b4abe1b proper import of Main HOL;
wenzelm
parents: 19736
diff changeset
    10
theory Sexp imports Main begin
d3616b4abe1b proper import of Main HOL;
wenzelm
parents: 19736
diff changeset
    11
d3616b4abe1b proper import of Main HOL;
wenzelm
parents: 19736
diff changeset
    12
types
20820
58693343905f removed obsolete Datatype_Universe.thy (cf. Datatype.thy);
wenzelm
parents: 20801
diff changeset
    13
  'a item = "'a Datatype.item"
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 20820
diff changeset
    14
abbreviation "Leaf == Datatype.Leaf"
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 20820
diff changeset
    15
abbreviation "Numb == Datatype.Numb"
20801
d3616b4abe1b proper import of Main HOL;
wenzelm
parents: 19736
diff changeset
    16
8840
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
    17
consts
13079
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    18
  sexp      :: "'a item set"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    19
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    20
inductive sexp
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    21
  intros
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    22
    LeafI:  "Leaf(a) \<in> sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    23
    NumbI:  "Numb(i) \<in> sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    24
    SconsI: "[| M \<in> sexp;  N \<in> sexp |] ==> Scons M N \<in> sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    25
19736
wenzelm
parents: 18413
diff changeset
    26
definition
8840
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
    27
  sexp_case :: "['a=>'b, nat=>'b, ['a item, 'a item]=>'b, 
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 20820
diff changeset
    28
                'a item] => 'b" where
20801
d3616b4abe1b proper import of Main HOL;
wenzelm
parents: 19736
diff changeset
    29
  "sexp_case c d e M = (THE z. (EX x.   M=Leaf(x) & z=c(x))  
d3616b4abe1b proper import of Main HOL;
wenzelm
parents: 19736
diff changeset
    30
                             | (EX k.   M=Numb(k) & z=d(k))  
d3616b4abe1b proper import of Main HOL;
wenzelm
parents: 19736
diff changeset
    31
                             | (EX N1 N2. M = Scons N1 N2  & z=e N1 N2))"
8840
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
    32
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 20820
diff changeset
    33
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 20820
diff changeset
    34
  pred_sexp :: "('a item * 'a item)set" where
19736
wenzelm
parents: 18413
diff changeset
    35
     "pred_sexp = (\<Union>M \<in> sexp. \<Union>N \<in> sexp. {(M, Scons M N), (N, Scons M N)})"
8840
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
    36
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 20820
diff changeset
    37
definition
13079
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    38
  sexp_rec  :: "['a item, 'a=>'b, nat=>'b,      
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 20820
diff changeset
    39
                ['a item, 'a item, 'b, 'b]=>'b] => 'b" where
19736
wenzelm
parents: 18413
diff changeset
    40
   "sexp_rec M c d e = wfrec pred_sexp
8840
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
    41
             (%g. sexp_case c d (%N1 N2. e N1 N2 (g N1) (g N2))) M"
13079
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    42
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    43
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    44
(** sexp_case **)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    45
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    46
lemma sexp_case_Leaf [simp]: "sexp_case c d e (Leaf a) = c(a)"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    47
by (simp add: sexp_case_def, blast)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    48
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    49
lemma sexp_case_Numb [simp]: "sexp_case c d e (Numb k) = d(k)"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    50
by (simp add: sexp_case_def, blast)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    51
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    52
lemma sexp_case_Scons [simp]: "sexp_case c d e (Scons M N) = e M N"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    53
by (simp add: sexp_case_def)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    54
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    55
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    56
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    57
(** Introduction rules for sexp constructors **)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    58
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    59
lemma sexp_In0I: "M \<in> sexp ==> In0(M) \<in> sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    60
apply (simp add: In0_def) 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    61
apply (erule sexp.NumbI [THEN sexp.SconsI])
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    62
done
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    63
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    64
lemma sexp_In1I: "M \<in> sexp ==> In1(M) \<in> sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    65
apply (simp add: In1_def) 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    66
apply (erule sexp.NumbI [THEN sexp.SconsI])
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    67
done
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    68
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    69
declare sexp.intros [intro,simp]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    70
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    71
lemma range_Leaf_subset_sexp: "range(Leaf) <= sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    72
by blast
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    73
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    74
lemma Scons_D: "Scons M N \<in> sexp ==> M \<in> sexp & N \<in> sexp"
18413
50c0c118e96d removed obsolete/unused setup_induction;
wenzelm
parents: 16417
diff changeset
    75
  by (induct S == "Scons M N" set: sexp) auto
13079
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    76
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    77
(** Introduction rules for 'pred_sexp' **)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    78
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    79
lemma pred_sexp_subset_Sigma: "pred_sexp <= sexp <*> sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    80
by (simp add: pred_sexp_def, blast)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    81
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    82
(* (a,b) \<in> pred_sexp^+ ==> a \<in> sexp *)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    83
lemmas trancl_pred_sexpD1 = 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    84
    pred_sexp_subset_Sigma
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    85
	 [THEN trancl_subset_Sigma, THEN subsetD, THEN SigmaD1]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    86
and trancl_pred_sexpD2 = 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    87
    pred_sexp_subset_Sigma
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    88
	 [THEN trancl_subset_Sigma, THEN subsetD, THEN SigmaD2]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    89
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    90
lemma pred_sexpI1: 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    91
    "[| M \<in> sexp;  N \<in> sexp |] ==> (M, Scons M N) \<in> pred_sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    92
by (simp add: pred_sexp_def, blast)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    93
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    94
lemma pred_sexpI2: 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    95
    "[| M \<in> sexp;  N \<in> sexp |] ==> (N, Scons M N) \<in> pred_sexp"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    96
by (simp add: pred_sexp_def, blast)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    97
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    98
(*Combinations involving transitivity and the rules above*)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
    99
lemmas pred_sexp_t1 [simp] = pred_sexpI1 [THEN r_into_trancl]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   100
and    pred_sexp_t2 [simp] = pred_sexpI2 [THEN r_into_trancl]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   101
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   102
lemmas pred_sexp_trans1 [simp] = trans_trancl [THEN transD, OF _ pred_sexp_t1]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   103
and    pred_sexp_trans2 [simp] = trans_trancl [THEN transD, OF _ pred_sexp_t2]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   104
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   105
(*Proves goals of the form (M,N):pred_sexp^+ provided M,N:sexp*)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   106
declare cut_apply [simp] 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   107
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   108
lemma pred_sexpE:
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   109
    "[| p \<in> pred_sexp;                                        
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   110
        !!M N. [| p = (M, Scons M N);  M \<in> sexp;  N \<in> sexp |] ==> R;  
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   111
        !!M N. [| p = (N, Scons M N);  M \<in> sexp;  N \<in> sexp |] ==> R   
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   112
     |] ==> R"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   113
by (simp add: pred_sexp_def, blast) 
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   114
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   115
lemma wf_pred_sexp: "wf(pred_sexp)"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   116
apply (rule pred_sexp_subset_Sigma [THEN wfI])
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   117
apply (erule sexp.induct)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   118
apply (blast elim!: pred_sexpE)+
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   119
done
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   120
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   121
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   122
(*** sexp_rec -- by wf recursion on pred_sexp ***)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   123
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   124
lemma sexp_rec_unfold_lemma:
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   125
     "(%M. sexp_rec M c d e) ==
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   126
      wfrec pred_sexp (%g. sexp_case c d (%N1 N2. e N1 N2 (g N1) (g N2)))"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   127
by (simp add: sexp_rec_def)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   128
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   129
lemmas sexp_rec_unfold = def_wfrec [OF sexp_rec_unfold_lemma wf_pred_sexp]
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   130
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   131
(* sexp_rec a c d e =
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   132
   sexp_case c d
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   133
    (%N1 N2.
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   134
        e N1 N2 (cut (%M. sexp_rec M c d e) pred_sexp a N1)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   135
         (cut (%M. sexp_rec M c d e) pred_sexp a N2)) a
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   136
*)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   137
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   138
(** conversion rules **)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   139
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   140
lemma sexp_rec_Leaf: "sexp_rec (Leaf a) c d h = c(a)"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   141
apply (subst sexp_rec_unfold)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   142
apply (rule sexp_case_Leaf)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   143
done
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   144
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   145
lemma sexp_rec_Numb: "sexp_rec (Numb k) c d h = d(k)"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   146
apply (subst sexp_rec_unfold)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   147
apply (rule sexp_case_Numb)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   148
done
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   149
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   150
lemma sexp_rec_Scons: "[| M \<in> sexp;  N \<in> sexp |] ==>  
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   151
     sexp_rec (Scons M N) c d h = h M N (sexp_rec M c d h) (sexp_rec N c d h)"
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   152
apply (rule sexp_rec_unfold [THEN trans])
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   153
apply (simp add: pred_sexpI1 pred_sexpI2)
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   154
done
e7738aa7267f conversion of Induct/{Slist,Sexp} to Isar scripts
paulson
parents: 11481
diff changeset
   155
8840
18b76c137c41 moved theory Sexp to Induct examples;
wenzelm
parents:
diff changeset
   156
end