src/HOL/Library/Product_Order.thy
changeset 60580 7e741e22d7fc
parent 60500 903bb1495239
child 60679 ade12ef2773c
--- a/src/HOL/Library/Product_Order.thy	Thu Jun 25 22:56:33 2015 +0200
+++ b/src/HOL/Library/Product_Order.thy	Thu Jun 25 23:33:47 2015 +0200
@@ -233,11 +233,13 @@
 
 instance prod ::
   (complete_distrib_lattice, complete_distrib_lattice) complete_distrib_lattice
-proof
-  case goal1 thus ?case
+proof (default, goals)
+  case 1
+  then show ?case
     by (auto simp: sup_prod_def Inf_prod_def INF_prod_alt_def sup_Inf sup_INF comp_def)
 next
-  case goal2 thus ?case
+  case 2
+  then show ?case
     by (auto simp: inf_prod_def Sup_prod_def SUP_prod_alt_def inf_Sup inf_SUP comp_def)
 qed