src/HOL/Library/Product_Order.thy
changeset 61166 5976fe402824
parent 60679 ade12ef2773c
child 62053 1c8252d07e32
--- a/src/HOL/Library/Product_Order.thy	Sun Sep 13 16:50:12 2015 +0200
+++ b/src/HOL/Library/Product_Order.thy	Sun Sep 13 20:20:16 2015 +0200
@@ -233,7 +233,7 @@
 (* Contribution: Alessandro Coglio *)
 
 instance prod :: (complete_distrib_lattice, complete_distrib_lattice) complete_distrib_lattice
-proof (standard, goals)
+proof (standard, goal_cases)
   case 1
   then show ?case
     by (auto simp: sup_prod_def Inf_prod_def INF_prod_alt_def sup_Inf sup_INF comp_def)