src/HOL/ex/ReflectionEx.thy
author wenzelm
Sat, 27 Nov 2010 15:36:35 +0100
changeset 40744 0e7c2957fc1d
parent 39246 9e58f0499f57
child 41413 64cd30d6b0b8
permissions -rw-r--r--
tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
29650
cc3958d31b1d Reflection.thy now in HOL/Library
haftmann
parents: 28866
diff changeset
     1
(*  Title:      HOL/ex/ReflectionEx.thy
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
     2
    Author:     Amine Chaieb, TU Muenchen
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
     3
*)
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
     4
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
     5
header {* Examples for generic reflection and reification *}
29650
cc3958d31b1d Reflection.thy now in HOL/Library
haftmann
parents: 28866
diff changeset
     6
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
     7
theory ReflectionEx
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
     8
imports Reflection
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
     9
begin
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    10
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    11
text{* This theory presents two methods: reify and reflection *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    12
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    13
text{* 
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
    14
Consider an HOL type 'a, the structure of which is not recongnisable on the theory level. This is the case of bool, arithmetical terms such as int, real etc \dots
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    15
In order to implement a simplification on terms of type 'a we often need its structure.
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    16
Traditionnaly such simplifications are written in ML, proofs are synthesized.
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    17
An other strategy is to declare an HOL-datatype tau and an HOL function (the interpretation) that maps elements of tau to elements of 'a. The functionality of @{text reify} is to compute a term s::tau, which is the representant of t. For this it needs equations for the interpretation.
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    18
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    19
NB: All the interpretations supported by @{text reify} must have the type @{text "'b list \<Rightarrow> tau \<Rightarrow> 'a"}.
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    20
The method @{text reify} can also be told which subterm of the current subgoal should be reified. The general call for @{text reify} is: @{text "reify eqs (t)"}, where @{text eqs} are the defining equations of the interpretation and @{text "(t)"} is an optional parameter which specifies the subterm to which reification should be applied to. If @{text "(t)"} is abscent, @{text reify} tries to reify the whole subgoal.
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    21
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    22
The method reflection uses @{text reify} and has a very similar signature: @{text "reflection corr_thm eqs (t)"}. Here again @{text eqs} and @{text "(t)"} are as described above and @{text corr_thm} is a thorem proving @{term "I vs (f t) = I vs t"}. We assume that @{text I} is the interpretation and @{text f} is some useful and executable simplification of type @{text "tau \<Rightarrow> tau"}. The method @{text reflection} applies reification and hence the theorem @{term "t = I xs s"} and hence using @{text corr_thm} derives @{term "t = I xs (f s)"}. It then uses normalization by evaluation to prove @{term "f s = s'"} which almost finishes the proof of @{term "t = t'"} where @{term "I xs s' = t'"}.
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    23
*}
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    24
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    25
text{* Example 1 : Propositional formulae and NNF.*}
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    26
text{* The type @{text fm} represents simple propositional formulae: *}
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    27
23547
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    28
datatype form = TrueF | FalseF | Less nat nat |
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    29
                And form form | Or form form | Neg form | ExQ form
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    30
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    31
fun interp :: "form \<Rightarrow> ('a::ord) list \<Rightarrow> bool" where
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    32
"interp TrueF e = True" |
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    33
"interp FalseF e = False" |
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    34
"interp (Less i j) e = (e!i < e!j)" |
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    35
"interp (And f1 f2) e = (interp f1 e & interp f2 e)" |
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    36
"interp (Or f1 f2) e = (interp f1 e | interp f2 e)" |
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    37
"interp (Neg f) e = (~ interp f e)" |
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    38
"interp (ExQ f) e = (EX x. interp f (x#e))"
23547
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    39
23608
e65e36dbe0d2 Some examples for reifying type variables
chaieb
parents: 23547
diff changeset
    40
lemmas interp_reify_eqs = interp.simps
e65e36dbe0d2 Some examples for reifying type variables
chaieb
parents: 23547
diff changeset
    41
declare interp_reify_eqs[reify]
23547
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    42
23608
e65e36dbe0d2 Some examples for reifying type variables
chaieb
parents: 23547
diff changeset
    43
lemma "EX x. x < y & x < z"
e65e36dbe0d2 Some examples for reifying type variables
chaieb
parents: 23547
diff changeset
    44
  apply (reify )
e65e36dbe0d2 Some examples for reifying type variables
chaieb
parents: 23547
diff changeset
    45
  oops
23547
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    46
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    47
datatype fm = And fm fm | Or fm fm | Imp fm fm | Iff fm fm | NOT fm | At nat
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    48
39246
9e58f0499f57 modernized primrec
haftmann
parents: 35419
diff changeset
    49
primrec Ifm :: "fm \<Rightarrow> bool list \<Rightarrow> bool" where
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
    50
  "Ifm (At n) vs = vs!n"
39246
9e58f0499f57 modernized primrec
haftmann
parents: 35419
diff changeset
    51
| "Ifm (And p q) vs = (Ifm p vs \<and> Ifm q vs)"
9e58f0499f57 modernized primrec
haftmann
parents: 35419
diff changeset
    52
| "Ifm (Or p q) vs = (Ifm p vs \<or> Ifm q vs)"
9e58f0499f57 modernized primrec
haftmann
parents: 35419
diff changeset
    53
| "Ifm (Imp p q) vs = (Ifm p vs \<longrightarrow> Ifm q vs)"
9e58f0499f57 modernized primrec
haftmann
parents: 35419
diff changeset
    54
| "Ifm (Iff p q) vs = (Ifm p vs = Ifm q vs)"
9e58f0499f57 modernized primrec
haftmann
parents: 35419
diff changeset
    55
| "Ifm (NOT p) vs = (\<not> (Ifm p vs))"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    56
23547
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    57
lemma "Q \<longrightarrow> (D & F & ((~ D) & (~ F)))"
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    58
apply (reify Ifm.simps)
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    59
oops
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    60
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    61
  text{* Method @{text reify} maps a bool to an fm. For this it needs the 
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    62
  semantics of fm, i.e.\ the rewrite rules in @{text Ifm.simps}. *}
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    63
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    64
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    65
  (* You can also just pick up a subterm to reify \<dots> *)
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    66
lemma "Q \<longrightarrow> (D & F & ((~ D) & (~ F)))"
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    67
apply (reify Ifm.simps ("((~ D) & (~ F))"))
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    68
oops
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    69
cb1203d8897c More examples
chaieb
parents: 23477
diff changeset
    70
  text{* Let's perform NNF. This is a version that tends to generate disjunctions *}
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    71
primrec fmsize :: "fm \<Rightarrow> nat" where
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    72
  "fmsize (At n) = 1"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    73
| "fmsize (NOT p) = 1 + fmsize p"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    74
| "fmsize (And p q) = 1 + fmsize p + fmsize q"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    75
| "fmsize (Or p q) = 1 + fmsize p + fmsize q"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    76
| "fmsize (Imp p q) = 2 + fmsize p + fmsize q"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    77
| "fmsize (Iff p q) = 2 + 2* fmsize p + 2* fmsize q"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    78
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    79
lemma [measure_function]: "is_measure fmsize" ..
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    80
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    81
fun nnf :: "fm \<Rightarrow> fm"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    82
where
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    83
  "nnf (At n) = At n"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    84
| "nnf (And p q) = And (nnf p) (nnf q)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    85
| "nnf (Or p q) = Or (nnf p) (nnf q)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    86
| "nnf (Imp p q) = Or (nnf (NOT p)) (nnf q)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    87
| "nnf (Iff p q) = Or (And (nnf p) (nnf q)) (And (nnf (NOT p)) (nnf (NOT q)))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    88
| "nnf (NOT (And p q)) = Or (nnf (NOT p)) (nnf (NOT q))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    89
| "nnf (NOT (Or p q)) = And (nnf (NOT p)) (nnf (NOT q))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    90
| "nnf (NOT (Imp p q)) = And (nnf p) (nnf (NOT q))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    91
| "nnf (NOT (Iff p q)) = Or (And (nnf p) (nnf (NOT q))) (And (nnf (NOT p)) (nnf q))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    92
| "nnf (NOT (NOT p)) = nnf p"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
    93
| "nnf (NOT p) = NOT p"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    94
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    95
  text{* The correctness theorem of nnf: it preserves the semantics of fm *}
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
    96
lemma nnf[reflection]: "Ifm (nnf p) vs = Ifm p vs"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    97
  by (induct p rule: nnf.induct) auto
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
    98
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
    99
  text{* Now let's perform NNF using our @{term nnf} function defined above. First to the whole subgoal. *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   100
lemma "(\<not> (A = B)) \<and> (B \<longrightarrow> (A \<noteq> (B | C \<and> (B \<longrightarrow> A | D)))) \<longrightarrow> A \<or> B \<and> D"
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   101
apply (reflection Ifm.simps)
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   102
oops
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   103
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   104
  text{* Now we specify on which subterm it should be applied*}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   105
lemma "(\<not> (A = B)) \<and> (B \<longrightarrow> (A \<noteq> (B | C \<and> (B \<longrightarrow> A | D)))) \<longrightarrow> A \<or> B \<and> D"
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   106
apply (reflection Ifm.simps only: "(B | C \<and> (B \<longrightarrow> A | D))")
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   107
oops
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   108
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   109
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   110
  (* Example 2 : Simple arithmetic formulae *)
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   111
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   112
  text{* The type @{text num} reflects linear expressions over natural number *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   113
datatype num = C nat | Add num num | Mul nat num | Var nat | CN nat nat num
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   114
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   115
text{* This is just technical to make recursive definitions easier. *}
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   116
primrec num_size :: "num \<Rightarrow> nat" 
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   117
where
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   118
  "num_size (C c) = 1"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   119
| "num_size (Var n) = 1"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   120
| "num_size (Add a b) = 1 + num_size a + num_size b"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   121
| "num_size (Mul c a) = 1 + num_size a"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   122
| "num_size (CN n c a) = 4 + num_size a "
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   123
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   124
  text{* The semantics of num *}
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   125
primrec Inum:: "num \<Rightarrow> nat list \<Rightarrow> nat"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   126
where
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   127
  Inum_C  : "Inum (C i) vs = i"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   128
| Inum_Var: "Inum (Var n) vs = vs!n"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   129
| Inum_Add: "Inum (Add s t) vs = Inum s vs + Inum t vs "
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   130
| Inum_Mul: "Inum (Mul c t) vs = c * Inum t vs "
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   131
| Inum_CN : "Inum (CN n c t) vs = c*(vs!n) + Inum t vs "
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   132
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   133
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   134
  text{* Let's reify some nat expressions \dots *}
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   135
lemma "4 * (2*x + (y::nat)) + f a \<noteq> 0"
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   136
  apply (reify Inum.simps ("4 * (2*x + (y::nat)) + f a"))
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   137
oops
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   138
text{* We're in a bad situation!! x, y and f a have been recongnized as a constants, which is correct but does not correspond to our intuition of the constructor C. It should encapsulate constants, i.e. numbers, i.e. numerals.*}
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   139
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   140
  text{* So let's leave the @{text "Inum_C"} equation at the end and see what happens \dots*}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   141
lemma "4 * (2*x + (y::nat)) \<noteq> 0"
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   142
  apply (reify Inum_Var Inum_Add Inum_Mul Inum_CN Inum_C ("4 * (2*x + (y::nat))"))
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   143
oops
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   144
text{* Hmmm let's specialize @{text Inum_C} with numerals.*}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   145
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   146
lemma Inum_number: "Inum (C (number_of t)) vs = number_of t" by simp
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   147
lemmas Inum_eqs = Inum_Var Inum_Add Inum_Mul Inum_CN Inum_number
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   148
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   149
  text{* Second attempt *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   150
lemma "1 * (2*x + (y::nat)) \<noteq> 0"
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   151
  apply (reify Inum_eqs ("1 * (2*x + (y::nat))"))
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   152
oops
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   153
  text{* That was fine, so let's try another one \dots *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   154
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   155
lemma "1 * (2* x + (y::nat) + 0 + 1) \<noteq> 0"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   156
  apply (reify Inum_eqs ("1 * (2*x + (y::nat) + 0 + 1)"))
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   157
oops
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   158
  text{* Oh!! 0 is not a variable \dots\ Oh! 0 is not a @{text "number_of"} \dots\ thing. The same for 1. So let's add those equations too *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   159
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   160
lemma Inum_01: "Inum (C 0) vs = 0" "Inum (C 1) vs = 1" "Inum (C(Suc n)) vs = Suc n"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   161
  by simp+
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   162
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   163
lemmas Inum_eqs'= Inum_eqs Inum_01
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   164
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   165
text{* Third attempt: *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   166
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   167
lemma "1 * (2*x + (y::nat) + 0 + 1) \<noteq> 0"
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   168
  apply (reify Inum_eqs' ("1 * (2*x + (y::nat) + 0 + 1)"))
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   169
oops
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   170
text{* Okay, let's try reflection. Some simplifications on num follow. You can skim until the main theorem @{text linum} *}
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   171
fun lin_add :: "num \<Rightarrow> num \<Rightarrow> num"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   172
where
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   173
  "lin_add (CN n1 c1 r1) (CN n2 c2 r2) =
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   174
  (if n1=n2 then 
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   175
  (let c = c1 + c2
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   176
  in (if c=0 then lin_add r1 r2 else CN n1 c (lin_add r1 r2)))
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   177
  else if n1 \<le> n2 then (CN n1 c1 (lin_add r1 (CN n2 c2 r2))) 
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   178
  else (CN n2 c2 (lin_add (CN n1 c1 r1) r2)))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   179
| "lin_add (CN n1 c1 r1) t = CN n1 c1 (lin_add r1 t)"  
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   180
| "lin_add t (CN n2 c2 r2) = CN n2 c2 (lin_add t r2)" 
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   181
| "lin_add (C b1) (C b2) = C (b1+b2)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   182
| "lin_add a b = Add a b"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   183
lemma lin_add: "Inum (lin_add t s) bs = Inum (Add t s) bs"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   184
apply (induct t s rule: lin_add.induct, simp_all add: Let_def)
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   185
apply (case_tac "c1+c2 = 0",case_tac "n1 \<le> n2", simp_all)
29667
53103fc8ffa3 Replaced group_ and ring_simps by algebra_simps;
nipkow
parents: 28866
diff changeset
   186
by (case_tac "n1 = n2", simp_all add: algebra_simps)
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   187
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   188
fun lin_mul :: "num \<Rightarrow> nat \<Rightarrow> num"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   189
where
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   190
  "lin_mul (C j) i = C (i*j)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   191
| "lin_mul (CN n c a) i = (if i=0 then (C 0) else CN n (i*c) (lin_mul a i))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   192
| "lin_mul t i = (Mul i t)"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   193
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   194
lemma lin_mul: "Inum (lin_mul t i) bs = Inum (Mul i t) bs"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   195
by (induct t i rule: lin_mul.induct, auto simp add: algebra_simps)
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   196
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   197
lemma [measure_function]: "is_measure num_size" ..
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   198
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   199
fun linum:: "num \<Rightarrow> num"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   200
where
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   201
  "linum (C b) = C b"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   202
| "linum (Var n) = CN n 1 (C 0)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   203
| "linum (Add t s) = lin_add (linum t) (linum s)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   204
| "linum (Mul c t) = lin_mul (linum t) c"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   205
| "linum (CN n c t) = lin_add (linum (Mul c (Var n))) (linum t)"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   206
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   207
lemma linum[reflection] : "Inum (linum t) bs = Inum t bs"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   208
by (induct t rule: linum.induct, simp_all add: lin_mul lin_add)
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   209
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   210
  text{* Now we can use linum to simplify nat terms using reflection *}
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   211
lemma "(Suc (Suc 1)) * (x + (Suc 1)*y) = 3*x + 6*y"
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   212
 apply (reflection Inum_eqs' only: "(Suc (Suc 1)) * (x + (Suc 1)*y)") 
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   213
oops
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   214
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   215
  text{* Let's lift this to formulae and see what happens *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   216
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   217
datatype aform = Lt num num  | Eq num num | Ge num num | NEq num num | 
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   218
  Conj aform aform | Disj aform aform | NEG aform | T | F
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   219
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   220
primrec linaformsize:: "aform \<Rightarrow> nat"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   221
where
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   222
  "linaformsize T = 1"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   223
| "linaformsize F = 1"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   224
| "linaformsize (Lt a b) = 1"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   225
| "linaformsize (Ge a b) = 1"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   226
| "linaformsize (Eq a b) = 1"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   227
| "linaformsize (NEq a b) = 1"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   228
| "linaformsize (NEG p) = 2 + linaformsize p"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   229
| "linaformsize (Conj p q) = 1 + linaformsize p + linaformsize q"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   230
| "linaformsize (Disj p q) = 1 + linaformsize p + linaformsize q"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   231
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   232
lemma [measure_function]: "is_measure linaformsize" ..
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   233
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   234
primrec is_aform :: "aform => nat list => bool"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   235
where
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   236
  "is_aform T vs = True"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   237
| "is_aform F vs = False"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   238
| "is_aform (Lt a b) vs = (Inum a vs < Inum b vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   239
| "is_aform (Eq a b) vs = (Inum a vs = Inum b vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   240
| "is_aform (Ge a b) vs = (Inum a vs \<ge> Inum b vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   241
| "is_aform (NEq a b) vs = (Inum a vs \<noteq> Inum b vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   242
| "is_aform (NEG p) vs = (\<not> (is_aform p vs))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   243
| "is_aform (Conj p q) vs = (is_aform p vs \<and> is_aform q vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   244
| "is_aform (Disj p q) vs = (is_aform p vs \<or> is_aform q vs)"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   245
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   246
  text{* Let's reify and do reflection *}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   247
lemma "(3::nat)*x + t < 0 \<and> (2 * x + y \<noteq> 17)"
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   248
 apply (reify Inum_eqs' is_aform.simps) 
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   249
oops
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   250
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   251
text{* Note that reification handles several interpretations at the same time*}
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   252
lemma "(3::nat)*x + t < 0 & x*x + t*x + 3 + 1 = z*t*4*z | x + x + 1 < 0"
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   253
 apply (reflection Inum_eqs' is_aform.simps only:"x + x + 1") 
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   254
oops
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   255
20337
36e2fae2c68a *** empty log message ***
chaieb
parents: 20319
diff changeset
   256
  text{* For reflection we now define a simple transformation on aform: NNF + linum on atoms *}
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   257
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   258
fun linaform:: "aform \<Rightarrow> aform"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   259
where
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   260
  "linaform (Lt s t) = Lt (linum s) (linum t)"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   261
| "linaform (Eq s t) = Eq (linum s) (linum t)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   262
| "linaform (Ge s t) = Ge (linum s) (linum t)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   263
| "linaform (NEq s t) = NEq (linum s) (linum t)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   264
| "linaform (Conj p q) = Conj (linaform p) (linaform q)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   265
| "linaform (Disj p q) = Disj (linaform p) (linaform q)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   266
| "linaform (NEG T) = F"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   267
| "linaform (NEG F) = T"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   268
| "linaform (NEG (Lt a b)) = Ge a b"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   269
| "linaform (NEG (Ge a b)) = Lt a b"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   270
| "linaform (NEG (Eq a b)) = NEq a b"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   271
| "linaform (NEG (NEq a b)) = Eq a b"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   272
| "linaform (NEG (NEG p)) = linaform p"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   273
| "linaform (NEG (Conj p q)) = Disj (linaform (NEG p)) (linaform (NEG q))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   274
| "linaform (NEG (Disj p q)) = Conj (linaform (NEG p)) (linaform (NEG q))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   275
| "linaform p = p"
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   276
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   277
lemma linaform: "is_aform (linaform p) vs = is_aform p vs"
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   278
  by (induct p rule: linaform.induct) (auto simp add: linum)
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   279
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   280
lemma "(((Suc(Suc (Suc 0)))*((x::nat) + (Suc (Suc 0)))) + (Suc (Suc (Suc 0))) * ((Suc(Suc (Suc 0)))*((x::nat) + (Suc (Suc 0))))< 0) \<and> (Suc 0  + Suc 0< 0)"
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   281
   apply (reflection Inum_eqs' is_aform.simps rules: linaform)  
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   282
oops
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   283
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   284
declare linaform[reflection]
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   285
lemma "(((Suc(Suc (Suc 0)))*((x::nat) + (Suc (Suc 0)))) + (Suc (Suc (Suc 0))) * ((Suc(Suc (Suc 0)))*((x::nat) + (Suc (Suc 0))))< 0) \<and> (Suc 0  + Suc 0< 0)"
28866
30cd9d89a0fb reactivated some dead theories (based on hints by Mark Hillebrand);
wenzelm
parents: 23650
diff changeset
   286
   apply (reflection Inum_eqs' is_aform.simps)
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   287
oops
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   288
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   289
text{* We now give an example where Interpretaions have 0 or more than only one envornement of different types and show that automatic reification also deals with binding *}
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   290
datatype rb = BC bool| BAnd rb rb | BOr rb rb
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   291
primrec Irb :: "rb \<Rightarrow> bool"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   292
where
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   293
  "Irb (BC p) = p"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   294
| "Irb (BAnd s t) = (Irb s \<and> Irb t)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   295
| "Irb (BOr s t) = (Irb s \<or> Irb t)"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   296
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   297
lemma "A \<and> (B \<or> D \<and> B) \<and> A \<and> (B \<or> D \<and> B) \<or> A \<and> (B \<or> D \<and> B) \<or> A \<and> (B \<or> D \<and> B)"
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   298
apply (reify Irb.simps)
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   299
oops
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   300
23650
0a6a719d24d5 Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb
parents: 23624
diff changeset
   301
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   302
datatype rint = IC int| IVar nat | IAdd rint rint | IMult rint rint | INeg rint | ISub rint rint
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   303
primrec Irint :: "rint \<Rightarrow> int list \<Rightarrow> int"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   304
where
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   305
  Irint_Var: "Irint (IVar n) vs = vs!n"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   306
| Irint_Neg: "Irint (INeg t) vs = - Irint t vs"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   307
| Irint_Add: "Irint (IAdd s t) vs = Irint s vs + Irint t vs"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   308
| Irint_Sub: "Irint (ISub s t) vs = Irint s vs - Irint t vs"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   309
| Irint_Mult: "Irint (IMult s t) vs = Irint s vs * Irint t vs"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   310
| Irint_C: "Irint (IC i) vs = i"
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   311
lemma Irint_C0: "Irint (IC 0) vs = 0"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   312
  by simp
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   313
lemma Irint_C1: "Irint (IC 1) vs = 1"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   314
  by simp
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   315
lemma Irint_Cnumberof: "Irint (IC (number_of x)) vs = number_of x"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   316
  by simp
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   317
lemmas Irint_simps = Irint_Var Irint_Neg Irint_Add Irint_Sub Irint_Mult Irint_C0 Irint_C1 Irint_Cnumberof 
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   318
lemma "(3::int) * x + y*y - 9 + (- z) = 0"
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   319
  apply (reify Irint_simps ("(3::int) * x + y*y - 9 + (- z)"))
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   320
  oops
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   321
datatype rlist = LVar nat| LEmpty| LCons rint rlist | LAppend rlist rlist
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   322
primrec Irlist :: "rlist \<Rightarrow> int list \<Rightarrow> (int list) list \<Rightarrow> (int list)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   323
where
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   324
  "Irlist (LEmpty) is vs = []"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   325
| "Irlist (LVar n) is vs = vs!n"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   326
| "Irlist (LCons i t) is vs = ((Irint i is)#(Irlist t is vs))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   327
| "Irlist (LAppend s t) is vs = (Irlist s is vs) @ (Irlist t is vs)"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   328
lemma "[(1::int)] = []"
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   329
  apply (reify Irlist.simps Irint_simps ("[1]:: int list"))
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   330
  oops
20374
01b711328990 Reification now handels binders.
chaieb
parents: 20337
diff changeset
   331
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   332
lemma "([(3::int) * x + y*y - 9 + (- z)] @ []) @ xs = [y*y - z - 9 + (3::int) * x]"
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   333
  apply (reify Irlist.simps Irint_simps ("([(3::int) * x + y*y - 9 + (- z)] @ []) @ xs"))
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   334
  oops
20374
01b711328990 Reification now handels binders.
chaieb
parents: 20337
diff changeset
   335
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   336
datatype rnat = NC nat| NVar nat| NSuc rnat | NAdd rnat rnat | NMult rnat rnat | NNeg rnat | NSub rnat rnat | Nlgth rlist
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   337
primrec Irnat :: "rnat \<Rightarrow> int list \<Rightarrow> (int list) list \<Rightarrow> nat list \<Rightarrow> nat"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   338
where
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   339
  Irnat_Suc: "Irnat (NSuc t) is ls vs = Suc (Irnat t is ls vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   340
| Irnat_Var: "Irnat (NVar n) is ls vs = vs!n"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   341
| Irnat_Neg: "Irnat (NNeg t) is ls vs = 0"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   342
| Irnat_Add: "Irnat (NAdd s t) is ls vs = Irnat s is ls vs + Irnat t is ls vs"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   343
| Irnat_Sub: "Irnat (NSub s t) is ls vs = Irnat s is ls vs - Irnat t is ls vs"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   344
| Irnat_Mult: "Irnat (NMult s t) is ls vs = Irnat s is ls vs * Irnat t is ls vs"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   345
| Irnat_lgth: "Irnat (Nlgth rxs) is ls vs = length (Irlist rxs is ls)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   346
| Irnat_C: "Irnat (NC i) is ls vs = i"
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   347
lemma Irnat_C0: "Irnat (NC 0) is ls vs = 0"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   348
by simp
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   349
lemma Irnat_C1: "Irnat (NC 1) is ls vs = 1"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   350
by simp
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   351
lemma Irnat_Cnumberof: "Irnat (NC (number_of x)) is ls vs = number_of x"
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   352
by simp
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   353
lemmas Irnat_simps = Irnat_Suc Irnat_Var Irnat_Neg Irnat_Add Irnat_Sub Irnat_Mult Irnat_lgth
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   354
  Irnat_C0 Irnat_C1 Irnat_Cnumberof
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   355
lemma "(Suc n) * length (([(3::int) * x + y*y - 9 + (- z)] @ []) @ xs) = length xs"
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   356
  apply (reify Irnat_simps Irlist.simps Irint_simps ("(Suc n) *length (([(3::int) * x + y*y - 9 + (- z)] @ []) @ xs)"))
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   357
  oops
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   358
datatype rifm = RT | RF | RVar nat
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   359
  | RNLT rnat rnat | RNILT rnat rint | RNEQ rnat rnat
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   360
  |RAnd rifm rifm | ROr rifm rifm | RImp rifm rifm| RIff rifm rifm
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   361
  | RNEX rifm | RIEX rifm| RLEX rifm | RNALL rifm | RIALL rifm| RLALL rifm
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   362
  | RBEX rifm | RBALL rifm
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   363
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   364
primrec Irifm :: "rifm \<Rightarrow> bool list \<Rightarrow> int list \<Rightarrow> (int list) list \<Rightarrow> nat list \<Rightarrow> bool"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   365
where
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   366
  "Irifm RT ps is ls ns = True"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   367
| "Irifm RF ps is ls ns = False"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   368
| "Irifm (RVar n) ps is ls ns = ps!n"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   369
| "Irifm (RNLT s t) ps is ls ns = (Irnat s is ls ns < Irnat t is ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   370
| "Irifm (RNILT s t) ps is ls ns = (int (Irnat s is ls ns) < Irint t is)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   371
| "Irifm (RNEQ s t) ps is ls ns = (Irnat s is ls ns = Irnat t is ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   372
| "Irifm (RAnd p q) ps is ls ns = (Irifm p ps is ls ns \<and> Irifm q ps is ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   373
| "Irifm (ROr p q) ps is ls ns = (Irifm p ps is ls ns \<or> Irifm q ps is ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   374
| "Irifm (RImp p q) ps is ls ns = (Irifm p ps is ls ns \<longrightarrow> Irifm q ps is ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   375
| "Irifm (RIff p q) ps is ls ns = (Irifm p ps is ls ns = Irifm q ps is ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   376
| "Irifm (RNEX p) ps is ls ns =  (\<exists>x. Irifm p ps is ls (x#ns))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   377
| "Irifm (RIEX p) ps is ls ns =  (\<exists>x. Irifm p ps (x#is) ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   378
| "Irifm (RLEX p) ps is ls ns =  (\<exists>x. Irifm p ps is (x#ls) ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   379
| "Irifm (RBEX p) ps is ls ns =  (\<exists>x. Irifm p (x#ps) is ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   380
| "Irifm (RNALL p) ps is ls ns = (\<forall>x. Irifm p ps is ls (x#ns))"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   381
| "Irifm (RIALL p) ps is ls ns = (\<forall>x. Irifm p ps (x#is) ls ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   382
| "Irifm (RLALL p) ps is ls ns = (\<forall>x. Irifm p ps is (x#ls) ns)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   383
| "Irifm (RBALL p) ps is ls ns = (\<forall>x. Irifm p (x#ps) is ls ns)"
20374
01b711328990 Reification now handels binders.
chaieb
parents: 20337
diff changeset
   384
20564
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   385
lemma " \<forall>x. \<exists>n. ((Suc n) * length (([(3::int) * x + (f t)*y - 9 + (- z)] @ []) @ xs) = length xs) \<and> m < 5*n - length (xs @ [2,3,4,x*z + 8 - y]) \<longrightarrow> (\<exists>p. \<forall>q. p \<and> q \<longrightarrow> r)"
6857bd9f1a79 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents: 20503
diff changeset
   386
  apply (reify Irifm.simps Irnat_simps Irlist.simps Irint_simps)
20374
01b711328990 Reification now handels binders.
chaieb
parents: 20337
diff changeset
   387
oops
01b711328990 Reification now handels binders.
chaieb
parents: 20337
diff changeset
   388
22199
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   389
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 31021
diff changeset
   390
(* An example for equations containing type variables *)
22199
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   391
datatype prod = Zero | One | Var nat | Mul prod prod 
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   392
  | Pw prod nat | PNM nat nat prod
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   393
primrec Iprod :: " prod \<Rightarrow> ('a::{linordered_idom}) list \<Rightarrow>'a" 
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   394
where
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   395
  "Iprod Zero vs = 0"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   396
| "Iprod One vs = 1"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   397
| "Iprod (Var n) vs = vs!n"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   398
| "Iprod (Mul a b) vs = (Iprod a vs * Iprod b vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   399
| "Iprod (Pw a n) vs = ((Iprod a vs) ^ n)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   400
| "Iprod (PNM n k t) vs = (vs ! n)^k * Iprod t vs"
39246
9e58f0499f57 modernized primrec
haftmann
parents: 35419
diff changeset
   401
22199
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   402
datatype sgn = Pos prod | Neg prod | ZeroEq prod | NZeroEq prod | Tr | F 
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   403
  | Or sgn sgn | And sgn sgn
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   404
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   405
primrec Isgn :: " sgn \<Rightarrow> ('a::{linordered_idom}) list \<Rightarrow>bool"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   406
where 
23624
82091387f6d7 The order for parameter for interpretation is now inversted:
chaieb
parents: 23608
diff changeset
   407
  "Isgn Tr vs = True"
35419
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   408
| "Isgn F vs = False"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   409
| "Isgn (ZeroEq t) vs = (Iprod t vs = 0)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   410
| "Isgn (NZeroEq t) vs = (Iprod t vs \<noteq> 0)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   411
| "Isgn (Pos t) vs = (Iprod t vs > 0)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   412
| "Isgn (Neg t) vs = (Iprod t vs < 0)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   413
| "Isgn (And p q) vs = (Isgn p vs \<and> Isgn q vs)"
d78659d1723e more recdef (and old primrec) hunting
krauss
parents: 35028
diff changeset
   414
| "Isgn (Or p q) vs = (Isgn p vs \<or> Isgn q vs)"
22199
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   415
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   416
lemmas eqs = Isgn.simps Iprod.simps
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   417
35028
108662d50512 more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
haftmann
parents: 32960
diff changeset
   418
lemma "(x::'a::{linordered_idom})^4 * y * z * y^2 * z^23 > 0"
22199
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   419
  apply (reify eqs)
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   420
  oops
b617ddd200eb Now deals with simples cases where the input equations contain type variables
chaieb
parents: 20564
diff changeset
   421
20319
a8761e8568de Generic reflection and reification (by Amine Chaieb).
wenzelm
parents:
diff changeset
   422
end