src/HOL/AxClasses/Lattice/LatPreInsts.ML
changeset 5069 3ea049f7979d
parent 4153 e534c4c32d54
child 5711 5a1cd4b4b20e
--- a/src/HOL/AxClasses/Lattice/LatPreInsts.ML	Mon Jun 22 17:13:09 1998 +0200
+++ b/src/HOL/AxClasses/Lattice/LatPreInsts.ML	Mon Jun 22 17:26:46 1998 +0200
@@ -4,12 +4,12 @@
 
 (** complete lattices **)
 
-goal thy "is_inf x y (Inf {x, y})";
+Goal "is_inf x y (Inf {x, y})";
   by (rtac (bin_is_Inf_eq RS subst) 1);
   by (rtac Inf_is_Inf 1);
 qed "Inf_is_inf";
 
-goal thy "is_sup x y (Sup {x, y})";
+Goal "is_sup x y (Sup {x, y})";
   by (rtac (bin_is_Sup_eq RS subst) 1);
   by (rtac Sup_is_Sup 1);
 qed "Sup_is_sup";
@@ -20,13 +20,13 @@
 
 (* pairs *)
 
-goalw thy [is_inf_def, le_prod_def] "is_inf p q (fst p && fst q, snd p && snd q)";
+Goalw [is_inf_def, le_prod_def] "is_inf p q (fst p && fst q, snd p && snd q)";
   by (Simp_tac 1);
   by Safe_tac;
   by (REPEAT_FIRST (fn i => resolve_tac [inf_lb1, inf_lb2, inf_ub_lbs] i ORELSE atac i));
 qed "prod_is_inf";
 
-goalw thy [is_sup_def, le_prod_def] "is_sup p q (fst p || fst q, snd p || snd q)";
+Goalw [is_sup_def, le_prod_def] "is_sup p q (fst p || fst q, snd p || snd q)";
   by (Simp_tac 1);
   by Safe_tac;
   by (REPEAT_FIRST (fn i => resolve_tac [sup_ub1, sup_ub2, sup_lb_ubs] i ORELSE atac i));
@@ -35,7 +35,7 @@
 
 (* functions *)
 
-goalw thy [is_inf_def, le_fun_def] "is_inf f g (%x. f x && g x)";
+Goalw [is_inf_def, le_fun_def] "is_inf f g (%x. f x && g x)";
   by Safe_tac;
   by (rtac inf_lb1 1);
   by (rtac inf_lb2 1);
@@ -43,7 +43,7 @@
   by (REPEAT_FIRST (Fast_tac));
 qed "fun_is_inf";
 
-goalw thy [is_sup_def, le_fun_def] "is_sup f g (%x. f x || g x)";
+Goalw [is_sup_def, le_fun_def] "is_sup f g (%x. f x || g x)";
   by Safe_tac;
   by (rtac sup_ub1 1);
   by (rtac sup_ub2 1);
@@ -55,7 +55,7 @@
 
 (** dual lattices **)
 
-goalw thy [is_inf_def, le_dual_def] "is_inf x y (Abs_dual (Rep_dual x || Rep_dual y))";
+Goalw [is_inf_def, le_dual_def] "is_inf x y (Abs_dual (Rep_dual x || Rep_dual y))";
   by (stac Abs_dual_inverse' 1);
   by Safe_tac;
   by (rtac sup_ub1 1);
@@ -65,7 +65,7 @@
   by (assume_tac 1);
 qed "dual_is_inf";
 
-goalw thy [is_sup_def, le_dual_def] "is_sup x y (Abs_dual (Rep_dual x && Rep_dual y))";
+Goalw [is_sup_def, le_dual_def] "is_sup x y (Abs_dual (Rep_dual x && Rep_dual y))";
   by (stac Abs_dual_inverse' 1);
   by Safe_tac;
   by (rtac inf_lb1 1);