src/HOL/HOLCF/IOA/ABP/Lemmas.thy
author huffman
Sat, 27 Nov 2010 16:08:10 -0800
changeset 40774 0437dbc127b3
parent 35174 src/HOLCF/IOA/ABP/Lemmas.thy@e15040ae75d7
child 40945 b8703f63bfb2
permissions -rw-r--r--
moved directory src/HOLCF to src/HOL/HOLCF; added HOLCF theories to src/HOL/IsaMakefile;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
3072
a31419014be5 Old ABP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff changeset
     1
(*  Title:      HOLCF/IOA/ABP/Lemmas.thy
12218
wenzelm
parents: 10215
diff changeset
     2
    Author:     Olaf Müller
3072
a31419014be5 Old ABP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff changeset
     3
*)
a31419014be5 Old ABP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff changeset
     4
17244
0b2ff9541727 converted to Isar theory format;
wenzelm
parents: 14981
diff changeset
     5
theory Lemmas
0b2ff9541727 converted to Isar theory format;
wenzelm
parents: 14981
diff changeset
     6
imports Main
0b2ff9541727 converted to Isar theory format;
wenzelm
parents: 14981
diff changeset
     7
begin
0b2ff9541727 converted to Isar theory format;
wenzelm
parents: 14981
diff changeset
     8
19738
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
     9
subsection {* Logic *}
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    10
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    11
lemma and_de_morgan_and_absorbe: "(~(A&B)) = ((~A)&B| ~B)"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    12
  by blast
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    13
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    14
lemma bool_if_impl_or: "(if C then A else B) --> (A|B)"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    15
  by auto
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    16
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    17
lemma exis_elim: "(? x. x=P & Q(x)) = Q(P)"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    18
  by blast
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    19
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    20
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    21
subsection {* Sets *}
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    22
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    23
lemma set_lemmas:
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    24
    "f(x) : (UN x. {f(x)})"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    25
    "f x y : (UN x y. {f x y})"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    26
    "!!a. (!x. a ~= f(x)) ==> a ~: (UN x. {f(x)})"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    27
    "!!a. (!x y. a ~= f x y) ==> a ~: (UN x y. {f x y})"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    28
  by auto
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    29
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    30
text {* 2 Lemmas to add to @{text "set_lemmas"}, used also for action handling, 
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    31
   namely for Intersections and the empty list (compatibility of IOA!). *}
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    32
lemma singleton_set: "(UN b.{x. x=f(b)})= (UN b.{f(b)})"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    33
  by blast
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    34
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    35
lemma de_morgan: "((A|B)=False) = ((~A)&(~B))"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    36
  by blast
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    37
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    38
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    39
subsection {* Lists *}
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    40
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    41
lemma cons_not_nil: "l ~= [] --> (? x xs. l = (x#xs))"
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    42
  by (induct l) simp_all
1ac610922636 removed legacy ML scripts;
wenzelm
parents: 17244
diff changeset
    43
17244
0b2ff9541727 converted to Isar theory format;
wenzelm
parents: 14981
diff changeset
    44
end