src/HOL/AxClasses/Lattice/LatPreInsts.ML
author clasohm
Tue, 12 Mar 1996 14:39:34 +0100
changeset 1573 6d66b59f94a9
parent 1440 de6f18da81bb
child 1899 0075a8d26a80
permissions -rw-r--r--
added constdefs section
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1440
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     1
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     2
open LatPreInsts;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     3
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     4
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     5
(** complete lattices **)
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     6
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     7
goal thy "is_inf x y (Inf {x, y})";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     8
  br (bin_is_Inf_eq RS subst) 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
     9
  br Inf_is_Inf 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    10
qed "Inf_is_inf";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    11
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    12
goal thy "is_sup x y (Sup {x, y})";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    13
  br (bin_is_Sup_eq RS subst) 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    14
  br Sup_is_Sup 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    15
qed "Sup_is_sup";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    16
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    17
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    18
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    19
(** product lattices **)
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    20
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    21
(* pairs *)
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    22
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    23
goalw thy [is_inf_def, le_prod_def] "is_inf p q (fst p && fst q, snd p && snd q)";
1573
6d66b59f94a9 added constdefs section
clasohm
parents: 1440
diff changeset
    24
  by (Simp_tac 1);
1440
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    25
  by (safe_tac HOL_cs);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    26
  by (REPEAT_FIRST (fn i => resolve_tac [inf_lb1, inf_lb2, inf_ub_lbs] i ORELSE atac i));
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    27
qed "prod_is_inf";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    28
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    29
goalw thy [is_sup_def, le_prod_def] "is_sup p q (fst p || fst q, snd p || snd q)";
1573
6d66b59f94a9 added constdefs section
clasohm
parents: 1440
diff changeset
    30
  by (Simp_tac 1);
1440
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    31
  by (safe_tac HOL_cs);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    32
  by (REPEAT_FIRST (fn i => resolve_tac [sup_ub1, sup_ub2, sup_lb_ubs] i ORELSE atac i));
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    33
qed "prod_is_sup";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    34
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    35
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    36
(* functions *)
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    37
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    38
goalw thy [is_inf_def, le_fun_def] "is_inf f g (%x. f x && g x)";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    39
  by (safe_tac HOL_cs);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    40
  br inf_lb1 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    41
  br inf_lb2 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    42
  br inf_ub_lbs 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    43
  by (REPEAT_FIRST (fast_tac HOL_cs));
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    44
qed "fun_is_inf";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    45
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    46
goalw thy [is_sup_def, le_fun_def] "is_sup f g (%x. f x || g x)";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    47
  by (safe_tac HOL_cs);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    48
  br sup_ub1 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    49
  br sup_ub2 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    50
  br sup_lb_ubs 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    51
  by (REPEAT_FIRST (fast_tac HOL_cs));
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    52
qed "fun_is_sup";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    53
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    54
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    55
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    56
(** dual lattices **)
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    57
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    58
goalw thy [is_inf_def, le_dual_def] "is_inf x y (Abs_dual (Rep_dual x || Rep_dual y))";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    59
  by (stac Abs_dual_inverse' 1);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    60
  by (safe_tac HOL_cs);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    61
  br sup_ub1 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    62
  br sup_ub2 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    63
  br sup_lb_ubs 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    64
  ba 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    65
  ba 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    66
qed "dual_is_inf";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    67
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    68
goalw thy [is_sup_def, le_dual_def] "is_sup x y (Abs_dual (Rep_dual x && Rep_dual y))";
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    69
  by (stac Abs_dual_inverse' 1);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    70
  by (safe_tac HOL_cs);
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    71
  br inf_lb1 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    72
  br inf_lb2 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    73
  br inf_ub_lbs 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    74
  ba 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    75
  ba 1;
de6f18da81bb added this stuff;
wenzelm
parents:
diff changeset
    76
qed "dual_is_sup";