src/HOL/AxClasses/Tutorial/Xor.ML
changeset 1247 18b1441fb603
child 1899 0075a8d26a80
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/AxClasses/Tutorial/Xor.ML	Fri Sep 01 14:27:36 1995 +0200
@@ -0,0 +1,14 @@
+(*  Title:      HOL/AxClasses/Tutorial/Xor.ML
+    ID:         $Id$
+    Author:     Markus Wenzel, TU Muenchen
+
+Proof the instantiation theorem bool :: agroup by hand.
+*)
+
+open AxClass;
+
+goal_arity Xor.thy ("bool", [], "agroup");
+by (axclass_tac Xor.thy []);
+by (rewrite_goals_tac [Xor.prod_bool_def, Xor.inv_bool_def, Xor.unit_bool_def]);
+by (ALLGOALS (fast_tac HOL_cs));
+qed "bool_in_agroup";